HomeHome Intuitionistic Logic Explorer
Theorem List (p. 16 of 133)
< Previous  Next >
Bad symbols? Try the
GIF version.

Mirrors  >  Metamath Home Page  >  ILE Home Page  >  Theorem List Contents  >  Recent Proofs       This page: Page List

Theorem List for Intuitionistic Logic Explorer - 1501-1600   *Has distinct variable group(s)
TypeLabelDescription
Statement
 
Theoremalimd 1501 Deduction from Theorem 19.20 of [Margaris] p. 90. (Contributed by Mario Carneiro, 24-Sep-2016.)
𝑥𝜑    &   (𝜑 → (𝜓𝜒))       (𝜑 → (∀𝑥𝜓 → ∀𝑥𝜒))
 
Theoremalrimi 1502 Inference from Theorem 19.21 of [Margaris] p. 90. (Contributed by Mario Carneiro, 24-Sep-2016.)
𝑥𝜑    &   (𝜑𝜓)       (𝜑 → ∀𝑥𝜓)
 
Theoremnfd 1503 Deduce that 𝑥 is not free in 𝜓 in a context. (Contributed by Mario Carneiro, 24-Sep-2016.)
𝑥𝜑    &   (𝜑 → (𝜓 → ∀𝑥𝜓))       (𝜑 → Ⅎ𝑥𝜓)
 
Theoremnfdh 1504 Deduce that 𝑥 is not free in 𝜓 in a context. (Contributed by Mario Carneiro, 24-Sep-2016.)
(𝜑 → ∀𝑥𝜑)    &   (𝜑 → (𝜓 → ∀𝑥𝜓))       (𝜑 → Ⅎ𝑥𝜓)
 
Theoremnfrimi 1505 Moving an antecedent outside . (Contributed by Jim Kingdon, 23-Mar-2018.)
𝑥𝜑    &   𝑥(𝜑𝜓)       (𝜑 → Ⅎ𝑥𝜓)
 
1.3.3  Axiom ax-17 - first use of the $d distinct variable statement
 
Axiomax-17 1506* Axiom to quantify a variable over a formula in which it does not occur. Axiom C5 in [Megill] p. 444 (p. 11 of the preprint). Also appears as Axiom B6 (p. 75) of system S2 of [Tarski] p. 77 and Axiom C5-1 of [Monk2] p. 113.

(Contributed by NM, 5-Aug-1993.)

(𝜑 → ∀𝑥𝜑)
 
Theorema17d 1507* ax-17 1506 with antecedent. (Contributed by NM, 1-Mar-2013.)
(𝜑 → (𝜓 → ∀𝑥𝜓))
 
Theoremnfv 1508* If 𝑥 is not present in 𝜑, then 𝑥 is not free in 𝜑. (Contributed by Mario Carneiro, 11-Aug-2016.)
𝑥𝜑
 
Theoremnfvd 1509* nfv 1508 with antecedent. Useful in proofs of deduction versions of bound-variable hypothesis builders such as nfimd 1564. (Contributed by Mario Carneiro, 6-Oct-2016.)
(𝜑 → Ⅎ𝑥𝜓)
 
1.3.4  Introduce Axiom of Existence
 
Axiomax-i9 1510 Axiom of Existence. One of the equality and substitution axioms of predicate calculus with equality. One thing this axiom tells us is that at least one thing exists (although ax-4 1487 and possibly others also tell us that, i.e. they are not valid in the empty domain of a "free logic"). In this form (not requiring that 𝑥 and 𝑦 be distinct) it was used in an axiom system of Tarski (see Axiom B7' in footnote 1 of [KalishMontague] p. 81.) Another name for this theorem is a9e 1674, which has additional remarks. (Contributed by Mario Carneiro, 31-Jan-2015.)
𝑥 𝑥 = 𝑦
 
Theoremax-9 1511 Derive ax-9 1511 from ax-i9 1510, the modified version for intuitionistic logic. Although ax-9 1511 does hold intuistionistically, in intuitionistic logic it is weaker than ax-i9 1510. (Contributed by NM, 3-Feb-2015.)
¬ ∀𝑥 ¬ 𝑥 = 𝑦
 
Theoremequidqe 1512 equid 1677 with some quantification and negation without using ax-4 1487 or ax-17 1506. (Contributed by NM, 13-Jan-2011.) (Proof shortened by Wolf Lammen, 27-Feb-2014.)
¬ ∀𝑦 ¬ 𝑥 = 𝑥
 
Theoremax4sp1 1513 A special case of ax-4 1487 without using ax-4 1487 or ax-17 1506. (Contributed by NM, 13-Jan-2011.)
(∀𝑦 ¬ 𝑥 = 𝑥 → ¬ 𝑥 = 𝑥)
 
1.3.5  Additional intuitionistic axioms
 
Axiomax-ial 1514 𝑥 is not free in 𝑥𝜑. One of the axioms of predicate logic. (Contributed by Mario Carneiro, 31-Jan-2015.)
(∀𝑥𝜑 → ∀𝑥𝑥𝜑)
 
Axiomax-i5r 1515 Axiom of quantifier collection. (Contributed by Mario Carneiro, 31-Jan-2015.)
((∀𝑥𝜑 → ∀𝑥𝜓) → ∀𝑥(∀𝑥𝜑𝜓))
 
1.3.6  Predicate calculus including ax-4, without distinct variables
 
Theoremspi 1516 Inference reversing generalization (specialization). (Contributed by NM, 5-Aug-1993.)
𝑥𝜑       𝜑
 
Theoremsps 1517 Generalization of antecedent. (Contributed by NM, 5-Aug-1993.)
(𝜑𝜓)       (∀𝑥𝜑𝜓)
 
Theoremspsd 1518 Deduction generalizing antecedent. (Contributed by NM, 17-Aug-1994.)
(𝜑 → (𝜓𝜒))       (𝜑 → (∀𝑥𝜓𝜒))
 
Theoremnfbidf 1519 An equality theorem for effectively not free. (Contributed by Mario Carneiro, 4-Oct-2016.)
𝑥𝜑    &   (𝜑 → (𝜓𝜒))       (𝜑 → (Ⅎ𝑥𝜓 ↔ Ⅎ𝑥𝜒))
 
Theoremhba1 1520 𝑥 is not free in 𝑥𝜑. Example in Appendix in [Megill] p. 450 (p. 19 of the preprint). Also Lemma 22 of [Monk2] p. 114. (Contributed by NM, 5-Aug-1993.)
(∀𝑥𝜑 → ∀𝑥𝑥𝜑)
 
Theoremnfa1 1521 𝑥 is not free in 𝑥𝜑. (Contributed by Mario Carneiro, 11-Aug-2016.)
𝑥𝑥𝜑
 
Theorema5i 1522 Inference generalizing a consequent. (Contributed by NM, 5-Aug-1993.)
(∀𝑥𝜑𝜓)       (∀𝑥𝜑 → ∀𝑥𝜓)
 
Theoremnfnf1 1523 𝑥 is not free in 𝑥𝜑. (Contributed by Mario Carneiro, 11-Aug-2016.)
𝑥𝑥𝜑
 
Theoremhbim 1524 If 𝑥 is not free in 𝜑 and 𝜓, it is not free in (𝜑𝜓). (Contributed by NM, 5-Aug-1993.) (Proof shortened by O'Cat, 3-Mar-2008.) (Revised by Mario Carneiro, 2-Feb-2015.)
(𝜑 → ∀𝑥𝜑)    &   (𝜓 → ∀𝑥𝜓)       ((𝜑𝜓) → ∀𝑥(𝜑𝜓))
 
Theoremhbor 1525 If 𝑥 is not free in 𝜑 and 𝜓, it is not free in (𝜑𝜓). (Contributed by NM, 5-Aug-1993.) (Revised by NM, 2-Feb-2015.)
(𝜑 → ∀𝑥𝜑)    &   (𝜓 → ∀𝑥𝜓)       ((𝜑𝜓) → ∀𝑥(𝜑𝜓))
 
Theoremhban 1526 If 𝑥 is not free in 𝜑 and 𝜓, it is not free in (𝜑𝜓). (Contributed by NM, 5-Aug-1993.) (Proof shortened by Mario Carneiro, 2-Feb-2015.)
(𝜑 → ∀𝑥𝜑)    &   (𝜓 → ∀𝑥𝜓)       ((𝜑𝜓) → ∀𝑥(𝜑𝜓))
 
Theoremhbbi 1527 If 𝑥 is not free in 𝜑 and 𝜓, it is not free in (𝜑𝜓). (Contributed by NM, 5-Aug-1993.)
(𝜑 → ∀𝑥𝜑)    &   (𝜓 → ∀𝑥𝜓)       ((𝜑𝜓) → ∀𝑥(𝜑𝜓))
 
Theoremhb3or 1528 If 𝑥 is not free in 𝜑, 𝜓, and 𝜒, it is not free in (𝜑𝜓𝜒). (Contributed by NM, 14-Sep-2003.)
(𝜑 → ∀𝑥𝜑)    &   (𝜓 → ∀𝑥𝜓)    &   (𝜒 → ∀𝑥𝜒)       ((𝜑𝜓𝜒) → ∀𝑥(𝜑𝜓𝜒))
 
Theoremhb3an 1529 If 𝑥 is not free in 𝜑, 𝜓, and 𝜒, it is not free in (𝜑𝜓𝜒). (Contributed by NM, 14-Sep-2003.)
(𝜑 → ∀𝑥𝜑)    &   (𝜓 → ∀𝑥𝜓)    &   (𝜒 → ∀𝑥𝜒)       ((𝜑𝜓𝜒) → ∀𝑥(𝜑𝜓𝜒))
 
Theoremhba2 1530 Lemma 24 of [Monk2] p. 114. (Contributed by NM, 29-May-2008.)
(∀𝑦𝑥𝜑 → ∀𝑥𝑦𝑥𝜑)
 
Theoremhbia1 1531 Lemma 23 of [Monk2] p. 114. (Contributed by NM, 29-May-2008.)
((∀𝑥𝜑 → ∀𝑥𝜓) → ∀𝑥(∀𝑥𝜑 → ∀𝑥𝜓))
 
Theorem19.3h 1532 A wff may be quantified with a variable not free in it. Theorem 19.3 of [Margaris] p. 89. (Contributed by NM, 5-Aug-1993.) (Revised by NM, 21-May-2007.)
(𝜑 → ∀𝑥𝜑)       (∀𝑥𝜑𝜑)
 
Theorem19.3 1533 A wff may be quantified with a variable not free in it. Theorem 19.3 of [Margaris] p. 89. (Contributed by NM, 5-Aug-1993.) (Revised by Mario Carneiro, 24-Sep-2016.)
𝑥𝜑       (∀𝑥𝜑𝜑)
 
Theorem19.16 1534 Theorem 19.16 of [Margaris] p. 90. (Contributed by NM, 12-Mar-1993.)
𝑥𝜑       (∀𝑥(𝜑𝜓) → (𝜑 ↔ ∀𝑥𝜓))
 
Theorem19.17 1535 Theorem 19.17 of [Margaris] p. 90. (Contributed by NM, 12-Mar-1993.)
𝑥𝜓       (∀𝑥(𝜑𝜓) → (∀𝑥𝜑𝜓))
 
Theorem19.21h 1536 Theorem 19.21 of [Margaris] p. 90. The hypothesis can be thought of as "𝑥 is not free in 𝜑." New proofs should use 19.21 1562 instead. (Contributed by NM, 5-Aug-1993.) (New usage is discouraged.)
(𝜑 → ∀𝑥𝜑)       (∀𝑥(𝜑𝜓) ↔ (𝜑 → ∀𝑥𝜓))
 
Theorem19.21bi 1537 Inference from Theorem 19.21 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.)
(𝜑 → ∀𝑥𝜓)       (𝜑𝜓)
 
Theorem19.21bbi 1538 Inference removing double quantifier. (Contributed by NM, 20-Apr-1994.)
(𝜑 → ∀𝑥𝑦𝜓)       (𝜑𝜓)
 
Theorem19.27h 1539 Theorem 19.27 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.)
(𝜓 → ∀𝑥𝜓)       (∀𝑥(𝜑𝜓) ↔ (∀𝑥𝜑𝜓))
 
Theorem19.27 1540 Theorem 19.27 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.)
𝑥𝜓       (∀𝑥(𝜑𝜓) ↔ (∀𝑥𝜑𝜓))
 
Theorem19.28h 1541 Theorem 19.28 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.)
(𝜑 → ∀𝑥𝜑)       (∀𝑥(𝜑𝜓) ↔ (𝜑 ∧ ∀𝑥𝜓))
 
Theorem19.28 1542 Theorem 19.28 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.)
𝑥𝜑       (∀𝑥(𝜑𝜓) ↔ (𝜑 ∧ ∀𝑥𝜓))
 
Theoremnfan1 1543 A closed form of nfan 1544. (Contributed by Mario Carneiro, 3-Oct-2016.)
𝑥𝜑    &   (𝜑 → Ⅎ𝑥𝜓)       𝑥(𝜑𝜓)
 
Theoremnfan 1544 If 𝑥 is not free in 𝜑 and 𝜓, it is not free in (𝜑𝜓). (Contributed by Mario Carneiro, 11-Aug-2016.) (Proof shortened by Wolf Lammen, 13-Jan-2018.)
𝑥𝜑    &   𝑥𝜓       𝑥(𝜑𝜓)
 
Theoremnf3an 1545 If 𝑥 is not free in 𝜑, 𝜓, and 𝜒, it is not free in (𝜑𝜓𝜒). (Contributed by Mario Carneiro, 11-Aug-2016.)
𝑥𝜑    &   𝑥𝜓    &   𝑥𝜒       𝑥(𝜑𝜓𝜒)
 
Theoremnford 1546 If in a context 𝑥 is not free in 𝜓 and 𝜒, it is not free in (𝜓𝜒). (Contributed by Jim Kingdon, 29-Oct-2019.)
(𝜑 → Ⅎ𝑥𝜓)    &   (𝜑 → Ⅎ𝑥𝜒)       (𝜑 → Ⅎ𝑥(𝜓𝜒))
 
Theoremnfand 1547 If in a context 𝑥 is not free in 𝜓 and 𝜒, it is not free in (𝜓𝜒). (Contributed by Mario Carneiro, 7-Oct-2016.)
(𝜑 → Ⅎ𝑥𝜓)    &   (𝜑 → Ⅎ𝑥𝜒)       (𝜑 → Ⅎ𝑥(𝜓𝜒))
 
Theoremnf3and 1548 Deduction form of bound-variable hypothesis builder nf3an 1545. (Contributed by NM, 17-Feb-2013.) (Revised by Mario Carneiro, 16-Oct-2016.)
(𝜑 → Ⅎ𝑥𝜓)    &   (𝜑 → Ⅎ𝑥𝜒)    &   (𝜑 → Ⅎ𝑥𝜃)       (𝜑 → Ⅎ𝑥(𝜓𝜒𝜃))
 
Theoremhbim1 1549 A closed form of hbim 1524. (Contributed by NM, 5-Aug-1993.)
(𝜑 → ∀𝑥𝜑)    &   (𝜑 → (𝜓 → ∀𝑥𝜓))       ((𝜑𝜓) → ∀𝑥(𝜑𝜓))
 
Theoremnfim1 1550 A closed form of nfim 1551. (Contributed by NM, 5-Aug-1993.) (Revised by Mario Carneiro, 24-Sep-2016.) (Proof shortened by Wolf Lammen, 2-Jan-2018.)
𝑥𝜑    &   (𝜑 → Ⅎ𝑥𝜓)       𝑥(𝜑𝜓)
 
Theoremnfim 1551 If 𝑥 is not free in 𝜑 and 𝜓, it is not free in (𝜑𝜓). (Contributed by Mario Carneiro, 11-Aug-2016.) (Proof shortened by Wolf Lammen, 2-Jan-2018.)
𝑥𝜑    &   𝑥𝜓       𝑥(𝜑𝜓)
 
Theoremhbimd 1552 Deduction form of bound-variable hypothesis builder hbim 1524. (Contributed by NM, 1-Jan-2002.) (Revised by NM, 2-Feb-2015.)
(𝜑 → ∀𝑥𝜑)    &   (𝜑 → (𝜓 → ∀𝑥𝜓))    &   (𝜑 → (𝜒 → ∀𝑥𝜒))       (𝜑 → ((𝜓𝜒) → ∀𝑥(𝜓𝜒)))
 
Theoremnfor 1553 If 𝑥 is not free in 𝜑 and 𝜓, it is not free in (𝜑𝜓). (Contributed by Jim Kingdon, 11-Mar-2018.)
𝑥𝜑    &   𝑥𝜓       𝑥(𝜑𝜓)
 
Theoremhbbid 1554 Deduction form of bound-variable hypothesis builder hbbi 1527. (Contributed by NM, 1-Jan-2002.)
(𝜑 → ∀𝑥𝜑)    &   (𝜑 → (𝜓 → ∀𝑥𝜓))    &   (𝜑 → (𝜒 → ∀𝑥𝜒))       (𝜑 → ((𝜓𝜒) → ∀𝑥(𝜓𝜒)))
 
Theoremnfal 1555 If 𝑥 is not free in 𝜑, it is not free in 𝑦𝜑. (Contributed by Mario Carneiro, 11-Aug-2016.)
𝑥𝜑       𝑥𝑦𝜑
 
Theoremnfnf 1556 If 𝑥 is not free in 𝜑, it is not free in 𝑦𝜑. (Contributed by Mario Carneiro, 11-Aug-2016.) (Proof shortened by Wolf Lammen, 30-Dec-2017.)
𝑥𝜑       𝑥𝑦𝜑
 
Theoremnfalt 1557 Closed form of nfal 1555. (Contributed by Jim Kingdon, 11-May-2018.)
(∀𝑦𝑥𝜑 → Ⅎ𝑥𝑦𝜑)
 
Theoremnfa2 1558 Lemma 24 of [Monk2] p. 114. (Contributed by Mario Carneiro, 24-Sep-2016.)
𝑥𝑦𝑥𝜑
 
Theoremnfia1 1559 Lemma 23 of [Monk2] p. 114. (Contributed by Mario Carneiro, 24-Sep-2016.)
𝑥(∀𝑥𝜑 → ∀𝑥𝜓)
 
Theorem19.21ht 1560 Closed form of Theorem 19.21 of [Margaris] p. 90. (Contributed by NM, 27-May-1997.) (New usage is discouraged.)
(∀𝑥(𝜑 → ∀𝑥𝜑) → (∀𝑥(𝜑𝜓) ↔ (𝜑 → ∀𝑥𝜓)))
 
Theorem19.21t 1561 Closed form of Theorem 19.21 of [Margaris] p. 90. (Contributed by NM, 27-May-1997.)
(Ⅎ𝑥𝜑 → (∀𝑥(𝜑𝜓) ↔ (𝜑 → ∀𝑥𝜓)))
 
Theorem19.21 1562 Theorem 19.21 of [Margaris] p. 90. The hypothesis can be thought of as "𝑥 is not free in 𝜑." (Contributed by NM, 5-Aug-1993.) (Revised by Mario Carneiro, 24-Sep-2016.)
𝑥𝜑       (∀𝑥(𝜑𝜓) ↔ (𝜑 → ∀𝑥𝜓))
 
Theoremstdpc5 1563 An axiom scheme of standard predicate calculus that emulates Axiom 5 of [Mendelson] p. 69. The hypothesis 𝑥𝜑 can be thought of as emulating "𝑥 is not free in 𝜑." With this definition, the meaning of "not free" is less restrictive than the usual textbook definition; for example 𝑥 would not (for us) be free in 𝑥 = 𝑥 by nfequid 1678. This theorem scheme can be proved as a metatheorem of Mendelson's axiom system, even though it is slightly stronger than his Axiom 5. (Contributed by NM, 22-Sep-1993.) (Revised by Mario Carneiro, 12-Oct-2016.) (Proof shortened by Wolf Lammen, 1-Jan-2018.)
𝑥𝜑       (∀𝑥(𝜑𝜓) → (𝜑 → ∀𝑥𝜓))
 
Theoremnfimd 1564 If in a context 𝑥 is not free in 𝜓 and 𝜒, then it is not free in (𝜓𝜒). (Contributed by Mario Carneiro, 24-Sep-2016.) (Proof shortened by Wolf Lammen, 30-Dec-2017.)
(𝜑 → Ⅎ𝑥𝜓)    &   (𝜑 → Ⅎ𝑥𝜒)       (𝜑 → Ⅎ𝑥(𝜓𝜒))
 
Theoremaaanh 1565 Rearrange universal quantifiers. (Contributed by NM, 12-Aug-1993.)
(𝜑 → ∀𝑦𝜑)    &   (𝜓 → ∀𝑥𝜓)       (∀𝑥𝑦(𝜑𝜓) ↔ (∀𝑥𝜑 ∧ ∀𝑦𝜓))
 
Theoremaaan 1566 Rearrange universal quantifiers. (Contributed by NM, 12-Aug-1993.)
𝑦𝜑    &   𝑥𝜓       (∀𝑥𝑦(𝜑𝜓) ↔ (∀𝑥𝜑 ∧ ∀𝑦𝜓))
 
Theoremnfbid 1567 If in a context 𝑥 is not free in 𝜓 and 𝜒, then it is not free in (𝜓𝜒). (Contributed by Mario Carneiro, 24-Sep-2016.) (Proof shortened by Wolf Lammen, 29-Dec-2017.)
(𝜑 → Ⅎ𝑥𝜓)    &   (𝜑 → Ⅎ𝑥𝜒)       (𝜑 → Ⅎ𝑥(𝜓𝜒))
 
Theoremnfbi 1568 If 𝑥 is not free in 𝜑 and 𝜓, then it is not free in (𝜑𝜓). (Contributed by Mario Carneiro, 11-Aug-2016.) (Proof shortened by Wolf Lammen, 2-Jan-2018.)
𝑥𝜑    &   𝑥𝜓       𝑥(𝜑𝜓)
 
1.3.7  The existential quantifier
 
Theorem19.8a 1569 If a wff is true, then it is true for at least one instance. Special case of Theorem 19.8 of [Margaris] p. 89. (Contributed by NM, 5-Aug-1993.)
(𝜑 → ∃𝑥𝜑)
 
Theorem19.8ad 1570 If a wff is true, it is true for at least one instance. Deduction form of 19.8a 1569. (Contributed by DAW, 13-Feb-2017.)
(𝜑𝜓)       (𝜑 → ∃𝑥𝜓)
 
Theorem19.23bi 1571 Inference from Theorem 19.23 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.)
(∃𝑥𝜑𝜓)       (𝜑𝜓)
 
Theoremexlimih 1572 Inference from Theorem 19.23 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.) (Proof shortened by Andrew Salmon, 13-May-2011.)
(𝜓 → ∀𝑥𝜓)    &   (𝜑𝜓)       (∃𝑥𝜑𝜓)
 
Theoremexlimi 1573 Inference from Theorem 19.23 of [Margaris] p. 90. (Contributed by Mario Carneiro, 24-Sep-2016.)
𝑥𝜓    &   (𝜑𝜓)       (∃𝑥𝜑𝜓)
 
Theoremexlimd2 1574 Deduction from Theorem 19.23 of [Margaris] p. 90. Similar to exlimdh 1575 but with one slightly different hypothesis. (Contributed by Jim Kingdon, 30-Dec-2017.)
(𝜑 → ∀𝑥𝜑)    &   (𝜑 → (𝜒 → ∀𝑥𝜒))    &   (𝜑 → (𝜓𝜒))       (𝜑 → (∃𝑥𝜓𝜒))
 
Theoremexlimdh 1575 Deduction from Theorem 19.23 of [Margaris] p. 90. (Contributed by NM, 28-Jan-1997.)
(𝜑 → ∀𝑥𝜑)    &   (𝜒 → ∀𝑥𝜒)    &   (𝜑 → (𝜓𝜒))       (𝜑 → (∃𝑥𝜓𝜒))
 
Theoremexlimd 1576 Deduction from Theorem 19.9 of [Margaris] p. 89. (Contributed by Mario Carneiro, 24-Sep-2016.) (Proof rewritten by Jim Kingdon, 18-Jun-2018.)
𝑥𝜑    &   𝑥𝜒    &   (𝜑 → (𝜓𝜒))       (𝜑 → (∃𝑥𝜓𝜒))
 
Theoremexlimiv 1577* Inference from Theorem 19.23 of [Margaris] p. 90.

This inference, along with our many variants is used to implement a metatheorem called "Rule C" that is given in many logic textbooks. See, for example, Rule C in [Mendelson] p. 81, Rule C in [Margaris] p. 40, or Rule C in Hirst and Hirst's A Primer for Logic and Proof p. 59 (PDF p. 65) at http://www.mathsci.appstate.edu/~jlh/primer/hirst.pdf.

In informal proofs, the statement "Let C be an element such that..." almost always means an implicit application of Rule C.

In essence, Rule C states that if we can prove that some element 𝑥 exists satisfying a wff, i.e. 𝑥𝜑(𝑥) where 𝜑(𝑥) has 𝑥 free, then we can use 𝜑( C ) as a hypothesis for the proof where C is a new (ficticious) constant not appearing previously in the proof, nor in any axioms used, nor in the theorem to be proved. The purpose of Rule C is to get rid of the existential quantifier.

We cannot do this in Metamath directly. Instead, we use the original 𝜑 (containing 𝑥) as an antecedent for the main part of the proof. We eventually arrive at (𝜑𝜓) where 𝜓 is the theorem to be proved and does not contain 𝑥. Then we apply exlimiv 1577 to arrive at (∃𝑥𝜑𝜓). Finally, we separately prove 𝑥𝜑 and detach it with modus ponens ax-mp 5 to arrive at the final theorem 𝜓. (Contributed by NM, 5-Aug-1993.) (Revised by NM, 25-Jul-2012.)

(𝜑𝜓)       (∃𝑥𝜑𝜓)
 
Theoremexim 1578 Theorem 19.22 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.) (Proof shortened by Wolf Lammen, 4-Jul-2014.)
(∀𝑥(𝜑𝜓) → (∃𝑥𝜑 → ∃𝑥𝜓))
 
Theoremeximi 1579 Inference adding existential quantifier to antecedent and consequent. (Contributed by NM, 5-Aug-1993.)
(𝜑𝜓)       (∃𝑥𝜑 → ∃𝑥𝜓)
 
Theorem2eximi 1580 Inference adding 2 existential quantifiers to antecedent and consequent. (Contributed by NM, 3-Feb-2005.)
(𝜑𝜓)       (∃𝑥𝑦𝜑 → ∃𝑥𝑦𝜓)
 
Theoremeximii 1581 Inference associated with eximi 1579. (Contributed by BJ, 3-Feb-2018.)
𝑥𝜑    &   (𝜑𝜓)       𝑥𝜓
 
Theoremalinexa 1582 A transformation of quantifiers and logical connectives. (Contributed by NM, 19-Aug-1993.)
(∀𝑥(𝜑 → ¬ 𝜓) ↔ ¬ ∃𝑥(𝜑𝜓))
 
Theoremexbi 1583 Theorem 19.18 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.)
(∀𝑥(𝜑𝜓) → (∃𝑥𝜑 ↔ ∃𝑥𝜓))
 
Theoremexbii 1584 Inference adding existential quantifier to both sides of an equivalence. (Contributed by NM, 24-May-1994.)
(𝜑𝜓)       (∃𝑥𝜑 ↔ ∃𝑥𝜓)
 
Theorem2exbii 1585 Inference adding 2 existential quantifiers to both sides of an equivalence. (Contributed by NM, 16-Mar-1995.)
(𝜑𝜓)       (∃𝑥𝑦𝜑 ↔ ∃𝑥𝑦𝜓)
 
Theorem3exbii 1586 Inference adding 3 existential quantifiers to both sides of an equivalence. (Contributed by NM, 2-May-1995.)
(𝜑𝜓)       (∃𝑥𝑦𝑧𝜑 ↔ ∃𝑥𝑦𝑧𝜓)
 
Theoremexancom 1587 Commutation of conjunction inside an existential quantifier. (Contributed by NM, 18-Aug-1993.)
(∃𝑥(𝜑𝜓) ↔ ∃𝑥(𝜓𝜑))
 
Theoremalrimdd 1588 Deduction from Theorem 19.21 of [Margaris] p. 90. (Contributed by Mario Carneiro, 24-Sep-2016.)
𝑥𝜑    &   (𝜑 → Ⅎ𝑥𝜓)    &   (𝜑 → (𝜓𝜒))       (𝜑 → (𝜓 → ∀𝑥𝜒))
 
Theoremalrimd 1589 Deduction from Theorem 19.21 of [Margaris] p. 90. (Contributed by Mario Carneiro, 24-Sep-2016.)
𝑥𝜑    &   𝑥𝜓    &   (𝜑 → (𝜓𝜒))       (𝜑 → (𝜓 → ∀𝑥𝜒))
 
Theoremeximdh 1590 Deduction from Theorem 19.22 of [Margaris] p. 90. (Contributed by NM, 20-May-1996.)
(𝜑 → ∀𝑥𝜑)    &   (𝜑 → (𝜓𝜒))       (𝜑 → (∃𝑥𝜓 → ∃𝑥𝜒))
 
Theoremeximd 1591 Deduction from Theorem 19.22 of [Margaris] p. 90. (Contributed by Mario Carneiro, 24-Sep-2016.)
𝑥𝜑    &   (𝜑 → (𝜓𝜒))       (𝜑 → (∃𝑥𝜓 → ∃𝑥𝜒))
 
Theoremnexd 1592 Deduction for generalization rule for negated wff. (Contributed by NM, 2-Jan-2002.)
(𝜑 → ∀𝑥𝜑)    &   (𝜑 → ¬ 𝜓)       (𝜑 → ¬ ∃𝑥𝜓)
 
Theoremexbidh 1593 Formula-building rule for existential quantifier (deduction form). (Contributed by NM, 5-Aug-1993.)
(𝜑 → ∀𝑥𝜑)    &   (𝜑 → (𝜓𝜒))       (𝜑 → (∃𝑥𝜓 ↔ ∃𝑥𝜒))
 
Theoremalbid 1594 Formula-building rule for universal quantifier (deduction form). (Contributed by Mario Carneiro, 24-Sep-2016.)
𝑥𝜑    &   (𝜑 → (𝜓𝜒))       (𝜑 → (∀𝑥𝜓 ↔ ∀𝑥𝜒))
 
Theoremexbid 1595 Formula-building rule for existential quantifier (deduction form). (Contributed by Mario Carneiro, 24-Sep-2016.)
𝑥𝜑    &   (𝜑 → (𝜓𝜒))       (𝜑 → (∃𝑥𝜓 ↔ ∃𝑥𝜒))
 
Theoremexsimpl 1596 Simplification of an existentially quantified conjunction. (Contributed by Rodolfo Medina, 25-Sep-2010.) (Proof shortened by Andrew Salmon, 29-Jun-2011.)
(∃𝑥(𝜑𝜓) → ∃𝑥𝜑)
 
Theoremexsimpr 1597 Simplification of an existentially quantified conjunction. (Contributed by Rodolfo Medina, 25-Sep-2010.) (Proof shortened by Andrew Salmon, 29-Jun-2011.)
(∃𝑥(𝜑𝜓) → ∃𝑥𝜓)
 
Theoremalexdc 1598 Theorem 19.6 of [Margaris] p. 89, given a decidability condition. The forward direction holds for all propositions, as seen at alexim 1624. (Contributed by Jim Kingdon, 2-Jun-2018.)
(∀𝑥DECID 𝜑 → (∀𝑥𝜑 ↔ ¬ ∃𝑥 ¬ 𝜑))
 
Theorem19.29 1599 Theorem 19.29 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.) (Proof shortened by Andrew Salmon, 13-May-2011.)
((∀𝑥𝜑 ∧ ∃𝑥𝜓) → ∃𝑥(𝜑𝜓))
 
Theorem19.29r 1600 Variation of Theorem 19.29 of [Margaris] p. 90. (Contributed by NM, 18-Aug-1993.)
((∃𝑥𝜑 ∧ ∀𝑥𝜓) → ∃𝑥(𝜑𝜓))
    < Previous  Next >

Page List
Jump to page: Contents  1 1-100 2 101-200 3 201-300 4 301-400 5 401-500 6 501-600 7 601-700 8 701-800 9 801-900 10 901-1000 11 1001-1100 12 1101-1200 13 1201-1300 14 1301-1400 15 1401-1500 16 1501-1600 17 1601-1700 18 1701-1800 19 1801-1900 20 1901-2000 21 2001-2100 22 2101-2200 23 2201-2300 24 2301-2400 25 2401-2500 26 2501-2600 27 2601-2700 28 2701-2800 29 2801-2900 30 2901-3000 31 3001-3100 32 3101-3200 33 3201-3300 34 3301-3400 35 3401-3500 36 3501-3600 37 3601-3700 38 3701-3800 39 3801-3900 40 3901-4000 41 4001-4100 42 4101-4200 43 4201-4300 44 4301-4400 45 4401-4500 46 4501-4600 47 4601-4700 48 4701-4800 49 4801-4900 50 4901-5000 51 5001-5100 52 5101-5200 53 5201-5300 54 5301-5400 55 5401-5500 56 5501-5600 57 5601-5700 58 5701-5800 59 5801-5900 60 5901-6000 61 6001-6100 62 6101-6200 63 6201-6300 64 6301-6400 65 6401-6500 66 6501-6600 67 6601-6700 68 6701-6800 69 6801-6900 70 6901-7000 71 7001-7100 72 7101-7200 73 7201-7300 74 7301-7400 75 7401-7500 76 7501-7600 77 7601-7700 78 7701-7800 79 7801-7900 80 7901-8000 81 8001-8100 82 8101-8200 83 8201-8300 84 8301-8400 85 8401-8500 86 8501-8600 87 8601-8700 88 8701-8800 89 8801-8900 90 8901-9000 91 9001-9100 92 9101-9200 93 9201-9300 94 9301-9400 95 9401-9500 96 9501-9600 97 9601-9700 98 9701-9800 99 9801-9900 100 9901-10000 101 10001-10100 102 10101-10200 103 10201-10300 104 10301-10400 105 10401-10500 106 10501-10600 107 10601-10700 108 10701-10800 109 10801-10900 110 10901-11000 111 11001-11100 112 11101-11200 113 11201-11300 114 11301-11400 115 11401-11500 116 11501-11600 117 11601-11700 118 11701-11800 119 11801-11900 120 11901-12000 121 12001-12100 122 12101-12200 123 12201-12300 124 12301-12400 125 12401-12500 126 12501-12600 127 12601-12700 128 12701-12800 129 12801-12900 130 12901-13000 131 13001-13100 132 13101-13200 133 13201-13250
  Copyright terms: Public domain < Previous  Next >