| Metamath
Proof Explorer Theorem List (p. 368 of 497) | < Previous Next > | |
| Bad symbols? Try the
GIF version. |
||
|
Mirrors > Metamath Home Page > MPE Home Page > Theorem List Contents > Recent Proofs This page: Page List |
||
| Color key: | (1-30845) |
(30846-32368) |
(32369-49617) |
| Type | Label | Description |
|---|---|---|
| Statement | ||
| Theorem | bj-dfnnf2 36701 | Alternate definition of df-bj-nnf 36688 using only primitive symbols (→, ¬, ∀) in each conjunct. (Contributed by BJ, 20-Aug-2023.) |
| ⊢ (Ⅎ'𝑥𝜑 ↔ ((𝜑 → ∀𝑥𝜑) ∧ (¬ 𝜑 → ∀𝑥 ¬ 𝜑))) | ||
| Theorem | bj-nnfnfTEMP 36702 | New nonfreeness implies old nonfreeness on minimal implicational calculus (the proof indicates it uses ax-3 8 because of set.mm's definition of the biconditional, but the proof actually holds in minimal implicational calculus). (Contributed by BJ, 28-Jul-2023.) The proof should not rely on df-nf 1784 except via df-nf 1784 directly. (Proof modification is discouraged.) |
| ⊢ (Ⅎ'𝑥𝜑 → Ⅎ𝑥𝜑) | ||
| Theorem | bj-wnfnf 36703 | When 𝜑 is substituted for 𝜓, this statement expresses nonfreeness in the weak form of nonfreeness (∃ → ∀). Note that this could also be proved from bj-nnfim 36710, bj-nnfe1 36724 and bj-nnfa1 36723. (Contributed by BJ, 9-Dec-2023.) |
| ⊢ Ⅎ'𝑥(∃𝑥𝜑 → ∀𝑥𝜓) | ||
| Theorem | bj-nnfnt 36704 | A variable is nonfree in a formula if and only if it is nonfree in its negation. The foward implication is intuitionistically valid (and that direction is sufficient for the purpose of recursively proving that some formulas have a given variable not free in them, like bj-nnfim 36710). Intuitionistically, ⊢ (Ⅎ'𝑥¬ 𝜑 ↔ Ⅎ'𝑥¬ ¬ 𝜑). See nfnt 1856. (Contributed by BJ, 28-Jul-2023.) |
| ⊢ (Ⅎ'𝑥𝜑 ↔ Ⅎ'𝑥 ¬ 𝜑) | ||
| Theorem | bj-nnftht 36705 | A variable is nonfree in a theorem. The antecedent is in the "strong necessity" modality of modal logic in order not to require sp 2183 (modal T), as in bj-nnfbi 36689. (Contributed by BJ, 28-Jul-2023.) |
| ⊢ ((𝜑 ∧ ∀𝑥𝜑) → Ⅎ'𝑥𝜑) | ||
| Theorem | bj-nnfth 36706 | A variable is nonfree in a theorem, inference form. (Contributed by BJ, 28-Jul-2023.) |
| ⊢ 𝜑 ⇒ ⊢ Ⅎ'𝑥𝜑 | ||
| Theorem | bj-nnfnth 36707 | A variable is nonfree in the negation of a theorem, inference form. (Contributed by BJ, 27-Aug-2023.) |
| ⊢ ¬ 𝜑 ⇒ ⊢ Ⅎ'𝑥𝜑 | ||
| Theorem | bj-nnfim1 36708 | A consequence of nonfreeness in the antecedent and the consequent of an implication. (Contributed by BJ, 27-Aug-2023.) |
| ⊢ ((Ⅎ'𝑥𝜑 ∧ Ⅎ'𝑥𝜓) → ((𝜑 → 𝜓) → (∃𝑥𝜑 → ∀𝑥𝜓))) | ||
| Theorem | bj-nnfim2 36709 | A consequence of nonfreeness in the antecedent and the consequent of an implication. (Contributed by BJ, 27-Aug-2023.) |
| ⊢ ((Ⅎ'𝑥𝜑 ∧ Ⅎ'𝑥𝜓) → ((∀𝑥𝜑 → ∃𝑥𝜓) → (𝜑 → 𝜓))) | ||
| Theorem | bj-nnfim 36710 | Nonfreeness in the antecedent and the consequent of an implication implies nonfreeness in the implication. (Contributed by BJ, 27-Aug-2023.) |
| ⊢ ((Ⅎ'𝑥𝜑 ∧ Ⅎ'𝑥𝜓) → Ⅎ'𝑥(𝜑 → 𝜓)) | ||
| Theorem | bj-nnfimd 36711 | Nonfreeness in the antecedent and the consequent of an implication implies nonfreeness in the implication, deduction form. (Contributed by BJ, 2-Dec-2023.) |
| ⊢ (𝜑 → Ⅎ'𝑥𝜓) & ⊢ (𝜑 → Ⅎ'𝑥𝜒) ⇒ ⊢ (𝜑 → Ⅎ'𝑥(𝜓 → 𝜒)) | ||
| Theorem | bj-nnfan 36712 | Nonfreeness in both conjuncts implies nonfreeness in the conjunction. (Contributed by BJ, 19-Nov-2023.) In classical logic, there is a proof using the definition of conjunction in terms of implication and negation, so using bj-nnfim 36710, bj-nnfnt 36704 and bj-nnfbi 36689, but we want a proof valid in intuitionistic logic. (Proof modification is discouraged.) |
| ⊢ ((Ⅎ'𝑥𝜑 ∧ Ⅎ'𝑥𝜓) → Ⅎ'𝑥(𝜑 ∧ 𝜓)) | ||
| Theorem | bj-nnfand 36713 | Nonfreeness in both conjuncts implies nonfreeness in the conjunction, deduction form. Note: compared with the proof of bj-nnfan 36712, it has two more essential steps but fewer total steps (since there are fewer intermediate formulas to build) and is easier to follow and understand. This statement is of intermediate complexity: for simpler statements, closed-style proofs like that of bj-nnfan 36712 will generally be shorter than deduction-style proofs while still easy to follow, while for more complex statements, the opposite will be true (and deduction-style proofs like that of bj-nnfand 36713 will generally be easier to understand). (Contributed by BJ, 19-Nov-2023.) (Proof modification is discouraged.) |
| ⊢ (𝜑 → Ⅎ'𝑥𝜓) & ⊢ (𝜑 → Ⅎ'𝑥𝜒) ⇒ ⊢ (𝜑 → Ⅎ'𝑥(𝜓 ∧ 𝜒)) | ||
| Theorem | bj-nnfor 36714 | Nonfreeness in both disjuncts implies nonfreeness in the disjunction. (Contributed by BJ, 19-Nov-2023.) In classical logic, there is a proof using the definition of disjunction in terms of implication and negation, so using bj-nnfim 36710, bj-nnfnt 36704 and bj-nnfbi 36689, but we want a proof valid in intuitionistic logic. (Proof modification is discouraged.) |
| ⊢ ((Ⅎ'𝑥𝜑 ∧ Ⅎ'𝑥𝜓) → Ⅎ'𝑥(𝜑 ∨ 𝜓)) | ||
| Theorem | bj-nnford 36715 | Nonfreeness in both disjuncts implies nonfreeness in the disjunction, deduction form. See comments for bj-nnfor 36714 and bj-nnfand 36713. (Contributed by BJ, 2-Dec-2023.) (Proof modification is discouraged.) |
| ⊢ (𝜑 → Ⅎ'𝑥𝜓) & ⊢ (𝜑 → Ⅎ'𝑥𝜒) ⇒ ⊢ (𝜑 → Ⅎ'𝑥(𝜓 ∨ 𝜒)) | ||
| Theorem | bj-nnfbit 36716 | Nonfreeness in both sides implies nonfreeness in the biconditional. (Contributed by BJ, 2-Dec-2023.) (Proof modification is discouraged.) |
| ⊢ ((Ⅎ'𝑥𝜑 ∧ Ⅎ'𝑥𝜓) → Ⅎ'𝑥(𝜑 ↔ 𝜓)) | ||
| Theorem | bj-nnfbid 36717 | Nonfreeness in both sides implies nonfreeness in the biconditional, deduction form. (Contributed by BJ, 2-Dec-2023.) (Proof modification is discouraged.) |
| ⊢ (𝜑 → Ⅎ'𝑥𝜓) & ⊢ (𝜑 → Ⅎ'𝑥𝜒) ⇒ ⊢ (𝜑 → Ⅎ'𝑥(𝜓 ↔ 𝜒)) | ||
| Theorem | bj-nnfv 36718* | A non-occurring variable is nonfree in a formula. (Contributed by BJ, 28-Jul-2023.) |
| ⊢ Ⅎ'𝑥𝜑 | ||
| Theorem | bj-nnf-alrim 36719 | Proof of the closed form of alrimi 2213 from modalK (compare alrimiv 1927). See also bj-alrim 36657. Actually, most proofs between 19.3t 2201 and 2sbbid 2247 could be proved without ax-12 2177. (Contributed by BJ, 20-Aug-2023.) |
| ⊢ (Ⅎ'𝑥𝜑 → (∀𝑥(𝜑 → 𝜓) → (𝜑 → ∀𝑥𝜓))) | ||
| Theorem | bj-nnf-exlim 36720 | Proof of the closed form of exlimi 2217 from modalK (compare exlimiv 1930). See also bj-sylget2 36586. (Contributed by BJ, 2-Dec-2023.) |
| ⊢ (Ⅎ'𝑥𝜓 → (∀𝑥(𝜑 → 𝜓) → (∃𝑥𝜑 → 𝜓))) | ||
| Theorem | bj-dfnnf3 36721 | Alternate definition of nonfreeness when sp 2183 is available. (Contributed by BJ, 28-Jul-2023.) The proof should not rely on df-nf 1784. (Proof modification is discouraged.) |
| ⊢ (Ⅎ'𝑥𝜑 ↔ (∃𝑥𝜑 → ∀𝑥𝜑)) | ||
| Theorem | bj-nfnnfTEMP 36722 | New nonfreeness is equivalent to old nonfreeness on core FOL axioms plus sp 2183. (Contributed by BJ, 28-Jul-2023.) The proof should not rely on df-nf 1784 except via df-nf 1784 directly. (Proof modification is discouraged.) |
| ⊢ (Ⅎ'𝑥𝜑 ↔ Ⅎ𝑥𝜑) | ||
| Theorem | bj-nnfa1 36723 | See nfa1 2151. (Contributed by BJ, 12-Aug-2023.) (Proof modification is discouraged.) |
| ⊢ Ⅎ'𝑥∀𝑥𝜑 | ||
| Theorem | bj-nnfe1 36724 | See nfe1 2150. (Contributed by BJ, 12-Aug-2023.) (Proof modification is discouraged.) |
| ⊢ Ⅎ'𝑥∃𝑥𝜑 | ||
| Theorem | bj-19.12 36725 | See 19.12 2327. Could be labeled "exalimalex" for "'there exists for all' implies 'for all there exists'". This proof is from excom 2162 and modal (B) on top of modalK logic. (Contributed by BJ, 12-Aug-2023.) The proof should not rely on df-nf 1784 or df-bj-nnf 36688, directly or indirectly. (Proof modification is discouraged.) |
| ⊢ (∃𝑥∀𝑦𝜑 → ∀𝑦∃𝑥𝜑) | ||
| Theorem | bj-nnflemaa 36726 | One of four lemmas for nonfreeness: antecedent and consequent both expressed using universal quantifier. Note: this is bj-hbalt 36645. (Contributed by BJ, 12-Aug-2023.) (Proof modification is discouraged.) |
| ⊢ (∀𝑥(𝜑 → ∀𝑦𝜑) → (∀𝑥𝜑 → ∀𝑦∀𝑥𝜑)) | ||
| Theorem | bj-nnflemee 36727 | One of four lemmas for nonfreeness: antecedent and consequent both expressed using existential quantifier. (Contributed by BJ, 12-Aug-2023.) (Proof modification is discouraged.) |
| ⊢ (∀𝑥(∃𝑦𝜑 → 𝜑) → (∃𝑦∃𝑥𝜑 → ∃𝑥𝜑)) | ||
| Theorem | bj-nnflemae 36728 | One of four lemmas for nonfreeness: antecedent expressed with universal quantifier and consequent expressed with existential quantifier. (Contributed by BJ, 12-Aug-2023.) (Proof modification is discouraged.) |
| ⊢ (∀𝑥(𝜑 → ∀𝑦𝜑) → (∃𝑥𝜑 → ∀𝑦∃𝑥𝜑)) | ||
| Theorem | bj-nnflemea 36729 | One of four lemmas for nonfreeness: antecedent expressed with existential quantifier and consequent expressed with universal quantifier. (Contributed by BJ, 12-Aug-2023.) (Proof modification is discouraged.) |
| ⊢ (∀𝑥(∃𝑦𝜑 → 𝜑) → (∃𝑦∀𝑥𝜑 → ∀𝑥𝜑)) | ||
| Theorem | bj-nnfalt 36730 | See nfal 2323 and bj-nfalt 36675. (Contributed by BJ, 12-Aug-2023.) (Proof modification is discouraged.) |
| ⊢ (∀𝑥Ⅎ'𝑦𝜑 → Ⅎ'𝑦∀𝑥𝜑) | ||
| Theorem | bj-nnfext 36731 | See nfex 2324 and bj-nfext 36676. (Contributed by BJ, 12-Aug-2023.) (Proof modification is discouraged.) |
| ⊢ (∀𝑥Ⅎ'𝑦𝜑 → Ⅎ'𝑦∃𝑥𝜑) | ||
| Theorem | bj-stdpc5t 36732 | Alias of bj-nnf-alrim 36719 for labeling consistency (a standard predicate calculus axiom). Closed form of stdpc5 2208 proved from modalK (obsoleting stdpc5v 1938). (Contributed by BJ, 2-Dec-2023.) Use bj-nnf-alrim 36719 instead. (New usaged is discouraged.) |
| ⊢ (Ⅎ'𝑥𝜑 → (∀𝑥(𝜑 → 𝜓) → (𝜑 → ∀𝑥𝜓))) | ||
| Theorem | bj-19.21t 36733 | Statement 19.21t 2206 proved from modalK (obsoleting 19.21v 1939). (Contributed by BJ, 2-Dec-2023.) |
| ⊢ (Ⅎ'𝑥𝜑 → (∀𝑥(𝜑 → 𝜓) ↔ (𝜑 → ∀𝑥𝜓))) | ||
| Theorem | bj-19.23t 36734 | Statement 19.23t 2210 proved from modalK (obsoleting 19.23v 1942). (Contributed by BJ, 2-Dec-2023.) |
| ⊢ (Ⅎ'𝑥𝜓 → (∀𝑥(𝜑 → 𝜓) ↔ (∃𝑥𝜑 → 𝜓))) | ||
| Theorem | bj-19.36im 36735 | One direction of 19.36 2230 from the same axioms as 19.36imv 1945. (Contributed by BJ, 2-Dec-2023.) |
| ⊢ (Ⅎ'𝑥𝜓 → (∃𝑥(𝜑 → 𝜓) → (∀𝑥𝜑 → 𝜓))) | ||
| Theorem | bj-19.37im 36736 | One direction of 19.37 2232 from the same axioms as 19.37imv 1947. (Contributed by BJ, 2-Dec-2023.) |
| ⊢ (Ⅎ'𝑥𝜑 → (∃𝑥(𝜑 → 𝜓) → (𝜑 → ∃𝑥𝜓))) | ||
| Theorem | bj-19.42t 36737 | Closed form of 19.42 2236 from the same axioms as 19.42v 1953. (Contributed by BJ, 2-Dec-2023.) |
| ⊢ (Ⅎ'𝑥𝜑 → (∃𝑥(𝜑 ∧ 𝜓) ↔ (𝜑 ∧ ∃𝑥𝜓))) | ||
| Theorem | bj-19.41t 36738 | Closed form of 19.41 2235 from the same axioms as 19.41v 1949. The same is doable with 19.27 2227, 19.28 2228, 19.31 2234, 19.32 2233, 19.44 2237, 19.45 2238. (Contributed by BJ, 2-Dec-2023.) |
| ⊢ (Ⅎ'𝑥𝜓 → (∃𝑥(𝜑 ∧ 𝜓) ↔ (∃𝑥𝜑 ∧ 𝜓))) | ||
| Theorem | bj-sbft 36739 | Version of sbft 2270 using Ⅎ', proved from core axioms. (Contributed by BJ, 19-Nov-2023.) |
| ⊢ (Ⅎ'𝑥𝜑 → ([𝑡 / 𝑥]𝜑 ↔ 𝜑)) | ||
| Theorem | bj-pm11.53vw 36740 | Version of pm11.53v 1944 with nonfreeness antecedents. One can also prove the theorem with antecedent (Ⅎ'𝑦∀𝑥𝜑 ∧ ∀𝑦Ⅎ'𝑥𝜓). (Contributed by BJ, 7-Oct-2024.) |
| ⊢ ((∀𝑥Ⅎ'𝑦𝜑 ∧ Ⅎ'𝑥∀𝑦𝜓) → (∀𝑥∀𝑦(𝜑 → 𝜓) ↔ (∃𝑥𝜑 → ∀𝑦𝜓))) | ||
| Theorem | bj-pm11.53v 36741 | Version of pm11.53v 1944 with nonfreeness antecedents. (Contributed by BJ, 7-Oct-2024.) |
| ⊢ ((∀𝑥Ⅎ'𝑦𝜑 ∧ ∀𝑦Ⅎ'𝑥𝜓) → (∀𝑥∀𝑦(𝜑 → 𝜓) ↔ (∃𝑥𝜑 → ∀𝑦𝜓))) | ||
| Theorem | bj-pm11.53a 36742* | A variant of pm11.53v 1944. One can similarly prove a variant with DV (𝑦, 𝜑) and ∀𝑦Ⅎ'𝑥𝜓 instead of DV (𝑥, 𝜓) and ∀𝑥Ⅎ'𝑦𝜑. (Contributed by BJ, 7-Oct-2024.) |
| ⊢ (∀𝑥Ⅎ'𝑦𝜑 → (∀𝑥∀𝑦(𝜑 → 𝜓) ↔ (∃𝑥𝜑 → ∀𝑦𝜓))) | ||
| Theorem | bj-equsvt 36743* | A variant of equsv 2002. (Contributed by BJ, 7-Oct-2024.) |
| ⊢ (Ⅎ'𝑥𝜑 → (∀𝑥(𝑥 = 𝑦 → 𝜑) ↔ 𝜑)) | ||
| Theorem | bj-equsalvwd 36744* | Variant of equsalvw 2003. (Contributed by BJ, 7-Oct-2024.) |
| ⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝜑 → Ⅎ'𝑥𝜒) & ⊢ ((𝜑 ∧ 𝑥 = 𝑦) → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∀𝑥(𝑥 = 𝑦 → 𝜓) ↔ 𝜒)) | ||
| Theorem | bj-equsexvwd 36745* | Variant of equsexvw 2004. (Contributed by BJ, 7-Oct-2024.) |
| ⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝜑 → Ⅎ'𝑥𝜒) & ⊢ ((𝜑 ∧ 𝑥 = 𝑦) → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∃𝑥(𝑥 = 𝑦 ∧ 𝜓) ↔ 𝜒)) | ||
| Theorem | bj-sbievwd 36746* | Variant of sbievw 2093. (Contributed by BJ, 7-Oct-2024.) |
| ⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝜑 → Ⅎ'𝑥𝜒) & ⊢ ((𝜑 ∧ 𝑥 = 𝑦) → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → ([𝑦 / 𝑥]𝜓 ↔ 𝜒)) | ||
| Theorem | bj-axc10 36747 | Alternate proof of axc10 2389. Shorter. One can prove a version with DV (𝑥, 𝑦) without ax-13 2376, by using ax6ev 1969 instead of ax6e 2387. (Contributed by BJ, 31-Mar-2021.) (Proof modification is discouraged.) |
| ⊢ (∀𝑥(𝑥 = 𝑦 → ∀𝑥𝜑) → 𝜑) | ||
| Theorem | bj-alequex 36748 | A fol lemma. See alequexv 2000 for a version with a disjoint variable condition requiring fewer axioms. Can be used to reduce the proof of spimt 2390 from 133 to 112 bytes. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (∀𝑥(𝑥 = 𝑦 → 𝜑) → ∃𝑥𝜑) | ||
| Theorem | bj-spimt2 36749 | A step in the proof of spimt 2390. (Contributed by BJ, 2-May-2019.) |
| ⊢ (∀𝑥(𝑥 = 𝑦 → (𝜑 → 𝜓)) → ((∃𝑥𝜓 → 𝜓) → (∀𝑥𝜑 → 𝜓))) | ||
| Theorem | bj-cbv3ta 36750 | Closed form of cbv3 2401. (Contributed by BJ, 2-May-2019.) |
| ⊢ (∀𝑥∀𝑦(𝑥 = 𝑦 → (𝜑 → 𝜓)) → ((∀𝑦(∃𝑥𝜓 → 𝜓) ∧ ∀𝑥(𝜑 → ∀𝑦𝜑)) → (∀𝑥𝜑 → ∀𝑦𝜓))) | ||
| Theorem | bj-cbv3tb 36751 | Closed form of cbv3 2401. (Contributed by BJ, 2-May-2019.) |
| ⊢ (∀𝑥∀𝑦(𝑥 = 𝑦 → (𝜑 → 𝜓)) → ((∀𝑦Ⅎ𝑥𝜓 ∧ ∀𝑥Ⅎ𝑦𝜑) → (∀𝑥𝜑 → ∀𝑦𝜓))) | ||
| Theorem | bj-hbsb3t 36752 | A theorem close to a closed form of hbsb3 2491. (Contributed by BJ, 2-May-2019.) |
| ⊢ (∀𝑥(𝜑 → ∀𝑦𝜑) → ([𝑦 / 𝑥]𝜑 → ∀𝑥[𝑦 / 𝑥]𝜑)) | ||
| Theorem | bj-hbsb3 36753 | Shorter proof of hbsb3 2491. (Contributed by BJ, 2-May-2019.) (Proof modification is discouraged.) |
| ⊢ (𝜑 → ∀𝑦𝜑) ⇒ ⊢ ([𝑦 / 𝑥]𝜑 → ∀𝑥[𝑦 / 𝑥]𝜑) | ||
| Theorem | bj-nfs1t 36754 | A theorem close to a closed form of nfs1 2492. (Contributed by BJ, 2-May-2019.) |
| ⊢ (∀𝑥(𝜑 → ∀𝑦𝜑) → Ⅎ𝑥[𝑦 / 𝑥]𝜑) | ||
| Theorem | bj-nfs1t2 36755 | A theorem close to a closed form of nfs1 2492. (Contributed by BJ, 2-May-2019.) |
| ⊢ (∀𝑥Ⅎ𝑦𝜑 → Ⅎ𝑥[𝑦 / 𝑥]𝜑) | ||
| Theorem | bj-nfs1 36756 | Shorter proof of nfs1 2492 (three essential steps instead of four). (Contributed by BJ, 2-May-2019.) (Proof modification is discouraged.) |
| ⊢ Ⅎ𝑦𝜑 ⇒ ⊢ Ⅎ𝑥[𝑦 / 𝑥]𝜑 | ||
It is known that ax-13 2376 is logically redundant (see ax13w 2136 and the head comment of the section "Logical redundancy of ax-10--13"). More precisely, one can remove dependency on ax-13 2376 from every theorem in set.mm which is totally unbundled (i.e., has disjoint variable conditions on all setvar variables). Indeed, start with the existing proof, and replace any occurrence of ax-13 2376 with ax13w 2136. This section is an experiment to see in practice if (partially) unbundled versions of existing theorems can be proved more efficiently without ax-13 2376 (and using ax6v 1968 / ax6ev 1969 instead of ax-6 1967 / ax6e 2387, as is currently done). One reason to be optimistic is that the first few utility theorems using ax-13 2376 (roughly 200 of them) are then used mainly with dummy variables, which one can assume distinct from any other, so that the unbundled versions of the utility theorems suffice. In this section, we prove versions of theorems in the main part with dv conditions and not requiring ax-13 2376, labeled bj-xxxv (we follow the proof of xxx but use ax6v 1968 and ax6ev 1969 instead of ax-6 1967 and ax6e 2387, and ax-5 1910 instead of ax13v 2377; shorter proofs may be possible). When no additional dv condition is required, we label it bj-xxx. It is important to keep all the bundled theorems already in set.mm, but one may also add the (partially) unbundled versions which dispense with ax-13 2376, so as to remove dependencies on ax-13 2376 from many existing theorems. UPDATE: it turns out that several theorems of the form bj-xxxv, or minor variations, are already in set.mm with label xxxw. It is also possible to remove dependencies on ax-11 2157, typically by replacing a nonfree hypothesis with a disjoint variable condition (see cbv3v2 2241 and following theorems). | ||
| Theorem | bj-axc10v 36757* | Version of axc10 2389 with a disjoint variable condition, which does not require ax-13 2376. (Contributed by BJ, 14-Jun-2019.) (Proof modification is discouraged.) |
| ⊢ (∀𝑥(𝑥 = 𝑦 → ∀𝑥𝜑) → 𝜑) | ||
| Theorem | bj-spimtv 36758* | Version of spimt 2390 with a disjoint variable condition, which does not require ax-13 2376. (Contributed by BJ, 14-Jun-2019.) (Proof modification is discouraged.) |
| ⊢ ((Ⅎ𝑥𝜓 ∧ ∀𝑥(𝑥 = 𝑦 → (𝜑 → 𝜓))) → (∀𝑥𝜑 → 𝜓)) | ||
| Theorem | bj-cbv3hv2 36759* | Version of cbv3h 2408 with two disjoint variable conditions, which does not require ax-11 2157 nor ax-13 2376. (Contributed by BJ, 24-Jun-2019.) (Proof modification is discouraged.) |
| ⊢ (𝜓 → ∀𝑥𝜓) & ⊢ (𝑥 = 𝑦 → (𝜑 → 𝜓)) ⇒ ⊢ (∀𝑥𝜑 → ∀𝑦𝜓) | ||
| Theorem | bj-cbv1hv 36760* | Version of cbv1h 2409 with a disjoint variable condition, which does not require ax-13 2376. (Contributed by BJ, 16-Jun-2019.) (Proof modification is discouraged.) |
| ⊢ (𝜑 → (𝜓 → ∀𝑦𝜓)) & ⊢ (𝜑 → (𝜒 → ∀𝑥𝜒)) & ⊢ (𝜑 → (𝑥 = 𝑦 → (𝜓 → 𝜒))) ⇒ ⊢ (∀𝑥∀𝑦𝜑 → (∀𝑥𝜓 → ∀𝑦𝜒)) | ||
| Theorem | bj-cbv2hv 36761* | Version of cbv2h 2410 with a disjoint variable condition, which does not require ax-13 2376. (Contributed by BJ, 16-Jun-2019.) (Proof modification is discouraged.) |
| ⊢ (𝜑 → (𝜓 → ∀𝑦𝜓)) & ⊢ (𝜑 → (𝜒 → ∀𝑥𝜒)) & ⊢ (𝜑 → (𝑥 = 𝑦 → (𝜓 ↔ 𝜒))) ⇒ ⊢ (∀𝑥∀𝑦𝜑 → (∀𝑥𝜓 ↔ ∀𝑦𝜒)) | ||
| Theorem | bj-cbv2v 36762* | Version of cbv2 2407 with a disjoint variable condition, which does not require ax-13 2376. (Contributed by BJ, 16-Jun-2019.) (Proof modification is discouraged.) |
| ⊢ Ⅎ𝑥𝜑 & ⊢ Ⅎ𝑦𝜑 & ⊢ (𝜑 → Ⅎ𝑦𝜓) & ⊢ (𝜑 → Ⅎ𝑥𝜒) & ⊢ (𝜑 → (𝑥 = 𝑦 → (𝜓 ↔ 𝜒))) ⇒ ⊢ (𝜑 → (∀𝑥𝜓 ↔ ∀𝑦𝜒)) | ||
| Theorem | bj-cbvaldv 36763* | Version of cbvald 2411 with a disjoint variable condition, which does not require ax-13 2376. (Contributed by BJ, 16-Jun-2019.) (Proof modification is discouraged.) |
| ⊢ Ⅎ𝑦𝜑 & ⊢ (𝜑 → Ⅎ𝑦𝜓) & ⊢ (𝜑 → (𝑥 = 𝑦 → (𝜓 ↔ 𝜒))) ⇒ ⊢ (𝜑 → (∀𝑥𝜓 ↔ ∀𝑦𝜒)) | ||
| Theorem | bj-cbvexdv 36764* | Version of cbvexd 2412 with a disjoint variable condition, which does not require ax-13 2376. (Contributed by BJ, 16-Jun-2019.) (Proof modification is discouraged.) |
| ⊢ Ⅎ𝑦𝜑 & ⊢ (𝜑 → Ⅎ𝑦𝜓) & ⊢ (𝜑 → (𝑥 = 𝑦 → (𝜓 ↔ 𝜒))) ⇒ ⊢ (𝜑 → (∃𝑥𝜓 ↔ ∃𝑦𝜒)) | ||
| Theorem | bj-cbval2vv 36765* | Version of cbval2vv 2417 with a disjoint variable condition, which does not require ax-13 2376. (Contributed by BJ, 16-Jun-2019.) (Proof modification is discouraged.) |
| ⊢ ((𝑥 = 𝑧 ∧ 𝑦 = 𝑤) → (𝜑 ↔ 𝜓)) ⇒ ⊢ (∀𝑥∀𝑦𝜑 ↔ ∀𝑧∀𝑤𝜓) | ||
| Theorem | bj-cbvex2vv 36766* | Version of cbvex2vv 2418 with a disjoint variable condition, which does not require ax-13 2376. (Contributed by BJ, 16-Jun-2019.) (Proof modification is discouraged.) |
| ⊢ ((𝑥 = 𝑧 ∧ 𝑦 = 𝑤) → (𝜑 ↔ 𝜓)) ⇒ ⊢ (∃𝑥∃𝑦𝜑 ↔ ∃𝑧∃𝑤𝜓) | ||
| Theorem | bj-cbvaldvav 36767* | Version of cbvaldva 2413 with a disjoint variable condition, which does not require ax-13 2376. (Contributed by BJ, 16-Jun-2019.) (Proof modification is discouraged.) |
| ⊢ ((𝜑 ∧ 𝑥 = 𝑦) → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∀𝑥𝜓 ↔ ∀𝑦𝜒)) | ||
| Theorem | bj-cbvexdvav 36768* | Version of cbvexdva 2414 with a disjoint variable condition, which does not require ax-13 2376. (Contributed by BJ, 16-Jun-2019.) (Proof modification is discouraged.) |
| ⊢ ((𝜑 ∧ 𝑥 = 𝑦) → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∃𝑥𝜓 ↔ ∃𝑦𝜒)) | ||
| Theorem | bj-cbvex4vv 36769* | Version of cbvex4v 2419 with a disjoint variable condition, which does not require ax-13 2376. (Contributed by BJ, 16-Jun-2019.) (Proof modification is discouraged.) |
| ⊢ ((𝑥 = 𝑣 ∧ 𝑦 = 𝑢) → (𝜑 ↔ 𝜓)) & ⊢ ((𝑧 = 𝑓 ∧ 𝑤 = 𝑔) → (𝜓 ↔ 𝜒)) ⇒ ⊢ (∃𝑥∃𝑦∃𝑧∃𝑤𝜑 ↔ ∃𝑣∃𝑢∃𝑓∃𝑔𝜒) | ||
| Theorem | bj-equsalhv 36770* |
Version of equsalh 2424 with a disjoint variable condition, which
does not
require ax-13 2376. Remark: this is the same as equsalhw 2291. TODO:
delete after moving the following paragraph somewhere.
Remarks: equsexvw 2004 has been moved to Main; Theorem ax13lem2 2380 has a DV version which is a simple consequence of ax5e 1912; Theorems nfeqf2 2381, dveeq2 2382, nfeqf1 2383, dveeq1 2384, nfeqf 2385, axc9 2386, ax13 2379, have dv versions which are simple consequences of ax-5 1910. (Contributed by BJ, 14-Jun-2019.) (Proof modification is discouraged.) (New usage is discouraged.) |
| ⊢ (𝜓 → ∀𝑥𝜓) & ⊢ (𝑥 = 𝑦 → (𝜑 ↔ 𝜓)) ⇒ ⊢ (∀𝑥(𝑥 = 𝑦 → 𝜑) ↔ 𝜓) | ||
| Theorem | bj-axc11nv 36771* | Version of axc11n 2430 with a disjoint variable condition; instance of aevlem 2055. TODO: delete after checking surrounding theorems. (Contributed by BJ, 31-May-2019.) (Proof modification is discouraged.) (New usage is discouraged.) |
| ⊢ (∀𝑥 𝑥 = 𝑦 → ∀𝑦 𝑦 = 𝑥) | ||
| Theorem | bj-aecomsv 36772* | Version of aecoms 2432 with a disjoint variable condition, provable from Tarski's FOL. The corresponding version of naecoms 2433 should not be very useful since ¬ ∀𝑥𝑥 = 𝑦, DV (𝑥, 𝑦) is true when the universe has at least two objects (see dtru 5411). (Contributed by BJ, 31-May-2019.) (Proof modification is discouraged.) |
| ⊢ (∀𝑥 𝑥 = 𝑦 → 𝜑) ⇒ ⊢ (∀𝑦 𝑦 = 𝑥 → 𝜑) | ||
| Theorem | bj-axc11v 36773* | Version of axc11 2434 with a disjoint variable condition, which does not require ax-13 2376 nor ax-10 2141. Remark: the following theorems (hbae 2435, nfae 2437, hbnae 2436, nfnae 2438, hbnaes 2439) would need to be totally unbundled to be proved without ax-13 2376, hence would be simple consequences of ax-5 1910 or nfv 1914. (Contributed by BJ, 31-May-2019.) (Proof modification is discouraged.) |
| ⊢ (∀𝑥 𝑥 = 𝑦 → (∀𝑥𝜑 → ∀𝑦𝜑)) | ||
| Theorem | bj-drnf2v 36774* | Version of drnf2 2448 with a disjoint variable condition, which does not require ax-10 2141, ax-11 2157, ax-12 2177, ax-13 2376. Instance of nfbidv 1922. Note that the version of axc15 2426 with a disjoint variable condition is actually ax12v2 2179 (up to adding a superfluous antecedent). (Contributed by BJ, 17-Jun-2019.) (Proof modification is discouraged.) |
| ⊢ (∀𝑥 𝑥 = 𝑦 → (𝜑 ↔ 𝜓)) ⇒ ⊢ (∀𝑥 𝑥 = 𝑦 → (Ⅎ𝑧𝜑 ↔ Ⅎ𝑧𝜓)) | ||
| Theorem | bj-equs45fv 36775* | Version of equs45f 2463 with a disjoint variable condition, which does not require ax-13 2376. Note that the version of equs5 2464 with a disjoint variable condition is actually sbalex 2242 (up to adding a superfluous antecedent). (Contributed by BJ, 11-Sep-2019.) (Proof modification is discouraged.) |
| ⊢ Ⅎ𝑦𝜑 ⇒ ⊢ (∃𝑥(𝑥 = 𝑦 ∧ 𝜑) ↔ ∀𝑥(𝑥 = 𝑦 → 𝜑)) | ||
| Theorem | bj-hbs1 36776* | Version of hbsb2 2486 with a disjoint variable condition, which does not require ax-13 2376, and removal of ax-13 2376 from hbs1 2274. (Contributed by BJ, 23-Jun-2019.) (Proof modification is discouraged.) |
| ⊢ ([𝑦 / 𝑥]𝜑 → ∀𝑥[𝑦 / 𝑥]𝜑) | ||
| Theorem | bj-nfs1v 36777* | Version of nfsb2 2487 with a disjoint variable condition, which does not require ax-13 2376, and removal of ax-13 2376 from nfs1v 2156. (Contributed by BJ, 24-Jun-2019.) (Proof modification is discouraged.) |
| ⊢ Ⅎ𝑥[𝑦 / 𝑥]𝜑 | ||
| Theorem | bj-hbsb2av 36778* | Version of hbsb2a 2488 with a disjoint variable condition, which does not require ax-13 2376. (Contributed by BJ, 11-Sep-2019.) (Proof modification is discouraged.) |
| ⊢ ([𝑦 / 𝑥]∀𝑦𝜑 → ∀𝑥[𝑦 / 𝑥]𝜑) | ||
| Theorem | bj-hbsb3v 36779* | Version of hbsb3 2491 with a disjoint variable condition, which does not require ax-13 2376. (Remark: the unbundled version of nfs1 2492 is given by bj-nfs1v 36777.) (Contributed by BJ, 11-Sep-2019.) (Proof modification is discouraged.) |
| ⊢ (𝜑 → ∀𝑦𝜑) ⇒ ⊢ ([𝑦 / 𝑥]𝜑 → ∀𝑥[𝑦 / 𝑥]𝜑) | ||
| Theorem | bj-nfsab1 36780* | Remove dependency on ax-13 2376 from nfsab1 2721. UPDATE / TODO: nfsab1 2721 does not use ax-13 2376 either anymore; bj-nfsab1 36780 is shorter than nfsab1 2721 but uses ax-12 2177. (Contributed by BJ, 23-Jun-2019.) (Proof modification is discouraged.) |
| ⊢ Ⅎ𝑥 𝑦 ∈ {𝑥 ∣ 𝜑} | ||
| Theorem | bj-dtrucor2v 36781* | Version of dtrucor2 5342 with a disjoint variable condition, which does not require ax-13 2376 (nor ax-4 1809, ax-5 1910, ax-7 2007, ax-12 2177). (Contributed by BJ, 16-Jul-2019.) (Proof modification is discouraged.) |
| ⊢ (𝑥 = 𝑦 → 𝑥 ≠ 𝑦) ⇒ ⊢ (𝜑 ∧ ¬ 𝜑) | ||
The closed formula ∀𝑥∀𝑦𝑥 = 𝑦 approximately means that the var metavariables 𝑥 and 𝑦 represent the same variable vi. In a domain with at most one object, however, this formula is always true, hence the "approximately" in the previous sentence. | ||
| Theorem | bj-hbaeb2 36782 | Biconditional version of a form of hbae 2435 with commuted quantifiers, not requiring ax-11 2157. (Contributed by BJ, 12-Dec-2019.) (Proof modification is discouraged.) |
| ⊢ (∀𝑥 𝑥 = 𝑦 ↔ ∀𝑥∀𝑧 𝑥 = 𝑦) | ||
| Theorem | bj-hbaeb 36783 | Biconditional version of hbae 2435. (Contributed by BJ, 6-Oct-2018.) (Proof modification is discouraged.) |
| ⊢ (∀𝑥 𝑥 = 𝑦 ↔ ∀𝑧∀𝑥 𝑥 = 𝑦) | ||
| Theorem | bj-hbnaeb 36784 | Biconditional version of hbnae 2436 (to replace it?). (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (¬ ∀𝑥 𝑥 = 𝑦 ↔ ∀𝑧 ¬ ∀𝑥 𝑥 = 𝑦) | ||
| Theorem | bj-dvv 36785 | A special instance of bj-hbaeb2 36782. A lemma for distinct var metavariables. Note that the right-hand side is a closed formula (a sentence). (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (∀𝑥 𝑥 = 𝑦 ↔ ∀𝑥∀𝑦 𝑥 = 𝑦) | ||
As a rule of thumb, if a theorem of the form ⊢ (𝜑 ↔ 𝜓) ⇒ ⊢ (𝜒 ↔ 𝜃) is in the database, and the "more precise" theorems ⊢ (𝜑 → 𝜓) ⇒ ⊢ (𝜒 → 𝜃) and ⊢ (𝜓 → 𝜑) ⇒ ⊢ (𝜃 → 𝜒) also hold (see bj-bisym 36554), then they should be added to the database. The present case is similar. Similar additions can be done regarding equsex 2422 (and equsalh 2424 and equsexh 2425). Even if only one of these two theorems holds, it should be added to the database. | ||
| Theorem | bj-equsal1t 36786 | Duplication of wl-equsal1t 37506, with shorter proof. If one imposes a disjoint variable condition on x,y , then one can use alequexv 2000 and reduce axiom dependencies, and similarly for the following theorems. Note: wl-equsalcom 37507 is also interesting. (Contributed by BJ, 6-Oct-2018.) |
| ⊢ (Ⅎ𝑥𝜑 → (∀𝑥(𝑥 = 𝑦 → 𝜑) ↔ 𝜑)) | ||
| Theorem | bj-equsal1ti 36787 | Inference associated with bj-equsal1t 36786. (Contributed by BJ, 30-Sep-2018.) |
| ⊢ Ⅎ𝑥𝜑 ⇒ ⊢ (∀𝑥(𝑥 = 𝑦 → 𝜑) ↔ 𝜑) | ||
| Theorem | bj-equsal1 36788 | One direction of equsal 2421. (Contributed by BJ, 30-Sep-2018.) |
| ⊢ Ⅎ𝑥𝜓 & ⊢ (𝑥 = 𝑦 → (𝜑 → 𝜓)) ⇒ ⊢ (∀𝑥(𝑥 = 𝑦 → 𝜑) → 𝜓) | ||
| Theorem | bj-equsal2 36789 | One direction of equsal 2421. (Contributed by BJ, 30-Sep-2018.) |
| ⊢ Ⅎ𝑥𝜑 & ⊢ (𝑥 = 𝑦 → (𝜑 → 𝜓)) ⇒ ⊢ (𝜑 → ∀𝑥(𝑥 = 𝑦 → 𝜓)) | ||
| Theorem | bj-equsal 36790 | Shorter proof of equsal 2421. (Contributed by BJ, 30-Sep-2018.) Proof modification is discouraged to avoid using equsal 2421, but "min */exc equsal" is ok. (Proof modification is discouraged.) |
| ⊢ Ⅎ𝑥𝜓 & ⊢ (𝑥 = 𝑦 → (𝜑 ↔ 𝜓)) ⇒ ⊢ (∀𝑥(𝑥 = 𝑦 → 𝜑) ↔ 𝜓) | ||
References are made to the second edition (1927, reprinted 1963) of Principia Mathematica, Vol. 1. Theorems are referred to in the form "PM*xx.xx". | ||
| Theorem | stdpc5t 36791 | Closed form of stdpc5 2208. (Possible to place it before 19.21t 2206 and use it to prove 19.21t 2206). (Contributed by BJ, 15-Sep-2018.) (Proof modification is discouraged.) |
| ⊢ (Ⅎ𝑥𝜑 → (∀𝑥(𝜑 → 𝜓) → (𝜑 → ∀𝑥𝜓))) | ||
| Theorem | bj-stdpc5 36792 | More direct proof of stdpc5 2208. (Contributed by BJ, 15-Sep-2018.) (Proof modification is discouraged.) |
| ⊢ Ⅎ𝑥𝜑 ⇒ ⊢ (∀𝑥(𝜑 → 𝜓) → (𝜑 → ∀𝑥𝜓)) | ||
| Theorem | 2stdpc5 36793 | A double stdpc5 2208 (one direction of PM*11.3). See also 2stdpc4 2070 and 19.21vv 44348. (Contributed by BJ, 15-Sep-2018.) (Proof modification is discouraged.) |
| ⊢ Ⅎ𝑥𝜑 & ⊢ Ⅎ𝑦𝜑 ⇒ ⊢ (∀𝑥∀𝑦(𝜑 → 𝜓) → (𝜑 → ∀𝑥∀𝑦𝜓)) | ||
| Theorem | bj-19.21t0 36794 | Proof of 19.21t 2206 from stdpc5t 36791. (Contributed by BJ, 15-Sep-2018.) (Proof modification is discouraged.) |
| ⊢ (Ⅎ𝑥𝜑 → (∀𝑥(𝜑 → 𝜓) ↔ (𝜑 → ∀𝑥𝜓))) | ||
| Theorem | exlimii 36795 | Inference associated with exlimi 2217. Inferring a theorem when it is implied by an antecedent which may be true. (Contributed by BJ, 15-Sep-2018.) |
| ⊢ Ⅎ𝑥𝜓 & ⊢ (𝜑 → 𝜓) & ⊢ ∃𝑥𝜑 ⇒ ⊢ 𝜓 | ||
| Theorem | ax11-pm 36796 | Proof of ax-11 2157 similar to PM's proof of alcom 2159 (PM*11.2). For a proof closer to PM's proof, see ax11-pm2 36800. Axiom ax-11 2157 is used in the proof only through nfa2 2176. (Contributed by BJ, 15-Sep-2018.) (Proof modification is discouraged.) |
| ⊢ (∀𝑥∀𝑦𝜑 → ∀𝑦∀𝑥𝜑) | ||
| Theorem | ax6er 36797 | Commuted form of ax6e 2387. (Could be placed right after ax6e 2387). (Contributed by BJ, 15-Sep-2018.) |
| ⊢ ∃𝑥 𝑦 = 𝑥 | ||
| Theorem | exlimiieq1 36798 | Inferring a theorem when it is implied by an equality which may be true. (Contributed by BJ, 30-Sep-2018.) |
| ⊢ Ⅎ𝑥𝜑 & ⊢ (𝑥 = 𝑦 → 𝜑) ⇒ ⊢ 𝜑 | ||
| Theorem | exlimiieq2 36799 | Inferring a theorem when it is implied by an equality which may be true. (Contributed by BJ, 15-Sep-2018.) (Revised by BJ, 30-Sep-2018.) |
| ⊢ Ⅎ𝑦𝜑 & ⊢ (𝑥 = 𝑦 → 𝜑) ⇒ ⊢ 𝜑 | ||
| Theorem | ax11-pm2 36800* | Proof of ax-11 2157 from the standard axioms of predicate calculus, similar to PM's proof of alcom 2159 (PM*11.2). This proof requires that 𝑥 and 𝑦 be distinct. Axiom ax-11 2157 is used in the proof only through nfal 2323, nfsb 2527, sbal 2169, sb8 2521. See also ax11-pm 36796. (Contributed by BJ, 15-Sep-2018.) (Proof modification is discouraged.) |
| ⊢ (∀𝑥∀𝑦𝜑 → ∀𝑦∀𝑥𝜑) | ||
| < Previous Next > |
| Copyright terms: Public domain | < Previous Next > |