HomeHome Intuitionistic Logic Explorer
Theorem List (p. 60 of 162)
< 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 - 5901-6000   *Has distinct variable group(s)
TypeLabelDescription
Statement
 
Theoremisoini2 5901 Isomorphisms are isomorphisms on their initial segments. (Contributed by Mario Carneiro, 29-Mar-2014.)
 |-  C  =  ( A  i^i  ( `' R " { X } )
 )   &    |-  D  =  ( B  i^i  ( `' S " { ( H `  X ) } )
 )   =>    |-  ( ( H  Isom  R ,  S  ( A ,  B )  /\  X  e.  A )  ->  ( H  |`  C ) 
 Isom  R ,  S  ( C ,  D ) )
 
Theoremisoselem 5902* Lemma for isose 5903. (Contributed by Mario Carneiro, 23-Jun-2015.)
 |-  ( ph  ->  H  Isom  R ,  S  ( A ,  B ) )   &    |-  ( ph  ->  ( H " x )  e.  _V )   =>    |-  ( ph  ->  ( R Se  A  ->  S Se  B ) )
 
Theoremisose 5903 An isomorphism preserves set-like relations. (Contributed by Mario Carneiro, 23-Jun-2015.)
 |-  ( H  Isom  R ,  S  ( A ,  B )  ->  ( R Se  A  <->  S Se 
 B ) )
 
Theoremisopolem 5904 Lemma for isopo 5905. (Contributed by Stefan O'Rear, 16-Nov-2014.)
 |-  ( H  Isom  R ,  S  ( A ,  B )  ->  ( S  Po  B  ->  R  Po  A ) )
 
Theoremisopo 5905 An isomorphism preserves partial ordering. (Contributed by Stefan O'Rear, 16-Nov-2014.)
 |-  ( H  Isom  R ,  S  ( A ,  B )  ->  ( R  Po  A 
 <->  S  Po  B ) )
 
Theoremisosolem 5906 Lemma for isoso 5907. (Contributed by Stefan O'Rear, 16-Nov-2014.)
 |-  ( H  Isom  R ,  S  ( A ,  B )  ->  ( S  Or  B  ->  R  Or  A ) )
 
Theoremisoso 5907 An isomorphism preserves strict ordering. (Contributed by Stefan O'Rear, 16-Nov-2014.)
 |-  ( H  Isom  R ,  S  ( A ,  B )  ->  ( R  Or  A 
 <->  S  Or  B ) )
 
Theoremf1oiso 5908* Any one-to-one onto function determines an isomorphism with an induced relation  S. Proposition 6.33 of [TakeutiZaring] p. 34. (Contributed by NM, 30-Apr-2004.)
 |-  ( ( H : A
 -1-1-onto-> B  /\  S  =  { <. z ,  w >.  | 
 E. x  e.  A  E. y  e.  A  ( ( z  =  ( H `  x )  /\  w  =  ( H `  y ) )  /\  x R y ) } )  ->  H  Isom  R ,  S  ( A ,  B ) )
 
Theoremf1oiso2 5909* Any one-to-one onto function determines an isomorphism with an induced relation  S. (Contributed by Mario Carneiro, 9-Mar-2013.)
 |-  S  =  { <. x ,  y >.  |  ( ( x  e.  B  /\  y  e.  B )  /\  ( `' H `  x ) R ( `' H `  y ) ) }   =>    |-  ( H : A -1-1-onto-> B  ->  H  Isom  R ,  S  ( A ,  B ) )
 
2.6.9  Cantor's Theorem
 
Theoremcanth 5910 No set  A is equinumerous to its power set (Cantor's theorem), i.e., no function can map  A onto its power set. Compare Theorem 6B(b) of [Enderton] p. 132. (Use nex 1524 if you want the form  -.  E. f
f : A -onto-> ~P A.) (Contributed by NM, 7-Aug-1994.) (Revised by Noah R Kingdon, 23-Jul-2024.)
 |-  A  e.  _V   =>    |-  -.  F : A -onto-> ~P A
 
2.6.10  Restricted iota (description binder)
 
Syntaxcrio 5911 Extend class notation with restricted description binder.
 class  ( iota_ x  e.  A  ph )
 
Definitiondf-riota 5912 Define restricted description binder. In case there is no unique  x such that  ( x  e.  A  /\  ph ) holds, it evaluates to the empty set. See also comments for df-iota 5241. (Contributed by NM, 15-Sep-2011.) (Revised by Mario Carneiro, 15-Oct-2016.) (Revised by NM, 2-Sep-2018.)
 |-  ( iota_ x  e.  A  ph )  =  ( iota
 x ( x  e.  A  /\  ph )
 )
 
Theoremriotaeqdv 5913* Formula-building deduction for iota. (Contributed by NM, 15-Sep-2011.)
 |-  ( ph  ->  A  =  B )   =>    |-  ( ph  ->  ( iota_ x  e.  A  ps )  =  ( iota_ x  e.  B  ps ) )
 
Theoremriotabidv 5914* Formula-building deduction for restricted iota. (Contributed by NM, 15-Sep-2011.)
 |-  ( ph  ->  ( ps 
 <->  ch ) )   =>    |-  ( ph  ->  (
 iota_ x  e.  A  ps )  =  ( iota_ x  e.  A  ch ) )
 
Theoremriotaeqbidv 5915* Equality deduction for restricted universal quantifier. (Contributed by NM, 15-Sep-2011.)
 |-  ( ph  ->  A  =  B )   &    |-  ( ph  ->  ( ps  <->  ch ) )   =>    |-  ( ph  ->  (
 iota_ x  e.  A  ps )  =  ( iota_ x  e.  B  ch ) )
 
Theoremriotaexg 5916* Restricted iota is a set. (Contributed by Jim Kingdon, 15-Jun-2020.)
 |-  ( A  e.  V  ->  ( iota_ x  e.  A  ps )  e.  _V )
 
Theoremiotaexel 5917* Set existence of an iota expression in which all values are contained within a set. (Contributed by Jim Kingdon, 28-Jun-2025.)
 |-  ( ( A  e.  V  /\  A. x (
 ph  ->  x  e.  A ) )  ->  ( iota
 x ph )  e.  _V )
 
Theoremriotav 5918 An iota restricted to the universe is unrestricted. (Contributed by NM, 18-Sep-2011.)
 |-  ( iota_ x  e.  _V  ph )  =  ( iota
 x ph )
 
Theoremriotauni 5919 Restricted iota in terms of class union. (Contributed by NM, 11-Oct-2011.)
 |-  ( E! x  e.  A  ph  ->  ( iota_ x  e.  A  ph )  =  U. { x  e.  A  |  ph } )
 
Theoremnfriota1 5920* The abstraction variable in a restricted iota descriptor isn't free. (Contributed by NM, 12-Oct-2011.) (Revised by Mario Carneiro, 15-Oct-2016.)
 |-  F/_ x ( iota_ x  e.  A  ph )
 
Theoremnfriotadxy 5921* Deduction version of nfriota 5922. (Contributed by Jim Kingdon, 12-Jan-2019.)
 |- 
 F/ y ph   &    |-  ( ph  ->  F/ x ps )   &    |-  ( ph  ->  F/_ x A )   =>    |-  ( ph  ->  F/_ x (
 iota_ y  e.  A  ps ) )
 
Theoremnfriota 5922* A variable not free in a wff remains so in a restricted iota descriptor. (Contributed by NM, 12-Oct-2011.)
 |- 
 F/ x ph   &    |-  F/_ x A   =>    |-  F/_ x ( iota_ y  e.  A  ph )
 
Theoremcbvriota 5923* Change bound variable in a restricted description binder. (Contributed by NM, 18-Mar-2013.) (Revised by Mario Carneiro, 15-Oct-2016.)
 |- 
 F/ y ph   &    |-  F/ x ps   &    |-  ( x  =  y  ->  (
 ph 
 <->  ps ) )   =>    |-  ( iota_ x  e.  A  ph )  =  ( iota_ y  e.  A  ps )
 
Theoremcbvriotav 5924* Change bound variable in a restricted description binder. (Contributed by NM, 18-Mar-2013.) (Revised by Mario Carneiro, 15-Oct-2016.)
 |-  ( x  =  y 
 ->  ( ph  <->  ps ) )   =>    |-  ( iota_ x  e.  A  ph )  =  ( iota_ y  e.  A  ps )
 
Theoremcsbriotag 5925* Interchange class substitution and restricted description binder. (Contributed by NM, 24-Feb-2013.)
 |-  ( A  e.  V  -> 
 [_ A  /  x ]_ ( iota_ y  e.  B  ph )  =  ( iota_ y  e.  B  [. A  /  x ]. ph )
 )
 
Theoremriotacl2 5926 Membership law for "the unique element in  A such that  ph."

(Contributed by NM, 21-Aug-2011.) (Revised by Mario Carneiro, 23-Dec-2016.)

 |-  ( E! x  e.  A  ph  ->  ( iota_ x  e.  A  ph )  e.  { x  e.  A  |  ph } )
 
Theoremriotacl 5927* Closure of restricted iota. (Contributed by NM, 21-Aug-2011.)
 |-  ( E! x  e.  A  ph  ->  ( iota_ x  e.  A  ph )  e.  A )
 
Theoremriotasbc 5928 Substitution law for descriptions. (Contributed by NM, 23-Aug-2011.) (Proof shortened by Mario Carneiro, 24-Dec-2016.)
 |-  ( E! x  e.  A  ph  ->  [. ( iota_ x  e.  A  ph )  /  x ]. ph )
 
Theoremriotabidva 5929* Equivalent wff's yield equal restricted class abstractions (deduction form). (rabbidva 2761 analog.) (Contributed by NM, 17-Jan-2012.)
 |-  ( ( ph  /\  x  e.  A )  ->  ( ps 
 <->  ch ) )   =>    |-  ( ph  ->  (
 iota_ x  e.  A  ps )  =  ( iota_ x  e.  A  ch ) )
 
Theoremriotabiia 5930 Equivalent wff's yield equal restricted iotas (inference form). (rabbiia 2758 analog.) (Contributed by NM, 16-Jan-2012.)
 |-  ( x  e.  A  ->  ( ph  <->  ps ) )   =>    |-  ( iota_ x  e.  A  ph )  =  ( iota_ x  e.  A  ps )
 
Theoremriota1 5931* Property of restricted iota. Compare iota1 5255. (Contributed by Mario Carneiro, 15-Oct-2016.)
 |-  ( E! x  e.  A  ph  ->  ( ( x  e.  A  /\  ph )  <->  ( iota_ x  e.  A  ph )  =  x ) )
 
Theoremriota1a 5932 Property of iota. (Contributed by NM, 23-Aug-2011.)
 |-  ( ( x  e.  A  /\  E! x  e.  A  ph )  ->  ( ph  <->  ( iota x ( x  e.  A  /\  ph ) )  =  x ) )
 
Theoremriota2df 5933* A deduction version of riota2f 5934. (Contributed by NM, 17-Feb-2013.) (Revised by Mario Carneiro, 15-Oct-2016.)
 |- 
 F/ x ph   &    |-  ( ph  ->  F/_ x B )   &    |-  ( ph  ->  F/ x ch )   &    |-  ( ph  ->  B  e.  A )   &    |-  ( ( ph  /\  x  =  B ) 
 ->  ( ps  <->  ch ) )   =>    |-  ( ( ph  /\ 
 E! x  e.  A  ps )  ->  ( ch  <->  (
 iota_ x  e.  A  ps )  =  B ) )
 
Theoremriota2f 5934* This theorem shows a condition that allows us to represent a descriptor with a class expression  B. (Contributed by NM, 23-Aug-2011.) (Revised by Mario Carneiro, 15-Oct-2016.)
 |-  F/_ x B   &    |-  F/ x ps   &    |-  ( x  =  B  ->  (
 ph 
 <->  ps ) )   =>    |-  ( ( B  e.  A  /\  E! x  e.  A  ph )  ->  ( ps  <->  ( iota_ x  e.  A  ph )  =  B ) )
 
Theoremriota2 5935* This theorem shows a condition that allows us to represent a descriptor with a class expression  B. (Contributed by NM, 23-Aug-2011.) (Revised by Mario Carneiro, 10-Dec-2016.)
 |-  ( x  =  B  ->  ( ph  <->  ps ) )   =>    |-  ( ( B  e.  A  /\  E! x  e.  A  ph )  ->  ( ps  <->  ( iota_ x  e.  A  ph )  =  B ) )
 
Theoremriotaprop 5936* Properties of a restricted definite description operator. Todo (df-riota 5912 update): can some uses of riota2f 5934 be shortened with this? (Contributed by NM, 23-Nov-2013.)
 |- 
 F/ x ps   &    |-  B  =  ( iota_ x  e.  A  ph )   &    |-  ( x  =  B  ->  ( ph  <->  ps ) )   =>    |-  ( E! x  e.  A  ph  ->  ( B  e.  A  /\  ps ) )
 
Theoremriota5f 5937* A method for computing restricted iota. (Contributed by NM, 16-Apr-2013.) (Revised by Mario Carneiro, 15-Oct-2016.)
 |-  ( ph  ->  F/_ x B )   &    |-  ( ph  ->  B  e.  A )   &    |-  (
 ( ph  /\  x  e.  A )  ->  ( ps 
 <->  x  =  B ) )   =>    |-  ( ph  ->  ( iota_ x  e.  A  ps )  =  B )
 
Theoremriota5 5938* A method for computing restricted iota. (Contributed by NM, 20-Oct-2011.) (Revised by Mario Carneiro, 6-Dec-2016.)
 |-  ( ph  ->  B  e.  A )   &    |-  ( ( ph  /\  x  e.  A ) 
 ->  ( ps  <->  x  =  B ) )   =>    |-  ( ph  ->  ( iota_ x  e.  A  ps )  =  B )
 
Theoremriotass2 5939* Restriction of a unique element to a smaller class. (Contributed by NM, 21-Aug-2011.) (Revised by NM, 22-Mar-2013.)
 |-  ( ( ( A 
 C_  B  /\  A. x  e.  A  ( ph  ->  ps ) )  /\  ( E. x  e.  A  ph 
 /\  E! x  e.  B  ps ) )  ->  ( iota_ x  e.  A  ph )  =  ( iota_ x  e.  B  ps ) )
 
Theoremriotass 5940* Restriction of a unique element to a smaller class. (Contributed by NM, 19-Oct-2005.) (Revised by Mario Carneiro, 24-Dec-2016.)
 |-  ( ( A  C_  B  /\  E. x  e.  A  ph  /\  E! x  e.  B  ph )  ->  ( iota_ x  e.  A  ph )  =  ( iota_ x  e.  B  ph )
 )
 
Theoremmoriotass 5941* Restriction of a unique element to a smaller class. (Contributed by NM, 19-Feb-2006.) (Revised by NM, 16-Jun-2017.)
 |-  ( ( A  C_  B  /\  E. x  e.  A  ph  /\  E* x  e.  B  ph )  ->  ( iota_ x  e.  A  ph )  =  ( iota_ x  e.  B  ph )
 )
 
Theoremsnriota 5942 A restricted class abstraction with a unique member can be expressed as a singleton. (Contributed by NM, 30-May-2006.)
 |-  ( E! x  e.  A  ph  ->  { x  e.  A  |  ph }  =  { ( iota_ x  e.  A  ph ) }
 )
 
Theoremeusvobj2 5943* Specify the same property in two ways when class  B ( y ) is single-valued. (Contributed by NM, 1-Nov-2010.) (Proof shortened by Mario Carneiro, 24-Dec-2016.)
 |-  B  e.  _V   =>    |-  ( E! x E. y  e.  A  x  =  B  ->  ( E. y  e.  A  x  =  B  <->  A. y  e.  A  x  =  B )
 )
 
Theoremeusvobj1 5944* Specify the same object in two ways when class  B ( y ) is single-valued. (Contributed by NM, 1-Nov-2010.) (Proof shortened by Mario Carneiro, 19-Nov-2016.)
 |-  B  e.  _V   =>    |-  ( E! x E. y  e.  A  x  =  B  ->  (
 iota x E. y  e.  A  x  =  B )  =  ( iota x
 A. y  e.  A  x  =  B )
 )
 
Theoremf1ofveu 5945* There is one domain element for each value of a one-to-one onto function. (Contributed by NM, 26-May-2006.)
 |-  ( ( F : A
 -1-1-onto-> B  /\  C  e.  B )  ->  E! x  e.  A  ( F `  x )  =  C )
 
Theoremf1ocnvfv3 5946* Value of the converse of a one-to-one onto function. (Contributed by NM, 26-May-2006.) (Proof shortened by Mario Carneiro, 24-Dec-2016.)
 |-  ( ( F : A
 -1-1-onto-> B  /\  C  e.  B )  ->  ( `' F `  C )  =  (
 iota_ x  e.  A  ( F `  x )  =  C ) )
 
Theoremriotaund 5947* Restricted iota equals the empty set when not meaningful. (Contributed by NM, 16-Jan-2012.) (Revised by Mario Carneiro, 15-Oct-2016.) (Revised by NM, 13-Sep-2018.)
 |-  ( -.  E! x  e.  A  ph  ->  ( iota_ x  e.  A  ph )  =  (/) )
 
Theoremacexmidlema 5948* Lemma for acexmid 5956. (Contributed by Jim Kingdon, 6-Aug-2019.)
 |-  A  =  { x  e.  { (/) ,  { (/) } }  |  ( x  =  (/)  \/  ph ) }   &    |-  B  =  { x  e.  { (/) ,  { (/)
 } }  |  ( x  =  { (/) }  \/  ph ) }   &    |-  C  =  { A ,  B }   =>    |-  ( { (/) }  e.  A  -> 
 ph )
 
Theoremacexmidlemb 5949* Lemma for acexmid 5956. (Contributed by Jim Kingdon, 6-Aug-2019.)
 |-  A  =  { x  e.  { (/) ,  { (/) } }  |  ( x  =  (/)  \/  ph ) }   &    |-  B  =  { x  e.  { (/) ,  { (/)
 } }  |  ( x  =  { (/) }  \/  ph ) }   &    |-  C  =  { A ,  B }   =>    |-  ( (/) 
 e.  B  ->  ph )
 
Theoremacexmidlemph 5950* Lemma for acexmid 5956. (Contributed by Jim Kingdon, 6-Aug-2019.)
 |-  A  =  { x  e.  { (/) ,  { (/) } }  |  ( x  =  (/)  \/  ph ) }   &    |-  B  =  { x  e.  { (/) ,  { (/)
 } }  |  ( x  =  { (/) }  \/  ph ) }   &    |-  C  =  { A ,  B }   =>    |-  ( ph  ->  A  =  B )
 
Theoremacexmidlemab 5951* Lemma for acexmid 5956. (Contributed by Jim Kingdon, 6-Aug-2019.)
 |-  A  =  { x  e.  { (/) ,  { (/) } }  |  ( x  =  (/)  \/  ph ) }   &    |-  B  =  { x  e.  { (/) ,  { (/)
 } }  |  ( x  =  { (/) }  \/  ph ) }   &    |-  C  =  { A ,  B }   =>    |-  (
 ( ( iota_ v  e.  A  E. u  e.  y  ( A  e.  u  /\  v  e.  u ) )  =  (/)  /\  ( iota_
 v  e.  B  E. u  e.  y  ( B  e.  u  /\  v  e.  u )
 )  =  { (/) } )  ->  -.  ph )
 
Theoremacexmidlemcase 5952* Lemma for acexmid 5956. Here we divide the proof into cases (based on the disjunction implicit in an unordered pair, not the sort of case elimination which relies on excluded middle).

The cases are (1) the choice function evaluated at  A equals  { (/) }, (2) the choice function evaluated at  B equals  (/), and (3) the choice function evaluated at  A equals 
(/) and the choice function evaluated at  B equals  { (/) }.

Because of the way we represent the choice function  y, the choice function evaluated at  A is  ( iota_ v  e.  A E. u  e.  y ( A  e.  u  /\  v  e.  u ) ) and the choice function evaluated at  B is  ( iota_ v  e.  B E. u  e.  y ( B  e.  u  /\  v  e.  u ) ). Other than the difference in notation these work just as  ( y `  A ) and  ( y `  B ) would if  y were a function as defined by df-fun 5282.

Although it isn't exactly about the division into cases, it is also convenient for this lemma to also include the step that if the choice function evaluated at  A equals  { (/) }, then  { (/) }  e.  A and likewise for  B.

(Contributed by Jim Kingdon, 7-Aug-2019.)

 |-  A  =  { x  e.  { (/) ,  { (/) } }  |  ( x  =  (/)  \/  ph ) }   &    |-  B  =  { x  e.  { (/) ,  { (/)
 } }  |  ( x  =  { (/) }  \/  ph ) }   &    |-  C  =  { A ,  B }   =>    |-  ( A. z  e.  C  E! v  e.  z  E. u  e.  y  ( z  e.  u  /\  v  e.  u )  ->  ( { (/) }  e.  A  \/  (/)  e.  B  \/  ( ( iota_ v  e.  A  E. u  e.  y  ( A  e.  u  /\  v  e.  u ) )  =  (/)  /\  ( iota_
 v  e.  B  E. u  e.  y  ( B  e.  u  /\  v  e.  u )
 )  =  { (/) } )
 ) )
 
Theoremacexmidlem1 5953* Lemma for acexmid 5956. List the cases identified in acexmidlemcase 5952 and hook them up to the lemmas which handle each case. (Contributed by Jim Kingdon, 7-Aug-2019.)
 |-  A  =  { x  e.  { (/) ,  { (/) } }  |  ( x  =  (/)  \/  ph ) }   &    |-  B  =  { x  e.  { (/) ,  { (/)
 } }  |  ( x  =  { (/) }  \/  ph ) }   &    |-  C  =  { A ,  B }   =>    |-  ( A. z  e.  C  E! v  e.  z  E. u  e.  y  ( z  e.  u  /\  v  e.  u )  ->  ( ph  \/  -.  ph ) )
 
Theoremacexmidlem2 5954* Lemma for acexmid 5956. This builds on acexmidlem1 5953 by noting that every element of  C is inhabited.

(Note that  y is not quite a function in the df-fun 5282 sense because it uses ordered pairs as described in opthreg 4612 rather than df-op 3647).

The set  A is also found in onsucelsucexmidlem 4585.

(Contributed by Jim Kingdon, 5-Aug-2019.)

 |-  A  =  { x  e.  { (/) ,  { (/) } }  |  ( x  =  (/)  \/  ph ) }   &    |-  B  =  { x  e.  { (/) ,  { (/)
 } }  |  ( x  =  { (/) }  \/  ph ) }   &    |-  C  =  { A ,  B }   =>    |-  ( A. z  e.  C  A. w  e.  z  E! v  e.  z  E. u  e.  y  (
 z  e.  u  /\  v  e.  u )  ->  ( ph  \/  -.  ph ) )
 
Theoremacexmidlemv 5955* Lemma for acexmid 5956.

This is acexmid 5956 with additional disjoint variable conditions, most notably between  ph and  x.

(Contributed by Jim Kingdon, 6-Aug-2019.)

 |- 
 E. y A. z  e.  x  A. w  e.  z  E! v  e.  z  E. u  e.  y  ( z  e.  u  /\  v  e.  u )   =>    |-  ( ph  \/  -.  ph )
 
Theoremacexmid 5956* The axiom of choice implies excluded middle. Theorem 1.3 in [Bauer] p. 483.

The statement of the axiom of choice given here is ac2 in the Metamath Proof Explorer (version of 3-Aug-2019). In particular, note that the choice function  y provides a value when  z is inhabited (as opposed to nonempty as in some statements of the axiom of choice).

Essentially the same proof can also be found at "The axiom of choice implies instances of EM", [Crosilla], p. "Set-theoretic principles incompatible with intuitionistic logic".

Often referred to as Diaconescu's theorem, or Diaconescu-Goodman-Myhill theorem, after Radu Diaconescu who discovered it in 1975 in the framework of topos theory and N. D. Goodman and John Myhill in 1978 in the framework of set theory (although it already appeared as an exercise in Errett Bishop's book Foundations of Constructive Analysis from 1967).

For this theorem stated using the df-ac 7334 and df-exmid 4247 syntaxes, see exmidac 7337. (Contributed by Jim Kingdon, 4-Aug-2019.)

 |- 
 E. y A. z  e.  x  A. w  e.  z  E! v  e.  z  E. u  e.  y  ( z  e.  u  /\  v  e.  u )   =>    |-  ( ph  \/  -.  ph )
 
2.6.11  Operations
 
Syntaxco 5957 Extend class notation to include the value of an operation  F (such as + ) for two arguments  A and  B. Note that the syntax is simply three class symbols in a row surrounded by parentheses. Since operation values are the only possible class expressions consisting of three class expressions in a row surrounded by parentheses, the syntax is unambiguous.
 class  ( A F B )
 
Syntaxcoprab 5958 Extend class notation to include class abstraction (class builder) of nested ordered pairs.
 class  { <. <. x ,  y >. ,  z >.  |  ph }
 
Syntaxcmpo 5959 Extend the definition of a class to include maps-to notation for defining an operation via a rule.
 class  ( x  e.  A ,  y  e.  B  |->  C )
 
Definitiondf-ov 5960 Define the value of an operation. Definition of operation value in [Enderton] p. 79. Note that the syntax is simply three class expressions in a row bracketed by parentheses. There are no restrictions of any kind on what those class expressions may be, although only certain kinds of class expressions - a binary operation  F and its arguments  A and  B- will be useful for proving meaningful theorems. For example, if class  F is the operation + and arguments  A and  B are 3 and 2 , the expression ( 3 + 2 ) can be proved to equal 5 . This definition is well-defined, although not very meaningful, when classes  A and/or  B are proper classes (i.e. are not sets); see ovprc1 5994 and ovprc2 5995. On the other hand, we often find uses for this definition when  F is a proper class.  F is normally equal to a class of nested ordered pairs of the form defined by df-oprab 5961. (Contributed by NM, 28-Feb-1995.)
 |-  ( A F B )  =  ( F ` 
 <. A ,  B >. )
 
Definitiondf-oprab 5961* Define the class abstraction (class builder) of a collection of nested ordered pairs (for use in defining operations). This is a special case of Definition 4.16 of [TakeutiZaring] p. 14. Normally  x,  y, and  z are distinct, although the definition doesn't strictly require it. See df-ov 5960 for the value of an operation. The brace notation is called "class abstraction" by Quine; it is also called a "class builder" in the literature. The value of the most common operation class builder is given by ovmpo 6094. (Contributed by NM, 12-Mar-1995.)
 |- 
 { <. <. x ,  y >. ,  z >.  |  ph }  =  { w  |  E. x E. y E. z ( w  = 
 <. <. x ,  y >. ,  z >.  /\  ph ) }
 
Definitiondf-mpo 5962* Define maps-to notation for defining an operation via a rule. Read as "the operation defined by the map from  x ,  y (in  A  X.  B) to  B ( x ,  y )". An extension of df-mpt 4115 for two arguments. (Contributed by NM, 17-Feb-2008.)
 |-  ( x  e.  A ,  y  e.  B  |->  C )  =  { <.
 <. x ,  y >. ,  z >.  |  (
 ( x  e.  A  /\  y  e.  B )  /\  z  =  C ) }
 
Theoremoveq 5963 Equality theorem for operation value. (Contributed by NM, 28-Feb-1995.)
 |-  ( F  =  G  ->  ( A F B )  =  ( A G B ) )
 
Theoremoveq1 5964 Equality theorem for operation value. (Contributed by NM, 28-Feb-1995.)
 |-  ( A  =  B  ->  ( A F C )  =  ( B F C ) )
 
Theoremoveq2 5965 Equality theorem for operation value. (Contributed by NM, 28-Feb-1995.)
 |-  ( A  =  B  ->  ( C F A )  =  ( C F B ) )
 
Theoremoveq12 5966 Equality theorem for operation value. (Contributed by NM, 16-Jul-1995.)
 |-  ( ( A  =  B  /\  C  =  D )  ->  ( A F C )  =  ( B F D ) )
 
Theoremoveq1i 5967 Equality inference for operation value. (Contributed by NM, 28-Feb-1995.)
 |-  A  =  B   =>    |-  ( A F C )  =  ( B F C )
 
Theoremoveq2i 5968 Equality inference for operation value. (Contributed by NM, 28-Feb-1995.)
 |-  A  =  B   =>    |-  ( C F A )  =  ( C F B )
 
Theoremoveq12i 5969 Equality inference for operation value. (Contributed by NM, 28-Feb-1995.) (Proof shortened by Andrew Salmon, 22-Oct-2011.)
 |-  A  =  B   &    |-  C  =  D   =>    |-  ( A F C )  =  ( B F D )
 
Theoremoveqi 5970 Equality inference for operation value. (Contributed by NM, 24-Nov-2007.)
 |-  A  =  B   =>    |-  ( C A D )  =  ( C B D )
 
Theoremoveq123i 5971 Equality inference for operation value. (Contributed by FL, 11-Jul-2010.)
 |-  A  =  C   &    |-  B  =  D   &    |-  F  =  G   =>    |-  ( A F B )  =  ( C G D )
 
Theoremoveq1d 5972 Equality deduction for operation value. (Contributed by NM, 13-Mar-1995.)
 |-  ( ph  ->  A  =  B )   =>    |-  ( ph  ->  ( A F C )  =  ( B F C ) )
 
Theoremoveq2d 5973 Equality deduction for operation value. (Contributed by NM, 13-Mar-1995.)
 |-  ( ph  ->  A  =  B )   =>    |-  ( ph  ->  ( C F A )  =  ( C F B ) )
 
Theoremoveqd 5974 Equality deduction for operation value. (Contributed by NM, 9-Sep-2006.)
 |-  ( ph  ->  A  =  B )   =>    |-  ( ph  ->  ( C A D )  =  ( C B D ) )
 
Theoremoveq12d 5975 Equality deduction for operation value. (Contributed by NM, 13-Mar-1995.) (Proof shortened by Andrew Salmon, 22-Oct-2011.)
 |-  ( ph  ->  A  =  B )   &    |-  ( ph  ->  C  =  D )   =>    |-  ( ph  ->  ( A F C )  =  ( B F D ) )
 
Theoremoveqan12d 5976 Equality deduction for operation value. (Contributed by NM, 10-Aug-1995.)
 |-  ( ph  ->  A  =  B )   &    |-  ( ps  ->  C  =  D )   =>    |-  ( ( ph  /\ 
 ps )  ->  ( A F C )  =  ( B F D ) )
 
Theoremoveqan12rd 5977 Equality deduction for operation value. (Contributed by NM, 10-Aug-1995.)
 |-  ( ph  ->  A  =  B )   &    |-  ( ps  ->  C  =  D )   =>    |-  ( ( ps 
 /\  ph )  ->  ( A F C )  =  ( B F D ) )
 
Theoremoveq123d 5978 Equality deduction for operation value. (Contributed by FL, 22-Dec-2008.)
 |-  ( ph  ->  F  =  G )   &    |-  ( ph  ->  A  =  B )   &    |-  ( ph  ->  C  =  D )   =>    |-  ( ph  ->  ( A F C )  =  ( B G D ) )
 
Theoremfvoveq1d 5979 Equality deduction for nested function and operation value. (Contributed by AV, 23-Jul-2022.)
 |-  ( ph  ->  A  =  B )   =>    |-  ( ph  ->  ( F `  ( A O C ) )  =  ( F `  ( B O C ) ) )
 
Theoremfvoveq1 5980 Equality theorem for nested function and operation value. Closed form of fvoveq1d 5979. (Contributed by AV, 23-Jul-2022.)
 |-  ( A  =  B  ->  ( F `  ( A O C ) )  =  ( F `  ( B O C ) ) )
 
Theoremovanraleqv 5981* Equality theorem for a conjunction with an operation values within a restricted universal quantification. Technical theorem to be used to reduce the size of a significant number of proofs. (Contributed by AV, 13-Aug-2022.)
 |-  ( B  =  X  ->  ( ph  <->  ps ) )   =>    |-  ( B  =  X  ->  ( A. x  e.  V  ( ph  /\  ( A  .x.  B )  =  C )  <->  A. x  e.  V  ( ps  /\  ( A 
 .x.  X )  =  C ) ) )
 
Theoremimbrov2fvoveq 5982 Equality theorem for nested function and operation value in an implication for a binary relation. Technical theorem to be used to reduce the size of a significant number of proofs. (Contributed by AV, 17-Aug-2022.)
 |-  ( X  =  Y  ->  ( ph  <->  ps ) )   =>    |-  ( X  =  Y  ->  ( ( ph  ->  ( F `  (
 ( G `  X )  .x.  O ) ) R A )  <->  ( ps  ->  ( F `  ( ( G `  Y ) 
 .x.  O ) ) R A ) ) )
 
Theoremovrspc2v 5983* If an operation value is element of a class for all operands of two classes, then the operation value is an element of the class for specific operands of the two classes. (Contributed by Mario Carneiro, 6-Dec-2014.)
 |-  ( ( ( X  e.  A  /\  Y  e.  B )  /\  A. x  e.  A  A. y  e.  B  ( x F y )  e.  C )  ->  ( X F Y )  e.  C )
 
Theoremoveqrspc2v 5984* Restricted specialization of operands, using implicit substitution. (Contributed by Mario Carneiro, 6-Dec-2014.)
 |-  ( ( ph  /\  ( x  e.  A  /\  y  e.  B )
 )  ->  ( x F y )  =  ( x G y ) )   =>    |-  ( ( ph  /\  ( X  e.  A  /\  Y  e.  B )
 )  ->  ( X F Y )  =  ( X G Y ) )
 
Theoremoveqdr 5985 Equality of two operations for any two operands. Useful in proofs using *propd theorems. (Contributed by Mario Carneiro, 29-Jun-2015.)
 |-  ( ph  ->  F  =  G )   =>    |-  ( ( ph  /\  ps )  ->  ( x F y )  =  ( x G y ) )
 
Theoremnfovd 5986 Deduction version of bound-variable hypothesis builder nfov 5987. (Contributed by NM, 13-Dec-2005.) (Proof shortened by Andrew Salmon, 22-Oct-2011.)
 |-  ( ph  ->  F/_ x A )   &    |-  ( ph  ->  F/_ x F )   &    |-  ( ph  ->  F/_ x B )   =>    |-  ( ph  ->  F/_ x ( A F B ) )
 
Theoremnfov 5987 Bound-variable hypothesis builder for operation value. (Contributed by NM, 4-May-2004.)
 |-  F/_ x A   &    |-  F/_ x F   &    |-  F/_ x B   =>    |-  F/_ x ( A F B )
 
Theoremoprabidlem 5988* Slight elaboration of exdistrfor 1824. A lemma for oprabid 5989. (Contributed by Jim Kingdon, 15-Jan-2019.)
 |-  ( E. x E. y ( x  =  z  /\  ps )  ->  E. x ( x  =  z  /\  E. y ps ) )
 
Theoremoprabid 5989 The law of concretion. Special case of Theorem 9.5 of [Quine] p. 61. Although this theorem would be useful with a distinct variable condition between  x,  y, and  z, we use ax-bndl 1533 to eliminate that constraint. (Contributed by Mario Carneiro, 20-Mar-2013.)
 |-  ( <. <. x ,  y >. ,  z >.  e.  { <.
 <. x ,  y >. ,  z >.  |  ph }  <->  ph )
 
Theoremfnovex 5990 The result of an operation is a set. (Contributed by Jim Kingdon, 15-Jan-2019.)
 |-  ( ( F  Fn  ( C  X.  D ) 
 /\  A  e.  C  /\  B  e.  D ) 
 ->  ( A F B )  e.  _V )
 
Theoremovexg 5991 Evaluating a set operation at two sets gives a set. (Contributed by Jim Kingdon, 19-Aug-2021.)
 |-  ( ( A  e.  V  /\  F  e.  W  /\  B  e.  X ) 
 ->  ( A F B )  e.  _V )
 
Theoremovssunirng 5992 The result of an operation value is always a subset of the union of the range. (Contributed by Mario Carneiro, 12-Jan-2017.)
 |-  ( ( X  e.  V  /\  Y  e.  W )  ->  ( X F Y )  C_  U. ran  F )
 
Theoremovprc 5993 The value of an operation when the one of the arguments is a proper class. Note: this theorem is dependent on our particular definitions of operation value, function value, and ordered pair. (Contributed by Mario Carneiro, 26-Apr-2015.)
 |- 
 Rel  dom  F   =>    |-  ( -.  ( A  e.  _V  /\  B  e.  _V )  ->  ( A F B )  =  (/) )
 
Theoremovprc1 5994 The value of an operation when the first argument is a proper class. (Contributed by NM, 16-Jun-2004.)
 |- 
 Rel  dom  F   =>    |-  ( -.  A  e.  _V 
 ->  ( A F B )  =  (/) )
 
Theoremovprc2 5995 The value of an operation when the second argument is a proper class. (Contributed by Mario Carneiro, 26-Apr-2015.)
 |- 
 Rel  dom  F   =>    |-  ( -.  B  e.  _V 
 ->  ( A F B )  =  (/) )
 
Theoremcsbov123g 5996 Move class substitution in and out of an operation. (Contributed by NM, 12-Nov-2005.) (Proof shortened by Mario Carneiro, 5-Dec-2016.)
 |-  ( A  e.  D  -> 
 [_ A  /  x ]_ ( B F C )  =  ( [_ A  /  x ]_ B [_ A  /  x ]_ F [_ A  /  x ]_ C ) )
 
Theoremcsbov12g 5997* Move class substitution in and out of an operation. (Contributed by NM, 12-Nov-2005.)
 |-  ( A  e.  V  -> 
 [_ A  /  x ]_ ( B F C )  =  ( [_ A  /  x ]_ B F [_ A  /  x ]_ C ) )
 
Theoremcsbov1g 5998* Move class substitution in and out of an operation. (Contributed by NM, 12-Nov-2005.)
 |-  ( A  e.  V  -> 
 [_ A  /  x ]_ ( B F C )  =  ( [_ A  /  x ]_ B F C ) )
 
Theoremcsbov2g 5999* Move class substitution in and out of an operation. (Contributed by NM, 12-Nov-2005.)
 |-  ( A  e.  V  -> 
 [_ A  /  x ]_ ( B F C )  =  ( B F [_ A  /  x ]_ C ) )
 
Theoremrspceov 6000* A frequently used special case of rspc2ev 2896 for operation values. (Contributed by NM, 21-Mar-2007.)
 |-  ( ( C  e.  A  /\  D  e.  B  /\  S  =  ( C F D ) ) 
 ->  E. x  e.  A  E. y  e.  B  S  =  ( x F y ) )
    < 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-13300 134 13301-13400 135 13401-13500 136 13501-13600 137 13601-13700 138 13701-13800 139 13801-13900 140 13901-14000 141 14001-14100 142 14101-14200 143 14201-14300 144 14301-14400 145 14401-14500 146 14501-14600 147 14601-14700 148 14701-14800 149 14801-14900 150 14901-15000 151 15001-15100 152 15101-15200 153 15201-15300 154 15301-15400 155 15401-15500 156 15501-15600 157 15601-15700 158 15701-15800 159 15801-15900 160 15901-16000 161 16001-16100 162 16101-16164
  Copyright terms: Public domain < Previous  Next >