![]() |
Metamath
Proof Explorer Theorem List (p. 19 of 489) | < 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-30950) |
![]() (30951-32473) |
![]() (32474-48899) |
Type | Label | Description |
---|---|---|
Statement | ||
Theorem | hbth 1801 |
No variable is (effectively) free in a theorem.
This and later "hypothesis-building" lemmas, with labels starting "hb...", allow to construct proofs of formulas of the form ⊢ (𝜑 → ∀𝑥𝜑) from smaller formulas of this form. These are useful for constructing hypotheses that state "𝑥 is (effectively) not free in 𝜑". (Contributed by NM, 11-May-1993.) This hb* idiom is generally being replaced by the nf* idiom (see nfth 1799), but keeps its interest in some cases. (Revised by BJ, 23-Sep-2022.) |
⊢ 𝜑 ⇒ ⊢ (𝜑 → ∀𝑥𝜑) | ||
Theorem | nftru 1802 | The true constant has no free variables. (This can also be proven in one step with nfv 1913, but this proof does not use ax-5 1909.) (Contributed by Mario Carneiro, 6-Oct-2016.) |
⊢ Ⅎ𝑥⊤ | ||
Theorem | nffal 1803 | The false constant has no free variables (see nftru 1802). (Contributed by BJ, 6-May-2019.) |
⊢ Ⅎ𝑥⊥ | ||
Theorem | sptruw 1804 | Version of sp 2184 when 𝜑 is true. Instance of a1i 11. Uses only Tarski's FOL axiom schemes. (Contributed by NM, 23-Apr-2017.) |
⊢ 𝜑 ⇒ ⊢ (∀𝑥𝜑 → 𝜑) | ||
Theorem | altru 1805 | For all sets, ⊤ is true. (Contributed by Anthony Hart, 13-Sep-2011.) |
⊢ ∀𝑥⊤ | ||
Theorem | alfal 1806 | For all sets, ¬ ⊥ is true. (Contributed by Anthony Hart, 13-Sep-2011.) |
⊢ ∀𝑥 ¬ ⊥ | ||
Axiom | ax-4 1807 | Axiom of Quantified Implication. Axiom C4 of [Monk2] p. 105 and Theorem 19.20 of [Margaris] p. 90. It is restated as alim 1808 for labeling consistency. It should be used only by alim 1808. (Contributed by NM, 21-May-2008.) Use alim 1808 instead. (New usage is discouraged.) |
⊢ (∀𝑥(𝜑 → 𝜓) → (∀𝑥𝜑 → ∀𝑥𝜓)) | ||
Theorem | alim 1808 | Restatement of Axiom ax-4 1807, for labeling consistency. It should be the only theorem using ax-4 1807. (Contributed by NM, 10-Jan-1993.) |
⊢ (∀𝑥(𝜑 → 𝜓) → (∀𝑥𝜑 → ∀𝑥𝜓)) | ||
Theorem | alimi 1809 | Inference quantifying both antecedent and consequent. (Contributed by NM, 5-Jan-1993.) |
⊢ (𝜑 → 𝜓) ⇒ ⊢ (∀𝑥𝜑 → ∀𝑥𝜓) | ||
Theorem | 2alimi 1810 | Inference doubly quantifying both antecedent and consequent. (Contributed by NM, 3-Feb-2005.) |
⊢ (𝜑 → 𝜓) ⇒ ⊢ (∀𝑥∀𝑦𝜑 → ∀𝑥∀𝑦𝜓) | ||
Theorem | ala1 1811 | Add an antecedent in a universally quantified formula. (Contributed by BJ, 6-Oct-2018.) |
⊢ (∀𝑥𝜑 → ∀𝑥(𝜓 → 𝜑)) | ||
Theorem | al2im 1812 | Closed form of al2imi 1813. Version of alim 1808 for a nested implication. (Contributed by Alan Sare, 31-Dec-2011.) |
⊢ (∀𝑥(𝜑 → (𝜓 → 𝜒)) → (∀𝑥𝜑 → (∀𝑥𝜓 → ∀𝑥𝜒))) | ||
Theorem | al2imi 1813 | Inference quantifying antecedent, nested antecedent, and consequent. (Contributed by NM, 10-Jan-1993.) |
⊢ (𝜑 → (𝜓 → 𝜒)) ⇒ ⊢ (∀𝑥𝜑 → (∀𝑥𝜓 → ∀𝑥𝜒)) | ||
Theorem | alanimi 1814 | Variant of al2imi 1813 with conjunctive antecedent. (Contributed by Andrew Salmon, 8-Jun-2011.) |
⊢ ((𝜑 ∧ 𝜓) → 𝜒) ⇒ ⊢ ((∀𝑥𝜑 ∧ ∀𝑥𝜓) → ∀𝑥𝜒) | ||
Theorem | alimdh 1815 | Deduction form of Theorem 19.20 of [Margaris] p. 90, see alim 1808. (Contributed by NM, 4-Jan-2002.) |
⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝜑 → (𝜓 → 𝜒)) ⇒ ⊢ (𝜑 → (∀𝑥𝜓 → ∀𝑥𝜒)) | ||
Theorem | albi 1816 | Theorem 19.15 of [Margaris] p. 90. (Contributed by NM, 24-Jan-1993.) |
⊢ (∀𝑥(𝜑 ↔ 𝜓) → (∀𝑥𝜑 ↔ ∀𝑥𝜓)) | ||
Theorem | albii 1817 | Inference adding universal quantifier to both sides of an equivalence. (Contributed by NM, 7-Aug-1994.) |
⊢ (𝜑 ↔ 𝜓) ⇒ ⊢ (∀𝑥𝜑 ↔ ∀𝑥𝜓) | ||
Theorem | 2albii 1818 | Inference adding two universal quantifiers to both sides of an equivalence. (Contributed by NM, 9-Mar-1997.) |
⊢ (𝜑 ↔ 𝜓) ⇒ ⊢ (∀𝑥∀𝑦𝜑 ↔ ∀𝑥∀𝑦𝜓) | ||
Theorem | 3albii 1819 | Inference adding three universal quantifiers to both sides of an equivalence. (Contributed by Peter Mazsa, 10-Aug-2018.) |
⊢ (𝜑 ↔ 𝜓) ⇒ ⊢ (∀𝑥∀𝑦∀𝑧𝜑 ↔ ∀𝑥∀𝑦∀𝑧𝜓) | ||
Theorem | sylgt 1820 | Closed form of sylg 1821. (Contributed by BJ, 2-May-2019.) |
⊢ (∀𝑥(𝜓 → 𝜒) → ((𝜑 → ∀𝑥𝜓) → (𝜑 → ∀𝑥𝜒))) | ||
Theorem | sylg 1821 | A syllogism combined with generalization. Inference associated with sylgt 1820. General form of alrimih 1822. (Contributed by NM, 9-Jan-1993.) Extract from proof of alrimih 1822. (Revised by BJ, 4-Oct-2019.) |
⊢ (𝜑 → ∀𝑥𝜓) & ⊢ (𝜓 → 𝜒) ⇒ ⊢ (𝜑 → ∀𝑥𝜒) | ||
Theorem | alrimih 1822 | Inference form of Theorem 19.21 of [Margaris] p. 90. See 19.21 2208 and 19.21h 2291. Instance of sylg 1821. (Contributed by NM, 9-Jan-1993.) |
⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝜑 → 𝜓) ⇒ ⊢ (𝜑 → ∀𝑥𝜓) | ||
Theorem | hbxfrbi 1823 | A utility lemma to transfer a bound-variable hypothesis builder into a definition. See hbxfreq 2875 for equality version. (Contributed by Jonathan Ben-Naim, 3-Jun-2011.) |
⊢ (𝜑 ↔ 𝜓) & ⊢ (𝜓 → ∀𝑥𝜓) ⇒ ⊢ (𝜑 → ∀𝑥𝜑) | ||
Theorem | alex 1824 | Universal quantifier in terms of existential quantifier and negation. Dual of df-ex 1778. See also the dual pair alnex 1779 / exnal 1825. Theorem 19.6 of [Margaris] p. 89. (Contributed by NM, 12-Mar-1993.) |
⊢ (∀𝑥𝜑 ↔ ¬ ∃𝑥 ¬ 𝜑) | ||
Theorem | exnal 1825 | Existential quantification of negation is equivalent to negation of universal quantification. Dual of alnex 1779. See also the dual pair df-ex 1778 / alex 1824. Theorem 19.14 of [Margaris] p. 90. (Contributed by NM, 12-Mar-1993.) |
⊢ (∃𝑥 ¬ 𝜑 ↔ ¬ ∀𝑥𝜑) | ||
Theorem | 2nalexn 1826 | Part of theorem *11.5 in [WhiteheadRussell] p. 164. (Contributed by Andrew Salmon, 24-May-2011.) |
⊢ (¬ ∀𝑥∀𝑦𝜑 ↔ ∃𝑥∃𝑦 ¬ 𝜑) | ||
Theorem | 2exnaln 1827 | Theorem *11.22 in [WhiteheadRussell] p. 160. (Contributed by Andrew Salmon, 24-May-2011.) |
⊢ (∃𝑥∃𝑦𝜑 ↔ ¬ ∀𝑥∀𝑦 ¬ 𝜑) | ||
Theorem | 2nexaln 1828 | Theorem *11.25 in [WhiteheadRussell] p. 160. (Contributed by Andrew Salmon, 24-May-2011.) |
⊢ (¬ ∃𝑥∃𝑦𝜑 ↔ ∀𝑥∀𝑦 ¬ 𝜑) | ||
Theorem | alimex 1829 | An equivalence between an implication with a universally quantified consequent and an implication with an existentially quantified antecedent. An interesting case is when the same formula is substituted for both 𝜑 and 𝜓, since then both implications express a type of nonfreeness. See also eximal 1780. (Contributed by BJ, 12-May-2019.) |
⊢ ((𝜑 → ∀𝑥𝜓) ↔ (∃𝑥 ¬ 𝜓 → ¬ 𝜑)) | ||
Theorem | aleximi 1830 | A variant of al2imi 1813: instead of applying ∀𝑥 quantifiers to the final implication, replace them with ∃𝑥. A shorter proof is possible using nfa1 2152, sps 2186 and eximd 2217, but it depends on more axioms. (Contributed by Wolf Lammen, 18-Aug-2019.) |
⊢ (𝜑 → (𝜓 → 𝜒)) ⇒ ⊢ (∀𝑥𝜑 → (∃𝑥𝜓 → ∃𝑥𝜒)) | ||
Theorem | alexbii 1831 | Biconditional form of aleximi 1830. (Contributed by BJ, 16-Nov-2020.) |
⊢ (𝜑 → (𝜓 ↔ 𝜒)) ⇒ ⊢ (∀𝑥𝜑 → (∃𝑥𝜓 ↔ ∃𝑥𝜒)) | ||
Theorem | exim 1832 | Theorem 19.22 of [Margaris] p. 90. (Contributed by NM, 10-Jan-1993.) (Proof shortened by Wolf Lammen, 4-Jul-2014.) |
⊢ (∀𝑥(𝜑 → 𝜓) → (∃𝑥𝜑 → ∃𝑥𝜓)) | ||
Theorem | eximi 1833 | Inference adding existential quantifier to antecedent and consequent. (Contributed by NM, 10-Jan-1993.) |
⊢ (𝜑 → 𝜓) ⇒ ⊢ (∃𝑥𝜑 → ∃𝑥𝜓) | ||
Theorem | 2eximi 1834 | Inference adding two existential quantifiers to antecedent and consequent. (Contributed by NM, 3-Feb-2005.) |
⊢ (𝜑 → 𝜓) ⇒ ⊢ (∃𝑥∃𝑦𝜑 → ∃𝑥∃𝑦𝜓) | ||
Theorem | eximii 1835 | Inference associated with eximi 1833. (Contributed by BJ, 3-Feb-2018.) |
⊢ ∃𝑥𝜑 & ⊢ (𝜑 → 𝜓) ⇒ ⊢ ∃𝑥𝜓 | ||
Theorem | exa1 1836 | Add an antecedent in an existentially quantified formula. (Contributed by BJ, 6-Oct-2018.) |
⊢ (∃𝑥𝜑 → ∃𝑥(𝜓 → 𝜑)) | ||
Theorem | 19.38 1837 | Theorem 19.38 of [Margaris] p. 90. The converse holds under nonfreeness conditions, see 19.38a 1838 and 19.38b 1839. (Contributed by NM, 12-Mar-1993.) Allow a shortening of 19.21t 2207. (Revised by Wolf Lammen, 2-Jan-2018.) |
⊢ ((∃𝑥𝜑 → ∀𝑥𝜓) → ∀𝑥(𝜑 → 𝜓)) | ||
Theorem | 19.38a 1838 | Under a nonfreeness hypothesis, the implication 19.38 1837 can be strengthened to an equivalence. See also 19.38b 1839. (Contributed by BJ, 3-Nov-2021.) (Proof shortened by Wolf Lammen, 9-Jul-2022.) |
⊢ (Ⅎ𝑥𝜑 → ((∃𝑥𝜑 → ∀𝑥𝜓) ↔ ∀𝑥(𝜑 → 𝜓))) | ||
Theorem | 19.38b 1839 | Under a nonfreeness hypothesis, the implication 19.38 1837 can be strengthened to an equivalence. See also 19.38a 1838. (Contributed by BJ, 3-Nov-2021.) (Proof shortened by Wolf Lammen, 9-Jul-2022.) |
⊢ (Ⅎ𝑥𝜓 → ((∃𝑥𝜑 → ∀𝑥𝜓) ↔ ∀𝑥(𝜑 → 𝜓))) | ||
Theorem | imnang 1840 | Quantified implication in terms of quantified negation of conjunction. (Contributed by BJ, 16-Jul-2021.) |
⊢ (∀𝑥(𝜑 → ¬ 𝜓) ↔ ∀𝑥 ¬ (𝜑 ∧ 𝜓)) | ||
Theorem | alinexa 1841 | A transformation of quantifiers and logical connectives. (Contributed by NM, 19-Aug-1993.) |
⊢ (∀𝑥(𝜑 → ¬ 𝜓) ↔ ¬ ∃𝑥(𝜑 ∧ 𝜓)) | ||
Theorem | exnalimn 1842 | Existential quantification of a conjunction expressed with only primitive symbols (→, ¬, ∀). (Contributed by NM, 10-May-1993.) State the most general instance. (Revised by BJ, 29-Sep-2019.) |
⊢ (∃𝑥(𝜑 ∧ 𝜓) ↔ ¬ ∀𝑥(𝜑 → ¬ 𝜓)) | ||
Theorem | alexn 1843 | A relationship between two quantifiers and negation. (Contributed by NM, 18-Aug-1993.) |
⊢ (∀𝑥∃𝑦 ¬ 𝜑 ↔ ¬ ∃𝑥∀𝑦𝜑) | ||
Theorem | 2exnexn 1844 | Theorem *11.51 in [WhiteheadRussell] p. 164. (Contributed by Andrew Salmon, 24-May-2011.) (Proof shortened by Wolf Lammen, 25-Sep-2014.) |
⊢ (∃𝑥∀𝑦𝜑 ↔ ¬ ∀𝑥∃𝑦 ¬ 𝜑) | ||
Theorem | exbi 1845 | Theorem 19.18 of [Margaris] p. 90. (Contributed by NM, 12-Mar-1993.) |
⊢ (∀𝑥(𝜑 ↔ 𝜓) → (∃𝑥𝜑 ↔ ∃𝑥𝜓)) | ||
Theorem | exbii 1846 | Inference adding existential quantifier to both sides of an equivalence. (Contributed by NM, 24-May-1994.) |
⊢ (𝜑 ↔ 𝜓) ⇒ ⊢ (∃𝑥𝜑 ↔ ∃𝑥𝜓) | ||
Theorem | 2exbii 1847 | Inference adding two existential quantifiers to both sides of an equivalence. (Contributed by NM, 16-Mar-1995.) |
⊢ (𝜑 ↔ 𝜓) ⇒ ⊢ (∃𝑥∃𝑦𝜑 ↔ ∃𝑥∃𝑦𝜓) | ||
Theorem | 3exbii 1848 | Inference adding three existential quantifiers to both sides of an equivalence. (Contributed by NM, 2-May-1995.) |
⊢ (𝜑 ↔ 𝜓) ⇒ ⊢ (∃𝑥∃𝑦∃𝑧𝜑 ↔ ∃𝑥∃𝑦∃𝑧𝜓) | ||
Theorem | nfbiit 1849 | Equivalence theorem for the nonfreeness predicate. Closed form of nfbii 1850. (Contributed by Giovanni Mascellani, 10-Apr-2018.) Reduce axiom usage. (Revised by BJ, 6-May-2019.) |
⊢ (∀𝑥(𝜑 ↔ 𝜓) → (Ⅎ𝑥𝜑 ↔ Ⅎ𝑥𝜓)) | ||
Theorem | nfbii 1850 | Equality theorem for the nonfreeness predicate. (Contributed by Mario Carneiro, 11-Aug-2016.) df-nf 1782 changed. (Revised by Wolf Lammen, 12-Sep-2021.) |
⊢ (𝜑 ↔ 𝜓) ⇒ ⊢ (Ⅎ𝑥𝜑 ↔ Ⅎ𝑥𝜓) | ||
Theorem | nfxfr 1851 | A utility lemma to transfer a bound-variable hypothesis builder into a definition. (Contributed by Mario Carneiro, 11-Aug-2016.) |
⊢ (𝜑 ↔ 𝜓) & ⊢ Ⅎ𝑥𝜓 ⇒ ⊢ Ⅎ𝑥𝜑 | ||
Theorem | nfxfrd 1852 | A utility lemma to transfer a bound-variable hypothesis builder into a definition. (Contributed by Mario Carneiro, 24-Sep-2016.) |
⊢ (𝜑 ↔ 𝜓) & ⊢ (𝜒 → Ⅎ𝑥𝜓) ⇒ ⊢ (𝜒 → Ⅎ𝑥𝜑) | ||
Theorem | nfnbi 1853 | A variable is nonfree in a proposition if and only if it is so in its negation. (Contributed by BJ, 6-May-2019.) (Proof shortened by Wolf Lammen, 6-Oct-2024.) |
⊢ (Ⅎ𝑥𝜑 ↔ Ⅎ𝑥 ¬ 𝜑) | ||
Theorem | nfnbiOLD 1854 | Obsolete version of nfnbi 1853 as of 6-Oct-2024. (Contributed by BJ, 6-May-2019.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ (Ⅎ𝑥𝜑 ↔ Ⅎ𝑥 ¬ 𝜑) | ||
Theorem | nfnt 1855 | If a variable is nonfree in a proposition, then it is nonfree in its negation. (Contributed by Mario Carneiro, 24-Sep-2016.) (Proof shortened by Wolf Lammen, 28-Dec-2017.) (Revised by BJ, 24-Jul-2019.) df-nf 1782 changed. (Revised by Wolf Lammen, 4-Oct-2021.) |
⊢ (Ⅎ𝑥𝜑 → Ⅎ𝑥 ¬ 𝜑) | ||
Theorem | nfn 1856 | Inference associated with nfnt 1855. (Contributed by Mario Carneiro, 11-Aug-2016.) df-nf 1782 changed. (Revised by Wolf Lammen, 18-Sep-2021.) |
⊢ Ⅎ𝑥𝜑 ⇒ ⊢ Ⅎ𝑥 ¬ 𝜑 | ||
Theorem | nfnd 1857 | Deduction associated with nfnt 1855. (Contributed by Mario Carneiro, 24-Sep-2016.) |
⊢ (𝜑 → Ⅎ𝑥𝜓) ⇒ ⊢ (𝜑 → Ⅎ𝑥 ¬ 𝜓) | ||
Theorem | exanali 1858 | A transformation of quantifiers and logical connectives. (Contributed by NM, 25-Mar-1996.) (Proof shortened by Wolf Lammen, 4-Sep-2014.) |
⊢ (∃𝑥(𝜑 ∧ ¬ 𝜓) ↔ ¬ ∀𝑥(𝜑 → 𝜓)) | ||
Theorem | 2exanali 1859 | Theorem *11.521 in [WhiteheadRussell] p. 164. (Contributed by Andrew Salmon, 24-May-2011.) |
⊢ (¬ ∃𝑥∃𝑦(𝜑 ∧ ¬ 𝜓) ↔ ∀𝑥∀𝑦(𝜑 → 𝜓)) | ||
Theorem | exancom 1860 | Commutation of conjunction inside an existential quantifier. (Contributed by NM, 18-Aug-1993.) |
⊢ (∃𝑥(𝜑 ∧ 𝜓) ↔ ∃𝑥(𝜓 ∧ 𝜑)) | ||
Theorem | exan 1861 | Place a conjunct in the scope of an existential quantifier. (Contributed by NM, 18-Aug-1993.) (Proof shortened by Andrew Salmon, 25-May-2011.) (Proof shortened by Wolf Lammen, 13-Jan-2018.) Reduce axiom dependencies. (Revised by BJ, 7-Jul-2021.) (Proof shortened by Wolf Lammen, 6-Nov-2022.) Expand hypothesis. (Revised by Steven Nguyen, 19-Jun-2023.) |
⊢ ∃𝑥𝜑 & ⊢ 𝜓 ⇒ ⊢ ∃𝑥(𝜑 ∧ 𝜓) | ||
Theorem | alrimdh 1862 | Deduction form of Theorem 19.21 of [Margaris] p. 90, see 19.21 2208 and 19.21h 2291. (Contributed by NM, 10-Feb-1997.) (Proof shortened by Andrew Salmon, 13-May-2011.) |
⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝜓 → ∀𝑥𝜓) & ⊢ (𝜑 → (𝜓 → 𝜒)) ⇒ ⊢ (𝜑 → (𝜓 → ∀𝑥𝜒)) | ||
Theorem | eximdh 1863 | Deduction from Theorem 19.22 of [Margaris] p. 90. (Contributed by NM, 20-May-1996.) |
⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝜑 → (𝜓 → 𝜒)) ⇒ ⊢ (𝜑 → (∃𝑥𝜓 → ∃𝑥𝜒)) | ||
Theorem | nexdh 1864 | Deduction for generalization rule for negated wff. (Contributed by NM, 2-Jan-2002.) |
⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝜑 → ¬ 𝜓) ⇒ ⊢ (𝜑 → ¬ ∃𝑥𝜓) | ||
Theorem | albidh 1865 | Formula-building rule for universal quantifier (deduction form). (Contributed by NM, 26-May-1993.) |
⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝜑 → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∀𝑥𝜓 ↔ ∀𝑥𝜒)) | ||
Theorem | exbidh 1866 | Formula-building rule for existential quantifier (deduction form). (Contributed by NM, 26-May-1993.) |
⊢ (𝜑 → ∀𝑥𝜑) & ⊢ (𝜑 → (𝜓 ↔ 𝜒)) ⇒ ⊢ (𝜑 → (∃𝑥𝜓 ↔ ∃𝑥𝜒)) | ||
Theorem | exsimpl 1867 | Simplification of an existentially quantified conjunction. (Contributed by Rodolfo Medina, 25-Sep-2010.) (Proof shortened by Andrew Salmon, 29-Jun-2011.) |
⊢ (∃𝑥(𝜑 ∧ 𝜓) → ∃𝑥𝜑) | ||
Theorem | exsimpr 1868 | Simplification of an existentially quantified conjunction. (Contributed by Rodolfo Medina, 25-Sep-2010.) (Proof shortened by Andrew Salmon, 29-Jun-2011.) |
⊢ (∃𝑥(𝜑 ∧ 𝜓) → ∃𝑥𝜓) | ||
Theorem | 19.26 1869 | Theorem 19.26 of [Margaris] p. 90. Also Theorem *10.22 of [WhiteheadRussell] p. 147. (Contributed by NM, 12-Mar-1993.) (Proof shortened by Wolf Lammen, 4-Jul-2014.) |
⊢ (∀𝑥(𝜑 ∧ 𝜓) ↔ (∀𝑥𝜑 ∧ ∀𝑥𝜓)) | ||
Theorem | 19.26-2 1870 | Theorem 19.26 1869 with two quantifiers. (Contributed by NM, 3-Feb-2005.) |
⊢ (∀𝑥∀𝑦(𝜑 ∧ 𝜓) ↔ (∀𝑥∀𝑦𝜑 ∧ ∀𝑥∀𝑦𝜓)) | ||
Theorem | 19.26-3an 1871 | Theorem 19.26 1869 with triple conjunction. (Contributed by NM, 13-Sep-2011.) |
⊢ (∀𝑥(𝜑 ∧ 𝜓 ∧ 𝜒) ↔ (∀𝑥𝜑 ∧ ∀𝑥𝜓 ∧ ∀𝑥𝜒)) | ||
Theorem | 19.29 1872 | Theorem 19.29 of [Margaris] p. 90. See also 19.29r 1873. (Contributed by NM, 21-Jun-1993.) (Proof shortened by Andrew Salmon, 13-May-2011.) |
⊢ ((∀𝑥𝜑 ∧ ∃𝑥𝜓) → ∃𝑥(𝜑 ∧ 𝜓)) | ||
Theorem | 19.29r 1873 | Variation of 19.29 1872. (Contributed by NM, 18-Aug-1993.) (Proof shortened by Wolf Lammen, 12-Nov-2020.) |
⊢ ((∃𝑥𝜑 ∧ ∀𝑥𝜓) → ∃𝑥(𝜑 ∧ 𝜓)) | ||
Theorem | 19.29r2 1874 | Variation of 19.29r 1873 with double quantification. (Contributed by NM, 3-Feb-2005.) |
⊢ ((∃𝑥∃𝑦𝜑 ∧ ∀𝑥∀𝑦𝜓) → ∃𝑥∃𝑦(𝜑 ∧ 𝜓)) | ||
Theorem | 19.29x 1875 | Variation of 19.29 1872 with mixed quantification. (Contributed by NM, 11-Feb-2005.) |
⊢ ((∃𝑥∀𝑦𝜑 ∧ ∀𝑥∃𝑦𝜓) → ∃𝑥∃𝑦(𝜑 ∧ 𝜓)) | ||
Theorem | 19.35 1876 | Theorem 19.35 of [Margaris] p. 90. This theorem is useful for moving an implication (in the form of the right-hand side) into the scope of a single existential quantifier. (Contributed by NM, 12-Mar-1993.) (Proof shortened by Wolf Lammen, 27-Jun-2014.) |
⊢ (∃𝑥(𝜑 → 𝜓) ↔ (∀𝑥𝜑 → ∃𝑥𝜓)) | ||
Theorem | 19.35i 1877 | Inference associated with 19.35 1876. (Contributed by NM, 21-Jun-1993.) |
⊢ ∃𝑥(𝜑 → 𝜓) ⇒ ⊢ (∀𝑥𝜑 → ∃𝑥𝜓) | ||
Theorem | 19.35ri 1878 | Inference associated with 19.35 1876. (Contributed by NM, 12-Mar-1993.) |
⊢ (∀𝑥𝜑 → ∃𝑥𝜓) ⇒ ⊢ ∃𝑥(𝜑 → 𝜓) | ||
Theorem | 19.25 1879 | Theorem 19.25 of [Margaris] p. 90. (Contributed by NM, 12-Mar-1993.) |
⊢ (∀𝑦∃𝑥(𝜑 → 𝜓) → (∃𝑦∀𝑥𝜑 → ∃𝑦∃𝑥𝜓)) | ||
Theorem | 19.30 1880 | Theorem 19.30 of [Margaris] p. 90. (Contributed by NM, 12-Mar-1993.) (Proof shortened by Andrew Salmon, 25-May-2011.) |
⊢ (∀𝑥(𝜑 ∨ 𝜓) → (∀𝑥𝜑 ∨ ∃𝑥𝜓)) | ||
Theorem | 19.43 1881 | Theorem 19.43 of [Margaris] p. 90. (Contributed by NM, 12-Mar-1993.) (Proof shortened by Wolf Lammen, 27-Jun-2014.) |
⊢ (∃𝑥(𝜑 ∨ 𝜓) ↔ (∃𝑥𝜑 ∨ ∃𝑥𝜓)) | ||
Theorem | 19.43OLD 1882 | Obsolete proof of 19.43 1881. Do not delete as it is referenced on the mmrecent.html 1881 page and in conventions-labels 30433. (Contributed by NM, 5-Aug-1993.) (Proof modification is discouraged.) (New usage is discouraged.) |
⊢ (∃𝑥(𝜑 ∨ 𝜓) ↔ (∃𝑥𝜑 ∨ ∃𝑥𝜓)) | ||
Theorem | 19.33 1883 | Theorem 19.33 of [Margaris] p. 90. (Contributed by NM, 12-Mar-1993.) |
⊢ ((∀𝑥𝜑 ∨ ∀𝑥𝜓) → ∀𝑥(𝜑 ∨ 𝜓)) | ||
Theorem | 19.33b 1884 | The antecedent provides a condition implying the converse of 19.33 1883. (Contributed by NM, 27-Mar-2004.) (Proof shortened by Andrew Salmon, 25-May-2011.) (Proof shortened by Wolf Lammen, 5-Jul-2014.) |
⊢ (¬ (∃𝑥𝜑 ∧ ∃𝑥𝜓) → (∀𝑥(𝜑 ∨ 𝜓) ↔ (∀𝑥𝜑 ∨ ∀𝑥𝜓))) | ||
Theorem | 19.40 1885 | Theorem 19.40 of [Margaris] p. 90. (Contributed by NM, 26-May-1993.) |
⊢ (∃𝑥(𝜑 ∧ 𝜓) → (∃𝑥𝜑 ∧ ∃𝑥𝜓)) | ||
Theorem | 19.40-2 1886 | Theorem *11.42 in [WhiteheadRussell] p. 163. Theorem 19.40 of [Margaris] p. 90 with two quantifiers. (Contributed by Andrew Salmon, 24-May-2011.) |
⊢ (∃𝑥∃𝑦(𝜑 ∧ 𝜓) → (∃𝑥∃𝑦𝜑 ∧ ∃𝑥∃𝑦𝜓)) | ||
Theorem | 19.40b 1887 | The antecedent provides a condition implying the converse of 19.40 1885. This is to 19.40 1885 what 19.33b 1884 is to 19.33 1883. (Contributed by BJ, 6-May-2019.) (Proof shortened by Wolf Lammen, 13-Nov-2020.) |
⊢ ((∀𝑥𝜑 ∨ ∀𝑥𝜓) → ((∃𝑥𝜑 ∧ ∃𝑥𝜓) ↔ ∃𝑥(𝜑 ∧ 𝜓))) | ||
Theorem | albiim 1888 | Split a biconditional and distribute quantifier. (Contributed by NM, 18-Aug-1993.) |
⊢ (∀𝑥(𝜑 ↔ 𝜓) ↔ (∀𝑥(𝜑 → 𝜓) ∧ ∀𝑥(𝜓 → 𝜑))) | ||
Theorem | 2albiim 1889 | Split a biconditional and distribute two quantifiers. (Contributed by NM, 3-Feb-2005.) |
⊢ (∀𝑥∀𝑦(𝜑 ↔ 𝜓) ↔ (∀𝑥∀𝑦(𝜑 → 𝜓) ∧ ∀𝑥∀𝑦(𝜓 → 𝜑))) | ||
Theorem | exintrbi 1890 | Add/remove a conjunct in the scope of an existential quantifier. (Contributed by Raph Levien, 3-Jul-2006.) |
⊢ (∀𝑥(𝜑 → 𝜓) → (∃𝑥𝜑 ↔ ∃𝑥(𝜑 ∧ 𝜓))) | ||
Theorem | exintr 1891 | Introduce a conjunct in the scope of an existential quantifier. (Contributed by NM, 11-Aug-1993.) (Proof shortened by BJ, 16-Sep-2022.) |
⊢ (∀𝑥(𝜑 → 𝜓) → (∃𝑥𝜑 → ∃𝑥(𝜑 ∧ 𝜓))) | ||
Theorem | alsyl 1892 | Universally quantified and uncurried (imported) form of syllogism. Theorem *10.3 in [WhiteheadRussell] p. 150. (Contributed by Andrew Salmon, 8-Jun-2011.) |
⊢ ((∀𝑥(𝜑 → 𝜓) ∧ ∀𝑥(𝜓 → 𝜒)) → ∀𝑥(𝜑 → 𝜒)) | ||
Theorem | nfimd 1893 | If in a context 𝑥 is not free in 𝜓 and 𝜒, then it is not free in (𝜓 → 𝜒). Deduction form of nfim 1895. (Contributed by Mario Carneiro, 24-Sep-2016.) (Proof shortened by Wolf Lammen, 30-Dec-2017.) df-nf 1782 changed. (Revised by Wolf Lammen, 18-Sep-2021.) Eliminate curried form of nfimt 1894. (Revised by Wolf Lammen, 10-Jul-2022.) |
⊢ (𝜑 → Ⅎ𝑥𝜓) & ⊢ (𝜑 → Ⅎ𝑥𝜒) ⇒ ⊢ (𝜑 → Ⅎ𝑥(𝜓 → 𝜒)) | ||
Theorem | nfimt 1894 | Closed form of nfim 1895 and nfimd 1893. (Contributed by BJ, 20-Oct-2021.) Eliminate curried form, former name nfimt2. (Revised by Wolf Lammen, 6-Jul-2022.) |
⊢ ((Ⅎ𝑥𝜑 ∧ Ⅎ𝑥𝜓) → Ⅎ𝑥(𝜑 → 𝜓)) | ||
Theorem | nfim 1895 | If 𝑥 is not free in 𝜑 and 𝜓, then it is not free in (𝜑 → 𝜓). Inference associated with nfimt 1894. (Contributed by Mario Carneiro, 11-Aug-2016.) (Proof shortened by Wolf Lammen, 2-Jan-2018.) df-nf 1782 changed. (Revised by Wolf Lammen, 17-Sep-2021.) |
⊢ Ⅎ𝑥𝜑 & ⊢ Ⅎ𝑥𝜓 ⇒ ⊢ Ⅎ𝑥(𝜑 → 𝜓) | ||
Theorem | nfand 1896 | If in a context 𝑥 is not free in 𝜓 and 𝜒, then it is not free in (𝜓 ∧ 𝜒). (Contributed by Mario Carneiro, 7-Oct-2016.) |
⊢ (𝜑 → Ⅎ𝑥𝜓) & ⊢ (𝜑 → Ⅎ𝑥𝜒) ⇒ ⊢ (𝜑 → Ⅎ𝑥(𝜓 ∧ 𝜒)) | ||
Theorem | nf3and 1897 | Deduction form of bound-variable hypothesis builder nf3an 1900. (Contributed by NM, 17-Feb-2013.) (Revised by Mario Carneiro, 16-Oct-2016.) |
⊢ (𝜑 → Ⅎ𝑥𝜓) & ⊢ (𝜑 → Ⅎ𝑥𝜒) & ⊢ (𝜑 → Ⅎ𝑥𝜃) ⇒ ⊢ (𝜑 → Ⅎ𝑥(𝜓 ∧ 𝜒 ∧ 𝜃)) | ||
Theorem | nfan 1898 | If 𝑥 is not free in 𝜑 and 𝜓, then it is not free in (𝜑 ∧ 𝜓). (Contributed by Mario Carneiro, 11-Aug-2016.) (Proof shortened by Wolf Lammen, 13-Jan-2018.) (Proof shortened by Wolf Lammen, 9-Oct-2021.) |
⊢ Ⅎ𝑥𝜑 & ⊢ Ⅎ𝑥𝜓 ⇒ ⊢ Ⅎ𝑥(𝜑 ∧ 𝜓) | ||
Theorem | nfnan 1899 | If 𝑥 is not free in 𝜑 and 𝜓, then it is not free in (𝜑 ⊼ 𝜓). (Contributed by Scott Fenton, 2-Jan-2018.) |
⊢ Ⅎ𝑥𝜑 & ⊢ Ⅎ𝑥𝜓 ⇒ ⊢ Ⅎ𝑥(𝜑 ⊼ 𝜓) | ||
Theorem | nf3an 1900 | If 𝑥 is not free in 𝜑, 𝜓, and 𝜒, then it is not free in (𝜑 ∧ 𝜓 ∧ 𝜒). (Contributed by Mario Carneiro, 11-Aug-2016.) |
⊢ Ⅎ𝑥𝜑 & ⊢ Ⅎ𝑥𝜓 & ⊢ Ⅎ𝑥𝜒 ⇒ ⊢ Ⅎ𝑥(𝜑 ∧ 𝜓 ∧ 𝜒) |
< Previous Next > |
Copyright terms: Public domain | < Previous Next > |