HomeHome Intuitionistic Logic Explorer
Theorem List (p. 15 of 102)
< Previous  Next >
Browser slow? Try the
Unicode version.

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

Theorem List for Intuitionistic Logic Explorer - 1401-1500   *Has distinct variable group(s)
TypeLabelDescription
Statement
 
Theoremsp 1401 Specialization. Another name for ax-4 1400. (Contributed by NM, 21-May-2008.)
 |-  ( A. x ph  -> 
 ph )
 
Theoremax-12 1402 Rederive the original version of the axiom from ax-i12 1398. (Contributed by Mario Carneiro, 3-Feb-2015.)
 |-  ( -.  A. z  z  =  x  ->  ( -.  A. z  z  =  y  ->  ( x  =  y  ->  A. z  x  =  y ) ) )
 
Theoremax12or 1403 Another name for ax-i12 1398. (Contributed by NM, 3-Feb-2015.)
 |-  ( A. z  z  =  x  \/  ( A. z  z  =  y  \/  A. z ( x  =  y  ->  A. z  x  =  y ) ) )
 
Axiomax-13 1404 Axiom of Equality. One of the equality and substitution axioms for a non-logical predicate in our predicate calculus with equality. It substitutes equal variables into the left-hand side of the  e. binary predicate. Axiom scheme C12' in [Megill] p. 448 (p. 16 of the preprint). It is a special case of Axiom B8 (p. 75) of system S2 of [Tarski] p. 77. "Non-logical" means that the predicate is not a primitive of predicate calculus proper but instead is an extension to it. "Binary" means that the predicate has two arguments. In a system of predicate calculus with equality, like ours, equality is not usually considered to be a non-logical predicate. In systems of predicate calculus without equality, it typically would be. (Contributed by NM, 5-Aug-1993.)
 |-  ( x  =  y 
 ->  ( x  e.  z  ->  y  e.  z ) )
 
Axiomax-14 1405 Axiom of Equality. One of the equality and substitution axioms for a non-logical predicate in our predicate calculus with equality. It substitutes equal variables into the right-hand side of the  e. binary predicate. Axiom scheme C13' in [Megill] p. 448 (p. 16 of the preprint). It is a special case of Axiom B8 (p. 75) of system S2 of [Tarski] p. 77. (Contributed by NM, 5-Aug-1993.)
 |-  ( x  =  y 
 ->  ( z  e.  x  ->  z  e.  y ) )
 
Theoremhbequid 1406 Bound-variable hypothesis builder for  x  =  x. This theorem tells us that any variable, including  x, is effectively not free in  x  =  x, even though  x is technically free according to the traditional definition of free variable. (The proof uses only ax-5 1336, ax-8 1395, ax-12 1402, and ax-gen 1338. This shows that this can be proved without ax-9 1424, even though the theorem equid 1589 cannot be. A shorter proof using ax-9 1424 is obtainable from equid 1589 and hbth 1352.) (Contributed by NM, 13-Jan-2011.) (Proof shortened by Wolf Lammen, 23-Mar-2014.)
 |-  ( x  =  x 
 ->  A. y  x  =  x )
 
Theoremaxi12 1407 Proof that ax-i12 1398 follows from ax-bndl 1399. So that we can track which theorems rely on ax-bndl 1399, proofs should reference ax-i12 1398 rather than this theorem. (Contributed by Jim Kingdon, 17-Aug-2018.) (New usage is discouraged). (Proof modification is discouraged.)
 |-  ( A. z  z  =  x  \/  ( A. z  z  =  y  \/  A. z ( x  =  y  ->  A. z  x  =  y ) ) )
 
Theoremalequcom 1408 Commutation law for identical variable specifiers. The antecedent and consequent are true when  x and  y are substituted with the same variable. Lemma L12 in [Megill] p. 445 (p. 12 of the preprint). (Contributed by NM, 5-Aug-1993.)
 |-  ( A. x  x  =  y  ->  A. y  y  =  x )
 
Theoremalequcoms 1409 A commutation rule for identical variable specifiers. (Contributed by NM, 5-Aug-1993.)
 |-  ( A. x  x  =  y  ->  ph )   =>    |-  ( A. y  y  =  x  ->  ph )
 
Theoremnalequcoms 1410 A commutation rule for distinct variable specifiers. (Contributed by NM, 2-Jan-2002.) (Revised by Mario Carneiro, 2-Feb-2015.)
 |-  ( -.  A. x  x  =  y  ->  ph )   =>    |-  ( -.  A. y  y  =  x  ->  ph )
 
Theoremnfr 1411 Consequence of the definition of not-free. (Contributed by Mario Carneiro, 26-Sep-2016.)
 |-  ( F/ x ph  ->  ( ph  ->  A. x ph ) )
 
Theoremnfri 1412 Consequence of the definition of not-free. (Contributed by Mario Carneiro, 11-Aug-2016.)
 |- 
 F/ x ph   =>    |-  ( ph  ->  A. x ph )
 
Theoremnfrd 1413 Consequence of the definition of not-free in a context. (Contributed by Mario Carneiro, 11-Aug-2016.)
 |-  ( ph  ->  F/ x ps )   =>    |-  ( ph  ->  ( ps  ->  A. x ps )
 )
 
Theoremalimd 1414 Deduction from Theorem 19.20 of [Margaris] p. 90. (Contributed by Mario Carneiro, 24-Sep-2016.)
 |- 
 F/ x ph   &    |-  ( ph  ->  ( ps  ->  ch )
 )   =>    |-  ( ph  ->  ( A. x ps  ->  A. x ch ) )
 
Theoremalrimi 1415 Inference from Theorem 19.21 of [Margaris] p. 90. (Contributed by Mario Carneiro, 24-Sep-2016.)
 |- 
 F/ x ph   &    |-  ( ph  ->  ps )   =>    |-  ( ph  ->  A. x ps )
 
Theoremnfd 1416 Deduce that  x is not free in  ps in a context. (Contributed by Mario Carneiro, 24-Sep-2016.)
 |- 
 F/ x ph   &    |-  ( ph  ->  ( ps  ->  A. x ps ) )   =>    |-  ( ph  ->  F/ x ps )
 
Theoremnfdh 1417 Deduce that  x is not free in  ps in a context. (Contributed by Mario Carneiro, 24-Sep-2016.)
 |-  ( ph  ->  A. x ph )   &    |-  ( ph  ->  ( ps  ->  A. x ps ) )   =>    |-  ( ph  ->  F/ x ps )
 
Theoremnfrimi 1418 Moving an antecedent outside  F/. (Contributed by Jim Kingdon, 23-Mar-2018.)
 |- 
 F/ x ph   &    |-  F/ x (
 ph  ->  ps )   =>    |-  ( ph  ->  F/ x ps )
 
1.3.3  Axiom ax-17 - first use of the $d distinct variable statement
 
Axiomax-17 1419* 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.)

 |-  ( ph  ->  A. x ph )
 
Theorema17d 1420* ax-17 1419 with antecedent. (Contributed by NM, 1-Mar-2013.)
 |-  ( ph  ->  ( ps  ->  A. x ps )
 )
 
Theoremnfv 1421* If  x is not present in  ph, then  x is not free in  ph. (Contributed by Mario Carneiro, 11-Aug-2016.)
 |- 
 F/ x ph
 
Theoremnfvd 1422* nfv 1421 with antecedent. Useful in proofs of deduction versions of bound-variable hypothesis builders such as nfimd 1477. (Contributed by Mario Carneiro, 6-Oct-2016.)
 |-  ( ph  ->  F/ x ps )
 
1.3.4  Introduce Axiom of Existence
 
Axiomax-i9 1423 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 1400 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  x and  y 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 1586, which has additional remarks. (Contributed by Mario Carneiro, 31-Jan-2015.)
 |- 
 E. x  x  =  y
 
Theoremax-9 1424 Derive ax-9 1424 from ax-i9 1423, the modified version for intuitionistic logic. Although ax-9 1424 does hold intuistionistically, in intuitionistic logic it is weaker than ax-i9 1423. (Contributed by NM, 3-Feb-2015.)
 |- 
 -.  A. x  -.  x  =  y
 
Theoremequidqe 1425 equid 1589 with some quantification and negation without using ax-4 1400 or ax-17 1419. (Contributed by NM, 13-Jan-2011.) (Proof shortened by Wolf Lammen, 27-Feb-2014.)
 |- 
 -.  A. y  -.  x  =  x
 
Theoremax4sp1 1426 A special case of ax-4 1400 without using ax-4 1400 or ax-17 1419. (Contributed by NM, 13-Jan-2011.)
 |-  ( A. y  -.  x  =  x  ->  -.  x  =  x )
 
1.3.5  Additional intuitionistic axioms
 
Axiomax-ial 1427  x is not free in  A. x ph. One of the axioms of predicate logic. (Contributed by Mario Carneiro, 31-Jan-2015.)
 |-  ( A. x ph  ->  A. x A. x ph )
 
Axiomax-i5r 1428 Axiom of quantifier collection. (Contributed by Mario Carneiro, 31-Jan-2015.)
 |-  ( ( A. x ph 
 ->  A. x ps )  ->  A. x ( A. x ph  ->  ps )
 )
 
1.3.6  Predicate calculus including ax-4, without distinct variables
 
Theoremspi 1429 Inference rule reversing generalization. (Contributed by NM, 5-Aug-1993.)
 |- 
 A. x ph   =>    |-  ph
 
Theoremsps 1430 Generalization of antecedent. (Contributed by NM, 5-Aug-1993.)
 |-  ( ph  ->  ps )   =>    |-  ( A. x ph  ->  ps )
 
Theoremspsd 1431 Deduction generalizing antecedent. (Contributed by NM, 17-Aug-1994.)
 |-  ( ph  ->  ( ps  ->  ch ) )   =>    |-  ( ph  ->  (
 A. x ps  ->  ch ) )
 
Theoremnfbidf 1432 An equality theorem for effectively not free. (Contributed by Mario Carneiro, 4-Oct-2016.)
 |- 
 F/ x ph   &    |-  ( ph  ->  ( ps  <->  ch ) )   =>    |-  ( ph  ->  ( F/ x ps  <->  F/ x ch )
 )
 
Theoremhba1 1433  x is not free in  A. x ph. 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.)
 |-  ( A. x ph  ->  A. x A. x ph )
 
Theoremnfa1 1434  x is not free in  A. x ph. (Contributed by Mario Carneiro, 11-Aug-2016.)
 |- 
 F/ x A. x ph
 
Theorema5i 1435 Inference generalizing a consequent. (Contributed by NM, 5-Aug-1993.)
 |-  ( A. x ph  ->  ps )   =>    |-  ( A. x ph  ->  A. x ps )
 
Theoremnfnf1 1436  x is not free in  F/ x ph. (Contributed by Mario Carneiro, 11-Aug-2016.)
 |- 
 F/ x F/ x ph
 
Theoremhbim 1437 If  x is not free in  ph and  ps, it is not free in  ( ph  ->  ps ). (Contributed by NM, 5-Aug-1993.) (Proof shortened by O'Cat, 3-Mar-2008.) (Revised by Mario Carneiro, 2-Feb-2015.)
 |-  ( ph  ->  A. x ph )   &    |-  ( ps  ->  A. x ps )   =>    |-  ( ( ph  ->  ps )  ->  A. x ( ph  ->  ps )
 )
 
Theoremhbor 1438 If  x is not free in  ph and  ps, it is not free in  ( ph  \/  ps ). (Contributed by NM, 5-Aug-1993.) (Revised by NM, 2-Feb-2015.)
 |-  ( ph  ->  A. x ph )   &    |-  ( ps  ->  A. x ps )   =>    |-  ( ( ph  \/  ps )  ->  A. x ( ph  \/  ps )
 )
 
Theoremhban 1439 If  x is not free in  ph and  ps, it is not free in  ( ph  /\  ps ). (Contributed by NM, 5-Aug-1993.) (Proof shortened by Mario Carneiro, 2-Feb-2015.)
 |-  ( ph  ->  A. x ph )   &    |-  ( ps  ->  A. x ps )   =>    |-  ( ( ph  /\ 
 ps )  ->  A. x ( ph  /\  ps )
 )
 
Theoremhbbi 1440 If  x is not free in  ph and  ps, it is not free in  ( ph  <->  ps ). (Contributed by NM, 5-Aug-1993.)
 |-  ( ph  ->  A. x ph )   &    |-  ( ps  ->  A. x ps )   =>    |-  ( ( ph  <->  ps )  ->  A. x ( ph  <->  ps ) )
 
Theoremhb3or 1441 If  x is not free in  ph,  ps, and  ch, it is not free in  ( ph  \/  ps  \/  ch ). (Contributed by NM, 14-Sep-2003.)
 |-  ( ph  ->  A. x ph )   &    |-  ( ps  ->  A. x ps )   &    |-  ( ch  ->  A. x ch )   =>    |-  (
 ( ph  \/  ps  \/  ch )  ->  A. x (
 ph  \/  ps  \/  ch ) )
 
Theoremhb3an 1442 If  x is not free in  ph,  ps, and  ch, it is not free in  ( ph  /\  ps  /\  ch ). (Contributed by NM, 14-Sep-2003.)
 |-  ( ph  ->  A. x ph )   &    |-  ( ps  ->  A. x ps )   &    |-  ( ch  ->  A. x ch )   =>    |-  (
 ( ph  /\  ps  /\  ch )  ->  A. x (
 ph  /\  ps  /\  ch ) )
 
Theoremhba2 1443 Lemma 24 of [Monk2] p. 114. (Contributed by NM, 29-May-2008.)
 |-  ( A. y A. x ph  ->  A. x A. y A. x ph )
 
Theoremhbia1 1444 Lemma 23 of [Monk2] p. 114. (Contributed by NM, 29-May-2008.)
 |-  ( ( A. x ph 
 ->  A. x ps )  ->  A. x ( A. x ph  ->  A. x ps ) )
 
Theorem19.3h 1445 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.)
 |-  ( ph  ->  A. x ph )   =>    |-  ( A. x ph  <->  ph )
 
Theorem19.3 1446 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.)
 |- 
 F/ x ph   =>    |-  ( A. x ph  <->  ph )
 
Theorem19.16 1447 Theorem 19.16 of [Margaris] p. 90. (Contributed by NM, 12-Mar-1993.)
 |- 
 F/ x ph   =>    |-  ( A. x (
 ph 
 <->  ps )  ->  ( ph 
 <-> 
 A. x ps )
 )
 
Theorem19.17 1448 Theorem 19.17 of [Margaris] p. 90. (Contributed by NM, 12-Mar-1993.)
 |- 
 F/ x ps   =>    |-  ( A. x ( ph  <->  ps )  ->  ( A. x ph  <->  ps ) )
 
Theorem19.21h 1449 Theorem 19.21 of [Margaris] p. 90. The hypothesis can be thought of as " x is not free in  ph." New proofs should use 19.21 1475 instead. (Contributed by NM, 5-Aug-1993.) (New usage is discouraged.)
 |-  ( ph  ->  A. x ph )   =>    |-  ( A. x (
 ph  ->  ps )  <->  ( ph  ->  A. x ps ) )
 
Theorem19.21bi 1450 Inference from Theorem 19.21 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.)
 |-  ( ph  ->  A. x ps )   =>    |-  ( ph  ->  ps )
 
Theorem19.21bbi 1451 Inference removing double quantifier. (Contributed by NM, 20-Apr-1994.)
 |-  ( ph  ->  A. x A. y ps )   =>    |-  ( ph  ->  ps )
 
Theorem19.27h 1452 Theorem 19.27 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.)
 |-  ( ps  ->  A. x ps )   =>    |-  ( A. x (
 ph  /\  ps )  <->  (
 A. x ph  /\  ps ) )
 
Theorem19.27 1453 Theorem 19.27 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.)
 |- 
 F/ x ps   =>    |-  ( A. x ( ph  /\  ps )  <->  (
 A. x ph  /\  ps ) )
 
Theorem19.28h 1454 Theorem 19.28 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.)
 |-  ( ph  ->  A. x ph )   =>    |-  ( A. x (
 ph  /\  ps )  <->  (
 ph  /\  A. x ps ) )
 
Theorem19.28 1455 Theorem 19.28 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.)
 |- 
 F/ x ph   =>    |-  ( A. x (
 ph  /\  ps )  <->  (
 ph  /\  A. x ps ) )
 
Theoremnfan1 1456 A closed form of nfan 1457. (Contributed by Mario Carneiro, 3-Oct-2016.)
 |- 
 F/ x ph   &    |-  ( ph  ->  F/ x ps )   =>    |-  F/ x (
 ph  /\  ps )
 
Theoremnfan 1457 If  x is not free in  ph and  ps, it is not free in  ( ph  /\  ps ). (Contributed by Mario Carneiro, 11-Aug-2016.) (Proof shortened by Wolf Lammen, 13-Jan-2018.)
 |- 
 F/ x ph   &    |-  F/ x ps   =>    |-  F/ x ( ph  /\  ps )
 
Theoremnf3an 1458 If  x is not free in  ph,  ps, and  ch, it is not free in  ( ph  /\  ps  /\  ch ). (Contributed by Mario Carneiro, 11-Aug-2016.)
 |- 
 F/ x ph   &    |-  F/ x ps   &    |-  F/ x ch   =>    |- 
 F/ x ( ph  /\ 
 ps  /\  ch )
 
Theoremnford 1459 If in a context  x is not free in  ps and  ch, it is not free in  ( ps  \/  ch ). (Contributed by Jim Kingdon, 29-Oct-2019.)
 |-  ( ph  ->  F/ x ps )   &    |-  ( ph  ->  F/ x ch )   =>    |-  ( ph  ->  F/ x ( ps  \/  ch ) )
 
Theoremnfand 1460 If in a context  x is not free in  ps and  ch, it is not free in  ( ps  /\  ch ). (Contributed by Mario Carneiro, 7-Oct-2016.)
 |-  ( ph  ->  F/ x ps )   &    |-  ( ph  ->  F/ x ch )   =>    |-  ( ph  ->  F/ x ( ps  /\  ch ) )
 
Theoremnf3and 1461 Deduction form of bound-variable hypothesis builder nf3an 1458. (Contributed by NM, 17-Feb-2013.) (Revised by Mario Carneiro, 16-Oct-2016.)
 |-  ( ph  ->  F/ x ps )   &    |-  ( ph  ->  F/ x ch )   &    |-  ( ph  ->  F/ x th )   =>    |-  ( ph  ->  F/ x ( ps  /\  ch  /\  th ) )
 
Theoremhbim1 1462 A closed form of hbim 1437. (Contributed by NM, 5-Aug-1993.)
 |-  ( ph  ->  A. x ph )   &    |-  ( ph  ->  ( ps  ->  A. x ps ) )   =>    |-  ( ( ph  ->  ps )  ->  A. x (
 ph  ->  ps ) )
 
Theoremnfim1 1463 A closed form of nfim 1464. (Contributed by NM, 5-Aug-1993.) (Revised by Mario Carneiro, 24-Sep-2016.) (Proof shortened by Wolf Lammen, 2-Jan-2018.)
 |- 
 F/ x ph   &    |-  ( ph  ->  F/ x ps )   =>    |-  F/ x (
 ph  ->  ps )
 
Theoremnfim 1464 If  x is not free in  ph and  ps, it is not free in  ( ph  ->  ps ). (Contributed by Mario Carneiro, 11-Aug-2016.) (Proof shortened by Wolf Lammen, 2-Jan-2018.)
 |- 
 F/ x ph   &    |-  F/ x ps   =>    |-  F/ x ( ph  ->  ps )
 
Theoremhbimd 1465 Deduction form of bound-variable hypothesis builder hbim 1437. (Contributed by NM, 1-Jan-2002.) (Revised by NM, 2-Feb-2015.)
 |-  ( ph  ->  A. x ph )   &    |-  ( ph  ->  ( ps  ->  A. x ps ) )   &    |-  ( ph  ->  ( ch  ->  A. x ch ) )   =>    |-  ( ph  ->  (
 ( ps  ->  ch )  ->  A. x ( ps 
 ->  ch ) ) )
 
Theoremnfor 1466 If  x is not free in  ph and  ps, it is not free in  ( ph  \/  ps ). (Contributed by Jim Kingdon, 11-Mar-2018.)
 |- 
 F/ x ph   &    |-  F/ x ps   =>    |-  F/ x ( ph  \/  ps )
 
Theoremhbbid 1467 Deduction form of bound-variable hypothesis builder hbbi 1440. (Contributed by NM, 1-Jan-2002.)
 |-  ( ph  ->  A. x ph )   &    |-  ( ph  ->  ( ps  ->  A. x ps ) )   &    |-  ( ph  ->  ( ch  ->  A. x ch ) )   =>    |-  ( ph  ->  (
 ( ps  <->  ch )  ->  A. x ( ps  <->  ch ) ) )
 
Theoremnfal 1468 If  x is not free in  ph, it is not free in  A. y ph. (Contributed by Mario Carneiro, 11-Aug-2016.)
 |- 
 F/ x ph   =>    |- 
 F/ x A. y ph
 
Theoremnfnf 1469 If  x is not free in  ph, it is not free in  F/ y ph. (Contributed by Mario Carneiro, 11-Aug-2016.) (Proof shortened by Wolf Lammen, 30-Dec-2017.)
 |- 
 F/ x ph   =>    |- 
 F/ x F/ y ph
 
Theoremnfalt 1470 Closed form of nfal 1468. (Contributed by Jim Kingdon, 11-May-2018.)
 |-  ( A. y F/ x ph  ->  F/ x A. y ph )
 
Theoremnfa2 1471 Lemma 24 of [Monk2] p. 114. (Contributed by Mario Carneiro, 24-Sep-2016.)
 |- 
 F/ x A. y A. x ph
 
Theoremnfia1 1472 Lemma 23 of [Monk2] p. 114. (Contributed by Mario Carneiro, 24-Sep-2016.)
 |- 
 F/ x ( A. x ph  ->  A. x ps )
 
Theorem19.21ht 1473 Closed form of Theorem 19.21 of [Margaris] p. 90. (Contributed by NM, 27-May-1997.) (New usage is discouraged.)
 |-  ( A. x (
 ph  ->  A. x ph )  ->  ( A. x (
 ph  ->  ps )  <->  ( ph  ->  A. x ps ) ) )
 
Theorem19.21t 1474 Closed form of Theorem 19.21 of [Margaris] p. 90. (Contributed by NM, 27-May-1997.)
 |-  ( F/ x ph  ->  ( A. x (
 ph  ->  ps )  <->  ( ph  ->  A. x ps ) ) )
 
Theorem19.21 1475 Theorem 19.21 of [Margaris] p. 90. The hypothesis can be thought of as " x is not free in  ph." (Contributed by NM, 5-Aug-1993.) (Revised by Mario Carneiro, 24-Sep-2016.)
 |- 
 F/ x ph   =>    |-  ( A. x (
 ph  ->  ps )  <->  ( ph  ->  A. x ps ) )
 
Theoremstdpc5 1476 An axiom scheme of standard predicate calculus that emulates Axiom 5 of [Mendelson] p. 69. The hypothesis  F/ x ph can be thought of as emulating " x is not free in  ph." With this definition, the meaning of "not free" is less restrictive than the usual textbook definition; for example  x would not (for us) be free in  x  =  x by nfequid 1590. 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.)
 |- 
 F/ x ph   =>    |-  ( A. x (
 ph  ->  ps )  ->  ( ph  ->  A. x ps )
 )
 
Theoremnfimd 1477 If in a context  x is not free in  ps and  ch, it is not free in  ( ps  ->  ch ). (Contributed by Mario Carneiro, 24-Sep-2016.) (Proof shortened by Wolf Lammen, 30-Dec-2017.)
 |-  ( ph  ->  F/ x ps )   &    |-  ( ph  ->  F/ x ch )   =>    |-  ( ph  ->  F/ x ( ps  ->  ch ) )
 
Theoremaaanh 1478 Rearrange universal quantifiers. (Contributed by NM, 12-Aug-1993.)
 |-  ( ph  ->  A. y ph )   &    |-  ( ps  ->  A. x ps )   =>    |-  ( A. x A. y ( ph  /\  ps ) 
 <->  ( A. x ph  /\ 
 A. y ps )
 )
 
Theoremaaan 1479 Rearrange universal quantifiers. (Contributed by NM, 12-Aug-1993.)
 |- 
 F/ y ph   &    |-  F/ x ps   =>    |-  ( A. x A. y (
 ph  /\  ps )  <->  (
 A. x ph  /\  A. y ps ) )
 
Theoremnfbid 1480 If in a context  x is not free in  ps and  ch, it is not free in  ( ps  <->  ch ). (Contributed by Mario Carneiro, 24-Sep-2016.) (Proof shortened by Wolf Lammen, 29-Dec-2017.)
 |-  ( ph  ->  F/ x ps )   &    |-  ( ph  ->  F/ x ch )   =>    |-  ( ph  ->  F/ x ( ps  <->  ch ) )
 
Theoremnfbi 1481 If  x is not free in  ph and  ps, it is not free in  ( ph  <->  ps ). (Contributed by Mario Carneiro, 11-Aug-2016.) (Proof shortened by Wolf Lammen, 2-Jan-2018.)
 |- 
 F/ x ph   &    |-  F/ x ps   =>    |-  F/ x ( ph  <->  ps )
 
1.3.7  The existential quantifier
 
Theorem19.8a 1482 If a wff is true, it is true for at least one instance. Special case of Theorem 19.8 of [Margaris] p. 89. (Contributed by NM, 5-Aug-1993.)
 |-  ( ph  ->  E. x ph )
 
Theorem19.23bi 1483 Inference from Theorem 19.23 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.)
 |-  ( E. x ph  ->  ps )   =>    |-  ( ph  ->  ps )
 
Theoremexlimih 1484 Inference from Theorem 19.23 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.) (Proof shortened by Andrew Salmon, 13-May-2011.)
 |-  ( ps  ->  A. x ps )   &    |-  ( ph  ->  ps )   =>    |-  ( E. x ph  ->  ps )
 
Theoremexlimi 1485 Inference from Theorem 19.23 of [Margaris] p. 90. (Contributed by Mario Carneiro, 24-Sep-2016.)
 |- 
 F/ x ps   &    |-  ( ph  ->  ps )   =>    |-  ( E. x ph  ->  ps )
 
Theoremexlimd2 1486 Deduction from Theorem 19.23 of [Margaris] p. 90. Similar to exlimdh 1487 but with one slightly different hypothesis. (Contributed by Jim Kingdon, 30-Dec-2017.)
 |-  ( ph  ->  A. x ph )   &    |-  ( ph  ->  ( ch  ->  A. x ch ) )   &    |-  ( ph  ->  ( ps  ->  ch )
 )   =>    |-  ( ph  ->  ( E. x ps  ->  ch )
 )
 
Theoremexlimdh 1487 Deduction from Theorem 19.23 of [Margaris] p. 90. (Contributed by NM, 28-Jan-1997.)
 |-  ( ph  ->  A. x ph )   &    |-  ( ch  ->  A. x ch )   &    |-  ( ph  ->  ( ps  ->  ch ) )   =>    |-  ( ph  ->  ( E. x ps  ->  ch )
 )
 
Theoremexlimd 1488 Deduction from Theorem 19.9 of [Margaris] p. 89. (Contributed by Mario Carneiro, 24-Sep-2016.) (Proof rewritten by Jim Kingdon, 18-Jun-2018.)
 |- 
 F/ x ph   &    |-  F/ x ch   &    |-  ( ph  ->  ( ps  ->  ch ) )   =>    |-  ( ph  ->  ( E. x ps  ->  ch )
 )
 
Theoremexlimiv 1489* 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  x exists satisfying a wff, i.e.  E. x ph ( x ) where  ph ( x ) has  x free, then we can use  ph ( 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  ph (containing  x) as an antecedent for the main part of the proof. We eventually arrive at  ( ph  ->  ps ) where  ps is the theorem to be proved and does not contain  x. Then we apply exlimiv 1489 to arrive at  ( E. x ph  ->  ps ). Finally, we separately prove  E. x ph and detach it with modus ponens ax-mp 7 to arrive at the final theorem  ps. (Contributed by NM, 5-Aug-1993.) (Revised by NM, 25-Jul-2012.)

 |-  ( ph  ->  ps )   =>    |-  ( E. x ph  ->  ps )
 
Theoremexim 1490 Theorem 19.22 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.) (Proof shortened by Wolf Lammen, 4-Jul-2014.)
 |-  ( A. x (
 ph  ->  ps )  ->  ( E. x ph  ->  E. x ps ) )
 
Theoremeximi 1491 Inference adding existential quantifier to antecedent and consequent. (Contributed by NM, 5-Aug-1993.)
 |-  ( ph  ->  ps )   =>    |-  ( E. x ph  ->  E. x ps )
 
Theorem2eximi 1492 Inference adding 2 existential quantifiers to antecedent and consequent. (Contributed by NM, 3-Feb-2005.)
 |-  ( ph  ->  ps )   =>    |-  ( E. x E. y ph  ->  E. x E. y ps )
 
Theoremeximii 1493 Inference associated with eximi 1491. (Contributed by BJ, 3-Feb-2018.)
 |- 
 E. x ph   &    |-  ( ph  ->  ps )   =>    |- 
 E. x ps
 
Theoremalinexa 1494 A transformation of quantifiers and logical connectives. (Contributed by NM, 19-Aug-1993.)
 |-  ( A. x (
 ph  ->  -.  ps )  <->  -. 
 E. x ( ph  /\ 
 ps ) )
 
Theoremexbi 1495 Theorem 19.18 of [Margaris] p. 90. (Contributed by NM, 5-Aug-1993.)
 |-  ( A. x (
 ph 
 <->  ps )  ->  ( E. x ph  <->  E. x ps )
 )
 
Theoremexbii 1496 Inference adding existential quantifier to both sides of an equivalence. (Contributed by NM, 24-May-1994.)
 |-  ( ph  <->  ps )   =>    |-  ( E. x ph  <->  E. x ps )
 
Theorem2exbii 1497 Inference adding 2 existential quantifiers to both sides of an equivalence. (Contributed by NM, 16-Mar-1995.)
 |-  ( ph  <->  ps )   =>    |-  ( E. x E. y ph  <->  E. x E. y ps )
 
Theorem3exbii 1498 Inference adding 3 existential quantifiers to both sides of an equivalence. (Contributed by NM, 2-May-1995.)
 |-  ( ph  <->  ps )   =>    |-  ( E. x E. y E. z ph  <->  E. x E. y E. z ps )
 
Theoremexancom 1499 Commutation of conjunction inside an existential quantifier. (Contributed by NM, 18-Aug-1993.)
 |-  ( E. x (
 ph  /\  ps )  <->  E. x ( ps  /\  ph ) )
 
Theoremalrimdd 1500 Deduction from Theorem 19.21 of [Margaris] p. 90. (Contributed by Mario Carneiro, 24-Sep-2016.)
 |- 
 F/ x ph   &    |-  ( ph  ->  F/ x ps )   &    |-  ( ph  ->  ( ps  ->  ch ) )   =>    |-  ( ph  ->  ( ps  ->  A. x ch )
 )
    < 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-10124
  Copyright terms: Public domain < Previous  Next >