HomeHome Intuitionistic Logic Explorer
Theorem List (p. 62 of 108)
< 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 - 6101-6200   *Has distinct variable group(s)
TypeLabelDescription
Statement
 
Theoremnndcel 6101 Set membership between two natural numbers is decidable. (Contributed by Jim Kingdon, 6-Sep-2019.)
 |-  ( ( A  e.  om 
 /\  B  e.  om )  -> DECID  A  e.  B )
 
Theoremnnsseleq 6102 For natural numbers, inclusion is equivalent to membership or equality. (Contributed by Jim Kingdon, 16-Sep-2021.)
 |-  ( ( A  e.  om 
 /\  B  e.  om )  ->  ( A  C_  B 
 <->  ( A  e.  B  \/  A  =  B ) ) )
 
Theoremnndifsnid 6103 If we remove a single element from a natural number then put it back in, we end up with the original natural number. This strengthens difsnss 3531 from subset to equality but the proof relies on equality being decidable. (Contributed by Jim Kingdon, 31-Aug-2021.)
 |-  ( ( A  e.  om 
 /\  B  e.  A )  ->  ( ( A 
 \  { B }
 )  u.  { B } )  =  A )
 
Theoremnnaordi 6104 Ordering property of addition. Proposition 8.4 of [TakeutiZaring] p. 58, limited to natural numbers. (Contributed by NM, 3-Feb-1996.) (Revised by Mario Carneiro, 15-Nov-2014.)
 |-  ( ( B  e.  om 
 /\  C  e.  om )  ->  ( A  e.  B  ->  ( C  +o  A )  e.  ( C  +o  B ) ) )
 
Theoremnnaord 6105 Ordering property of addition. Proposition 8.4 of [TakeutiZaring] p. 58, limited to natural numbers, and its converse. (Contributed by NM, 7-Mar-1996.) (Revised by Mario Carneiro, 15-Nov-2014.)
 |-  ( ( A  e.  om 
 /\  B  e.  om  /\  C  e.  om )  ->  ( A  e.  B  <->  ( C  +o  A )  e.  ( C  +o  B ) ) )
 
Theoremnnaordr 6106 Ordering property of addition of natural numbers. (Contributed by NM, 9-Nov-2002.)
 |-  ( ( A  e.  om 
 /\  B  e.  om  /\  C  e.  om )  ->  ( A  e.  B  <->  ( A  +o  C )  e.  ( B  +o  C ) ) )
 
Theoremnnaword 6107 Weak ordering property of addition. (Contributed by NM, 17-Sep-1995.) (Revised by Mario Carneiro, 15-Nov-2014.)
 |-  ( ( A  e.  om 
 /\  B  e.  om  /\  C  e.  om )  ->  ( A  C_  B  <->  ( C  +o  A ) 
 C_  ( C  +o  B ) ) )
 
Theoremnnacan 6108 Cancellation law for addition of natural numbers. (Contributed by NM, 27-Oct-1995.) (Revised by Mario Carneiro, 15-Nov-2014.)
 |-  ( ( A  e.  om 
 /\  B  e.  om  /\  C  e.  om )  ->  ( ( A  +o  B )  =  ( A  +o  C )  <->  B  =  C ) )
 
Theoremnnaword1 6109 Weak ordering property of addition. (Contributed by NM, 9-Nov-2002.) (Revised by Mario Carneiro, 15-Nov-2014.)
 |-  ( ( A  e.  om 
 /\  B  e.  om )  ->  A  C_  ( A  +o  B ) )
 
Theoremnnaword2 6110 Weak ordering property of addition. (Contributed by NM, 9-Nov-2002.)
 |-  ( ( A  e.  om 
 /\  B  e.  om )  ->  A  C_  ( B  +o  A ) )
 
Theoremnnawordi 6111 Adding to both sides of an inequality in  om (Contributed by Scott Fenton, 16-Apr-2012.) (Revised by Mario Carneiro, 12-May-2012.)
 |-  ( ( A  e.  om 
 /\  B  e.  om  /\  C  e.  om )  ->  ( A  C_  B  ->  ( A  +o  C )  C_  ( B  +o  C ) ) )
 
Theoremnnmordi 6112 Ordering property of multiplication. Half of Proposition 8.19 of [TakeutiZaring] p. 63, limited to natural numbers. (Contributed by NM, 18-Sep-1995.) (Revised by Mario Carneiro, 15-Nov-2014.)
 |-  ( ( ( B  e.  om  /\  C  e.  om )  /\  (/)  e.  C )  ->  ( A  e.  B  ->  ( C  .o  A )  e.  ( C  .o  B ) ) )
 
Theoremnnmord 6113 Ordering property of multiplication. Proposition 8.19 of [TakeutiZaring] p. 63, limited to natural numbers. (Contributed by NM, 22-Jan-1996.) (Revised by Mario Carneiro, 15-Nov-2014.)
 |-  ( ( A  e.  om 
 /\  B  e.  om  /\  C  e.  om )  ->  ( ( A  e.  B  /\  (/)  e.  C )  <-> 
 ( C  .o  A )  e.  ( C  .o  B ) ) )
 
Theoremnnmword 6114 Weak ordering property of ordinal multiplication. (Contributed by Mario Carneiro, 17-Nov-2014.)
 |-  ( ( ( A  e.  om  /\  B  e.  om  /\  C  e.  om )  /\  (/)  e.  C )  ->  ( A  C_  B 
 <->  ( C  .o  A )  C_  ( C  .o  B ) ) )
 
Theoremnnmcan 6115 Cancellation law for multiplication of natural numbers. (Contributed by NM, 26-Oct-1995.) (Revised by Mario Carneiro, 15-Nov-2014.)
 |-  ( ( ( A  e.  om  /\  B  e.  om  /\  C  e.  om )  /\  (/)  e.  A )  ->  ( ( A  .o  B )  =  ( A  .o  C ) 
 <->  B  =  C ) )
 
Theorem1onn 6116 One is a natural number. (Contributed by NM, 29-Oct-1995.)
 |- 
 1o  e.  om
 
Theorem2onn 6117 The ordinal 2 is a natural number. (Contributed by NM, 28-Sep-2004.)
 |- 
 2o  e.  om
 
Theorem3onn 6118 The ordinal 3 is a natural number. (Contributed by Mario Carneiro, 5-Jan-2016.)
 |- 
 3o  e.  om
 
Theorem4onn 6119 The ordinal 4 is a natural number. (Contributed by Mario Carneiro, 5-Jan-2016.)
 |- 
 4o  e.  om
 
Theoremnnm1 6120 Multiply an element of  om by  1o. (Contributed by Mario Carneiro, 17-Nov-2014.)
 |-  ( A  e.  om  ->  ( A  .o  1o )  =  A )
 
Theoremnnm2 6121 Multiply an element of  om by  2o (Contributed by Scott Fenton, 18-Apr-2012.) (Revised by Mario Carneiro, 17-Nov-2014.)
 |-  ( A  e.  om  ->  ( A  .o  2o )  =  ( A  +o  A ) )
 
Theoremnn2m 6122 Multiply an element of  om by  2o (Contributed by Scott Fenton, 16-Apr-2012.) (Revised by Mario Carneiro, 17-Nov-2014.)
 |-  ( A  e.  om  ->  ( 2o  .o  A )  =  ( A  +o  A ) )
 
Theoremnnaordex 6123* Equivalence for ordering. Compare Exercise 23 of [Enderton] p. 88. (Contributed by NM, 5-Dec-1995.) (Revised by Mario Carneiro, 15-Nov-2014.)
 |-  ( ( A  e.  om 
 /\  B  e.  om )  ->  ( A  e.  B 
 <-> 
 E. x  e.  om  ( (/)  e.  x  /\  ( A  +o  x )  =  B )
 ) )
 
Theoremnnawordex 6124* Equivalence for weak ordering of natural numbers. (Contributed by NM, 8-Nov-2002.) (Revised by Mario Carneiro, 15-Nov-2014.)
 |-  ( ( A  e.  om 
 /\  B  e.  om )  ->  ( A  C_  B 
 <-> 
 E. x  e.  om  ( A  +o  x )  =  B )
 )
 
Theoremnnm00 6125 The product of two natural numbers is zero iff at least one of them is zero. (Contributed by Jim Kingdon, 11-Nov-2004.)
 |-  ( ( A  e.  om 
 /\  B  e.  om )  ->  ( ( A  .o  B )  =  (/) 
 <->  ( A  =  (/)  \/  B  =  (/) ) ) )
 
2.6.24  Equivalence relations and classes
 
Syntaxwer 6126 Extend the definition of a wff to include the equivalence predicate.
 wff  R  Er  A
 
Syntaxcec 6127 Extend the definition of a class to include equivalence class.
 class  [ A ] R
 
Syntaxcqs 6128 Extend the definition of a class to include quotient set.
 class  ( A /. R )
 
Definitiondf-er 6129 Define the equivalence relation predicate. Our notation is not standard. A formal notation doesn't seem to exist in the literature; instead only informal English tends to be used. The present definition, although somewhat cryptic, nicely avoids dummy variables. In dfer2 6130 we derive a more typical definition. We show that an equivalence relation is reflexive, symmetric, and transitive in erref 6149, ersymb 6143, and ertr 6144. (Contributed by NM, 4-Jun-1995.) (Revised by Mario Carneiro, 2-Nov-2015.)
 |-  ( R  Er  A  <->  ( Rel  R  /\  dom  R  =  A  /\  ( `' R  u.  ( R  o.  R ) ) 
 C_  R ) )
 
Theoremdfer2 6130* Alternate definition of equivalence predicate. (Contributed by NM, 3-Jan-1997.) (Revised by Mario Carneiro, 12-Aug-2015.)
 |-  ( R  Er  A  <->  ( Rel  R  /\  dom  R  =  A  /\  A. x A. y A. z
 ( ( x R y  ->  y R x )  /\  ( ( x R y  /\  y R z )  ->  x R z ) ) ) )
 
Definitiondf-ec 6131 Define the  R-coset of  A. Exercise 35 of [Enderton] p. 61. This is called the equivalence class of  A modulo  R when  R is an equivalence relation (i.e. when  Er  R; see dfer2 6130). In this case,  A is a representative (member) of the equivalence class  [ A ] R, which contains all sets that are equivalent to  A. Definition of [Enderton] p. 57 uses the notation  [ A ] (subscript)  R, although we simply follow the brackets by  R since we don't have subscripted expressions. For an alternate definition, see dfec2 6132. (Contributed by NM, 23-Jul-1995.)
 |- 
 [ A ] R  =  ( R " { A } )
 
Theoremdfec2 6132* Alternate definition of  R-coset of  A. Definition 34 of [Suppes] p. 81. (Contributed by NM, 3-Jan-1997.) (Proof shortened by Mario Carneiro, 9-Jul-2014.)
 |-  ( A  e.  V  ->  [ A ] R  =  { y  |  A R y } )
 
Theoremecexg 6133 An equivalence class modulo a set is a set. (Contributed by NM, 24-Jul-1995.)
 |-  ( R  e.  B  ->  [ A ] R  e.  _V )
 
Theoremecexr 6134 An inhabited equivalence class implies the representative is a set. (Contributed by Mario Carneiro, 9-Jul-2014.)
 |-  ( A  e.  [ B ] R  ->  B  e.  _V )
 
Definitiondf-qs 6135* Define quotient set.  R is usually an equivalence relation. Definition of [Enderton] p. 58. (Contributed by NM, 23-Jul-1995.)
 |-  ( A /. R )  =  { y  |  E. x  e.  A  y  =  [ x ] R }
 
Theoremereq1 6136 Equality theorem for equivalence predicate. (Contributed by NM, 4-Jun-1995.) (Revised by Mario Carneiro, 12-Aug-2015.)
 |-  ( R  =  S  ->  ( R  Er  A  <->  S  Er  A ) )
 
Theoremereq2 6137 Equality theorem for equivalence predicate. (Contributed by Mario Carneiro, 12-Aug-2015.)
 |-  ( A  =  B  ->  ( R  Er  A  <->  R  Er  B ) )
 
Theoremerrel 6138 An equivalence relation is a relation. (Contributed by Mario Carneiro, 12-Aug-2015.)
 |-  ( R  Er  A  ->  Rel  R )
 
Theoremerdm 6139 The domain of an equivalence relation. (Contributed by Mario Carneiro, 12-Aug-2015.)
 |-  ( R  Er  A  ->  dom  R  =  A )
 
Theoremercl 6140 Elementhood in the field of an equivalence relation. (Contributed by Mario Carneiro, 12-Aug-2015.)
 |-  ( ph  ->  R  Er  X )   &    |-  ( ph  ->  A R B )   =>    |-  ( ph  ->  A  e.  X )
 
Theoremersym 6141 An equivalence relation is symmetric. (Contributed by NM, 4-Jun-1995.) (Revised by Mario Carneiro, 12-Aug-2015.)
 |-  ( ph  ->  R  Er  X )   &    |-  ( ph  ->  A R B )   =>    |-  ( ph  ->  B R A )
 
Theoremercl2 6142 Elementhood in the field of an equivalence relation. (Contributed by Mario Carneiro, 12-Aug-2015.)
 |-  ( ph  ->  R  Er  X )   &    |-  ( ph  ->  A R B )   =>    |-  ( ph  ->  B  e.  X )
 
Theoremersymb 6143 An equivalence relation is symmetric. (Contributed by NM, 30-Jul-1995.) (Revised by Mario Carneiro, 12-Aug-2015.)
 |-  ( ph  ->  R  Er  X )   =>    |-  ( ph  ->  ( A R B  <->  B R A ) )
 
Theoremertr 6144 An equivalence relation is transitive. (Contributed by NM, 4-Jun-1995.) (Revised by Mario Carneiro, 12-Aug-2015.)
 |-  ( ph  ->  R  Er  X )   =>    |-  ( ph  ->  (
 ( A R B  /\  B R C ) 
 ->  A R C ) )
 
Theoremertrd 6145 A transitivity relation for equivalences. (Contributed by Mario Carneiro, 9-Jul-2014.)
 |-  ( ph  ->  R  Er  X )   &    |-  ( ph  ->  A R B )   &    |-  ( ph  ->  B R C )   =>    |-  ( ph  ->  A R C )
 
Theoremertr2d 6146 A transitivity relation for equivalences. (Contributed by Mario Carneiro, 9-Jul-2014.)
 |-  ( ph  ->  R  Er  X )   &    |-  ( ph  ->  A R B )   &    |-  ( ph  ->  B R C )   =>    |-  ( ph  ->  C R A )
 
Theoremertr3d 6147 A transitivity relation for equivalences. (Contributed by Mario Carneiro, 9-Jul-2014.)
 |-  ( ph  ->  R  Er  X )   &    |-  ( ph  ->  B R A )   &    |-  ( ph  ->  B R C )   =>    |-  ( ph  ->  A R C )
 
Theoremertr4d 6148 A transitivity relation for equivalences. (Contributed by Mario Carneiro, 9-Jul-2014.)
 |-  ( ph  ->  R  Er  X )   &    |-  ( ph  ->  A R B )   &    |-  ( ph  ->  C R B )   =>    |-  ( ph  ->  A R C )
 
Theoremerref 6149 An equivalence relation is reflexive on its field. Compare Theorem 3M of [Enderton] p. 56. (Contributed by Mario Carneiro, 6-May-2013.) (Revised by Mario Carneiro, 12-Aug-2015.)
 |-  ( ph  ->  R  Er  X )   &    |-  ( ph  ->  A  e.  X )   =>    |-  ( ph  ->  A R A )
 
Theoremercnv 6150 The converse of an equivalence relation is itself. (Contributed by Mario Carneiro, 12-Aug-2015.)
 |-  ( R  Er  A  ->  `' R  =  R )
 
Theoremerrn 6151 The range and domain of an equivalence relation are equal. (Contributed by Rodolfo Medina, 11-Oct-2010.) (Revised by Mario Carneiro, 12-Aug-2015.)
 |-  ( R  Er  A  ->  ran  R  =  A )
 
Theoremerssxp 6152 An equivalence relation is a subset of the cartesian product of the field. (Contributed by Mario Carneiro, 12-Aug-2015.)
 |-  ( R  Er  A  ->  R  C_  ( A  X.  A ) )
 
Theoremerex 6153 An equivalence relation is a set if its domain is a set. (Contributed by Rodolfo Medina, 15-Oct-2010.) (Proof shortened by Mario Carneiro, 12-Aug-2015.)
 |-  ( R  Er  A  ->  ( A  e.  V  ->  R  e.  _V )
 )
 
Theoremerexb 6154 An equivalence relation is a set if and only if its domain is a set. (Contributed by Rodolfo Medina, 15-Oct-2010.) (Revised by Mario Carneiro, 12-Aug-2015.)
 |-  ( R  Er  A  ->  ( R  e.  _V  <->  A  e.  _V ) )
 
Theoremiserd 6155* A reflexive, symmetric, transitive relation is an equivalence relation on its domain. (Contributed by Mario Carneiro, 9-Jul-2014.) (Revised by Mario Carneiro, 12-Aug-2015.)
 |-  ( ph  ->  Rel  R )   &    |-  ( ( ph  /\  x R y )  ->  y R x )   &    |-  (
 ( ph  /\  ( x R y  /\  y R z ) ) 
 ->  x R z )   &    |-  ( ph  ->  ( x  e.  A  <->  x R x ) )   =>    |-  ( ph  ->  R  Er  A )
 
Theorembrdifun 6156 Evaluate the incomparability relation. (Contributed by Mario Carneiro, 9-Jul-2014.)
 |-  R  =  ( ( X  X.  X ) 
 \  (  .<  u.  `'  .<  ) )   =>    |-  ( ( A  e.  X  /\  B  e.  X )  ->  ( A R B 
 <->  -.  ( A  .<  B  \/  B  .<  A ) ) )
 
Theoremswoer 6157* Incomparability under a strict weak partial order is an equivalence relation. (Contributed by Mario Carneiro, 9-Jul-2014.) (Revised by Mario Carneiro, 12-Aug-2015.)
 |-  R  =  ( ( X  X.  X ) 
 \  (  .<  u.  `'  .<  ) )   &    |-  ( ( ph  /\  ( y  e.  X  /\  z  e.  X ) )  ->  ( y 
 .<  z  ->  -.  z  .<  y ) )   &    |-  (
 ( ph  /\  ( x  e.  X  /\  y  e.  X  /\  z  e.  X ) )  ->  ( x  .<  y  ->  ( x  .<  z  \/  z  .<  y )
 ) )   =>    |-  ( ph  ->  R  Er  X )
 
Theoremswoord1 6158* The incomparability equivalence relation is compatible with the original order. (Contributed by Mario Carneiro, 31-Dec-2014.)
 |-  R  =  ( ( X  X.  X ) 
 \  (  .<  u.  `'  .<  ) )   &    |-  ( ( ph  /\  ( y  e.  X  /\  z  e.  X ) )  ->  ( y 
 .<  z  ->  -.  z  .<  y ) )   &    |-  (
 ( ph  /\  ( x  e.  X  /\  y  e.  X  /\  z  e.  X ) )  ->  ( x  .<  y  ->  ( x  .<  z  \/  z  .<  y )
 ) )   &    |-  ( ph  ->  B  e.  X )   &    |-  ( ph  ->  C  e.  X )   &    |-  ( ph  ->  A R B )   =>    |-  ( ph  ->  ( A  .<  C  <->  B  .<  C ) )
 
Theoremswoord2 6159* The incomparability equivalence relation is compatible with the original order. (Contributed by Mario Carneiro, 31-Dec-2014.)
 |-  R  =  ( ( X  X.  X ) 
 \  (  .<  u.  `'  .<  ) )   &    |-  ( ( ph  /\  ( y  e.  X  /\  z  e.  X ) )  ->  ( y 
 .<  z  ->  -.  z  .<  y ) )   &    |-  (
 ( ph  /\  ( x  e.  X  /\  y  e.  X  /\  z  e.  X ) )  ->  ( x  .<  y  ->  ( x  .<  z  \/  z  .<  y )
 ) )   &    |-  ( ph  ->  B  e.  X )   &    |-  ( ph  ->  C  e.  X )   &    |-  ( ph  ->  A R B )   =>    |-  ( ph  ->  ( C  .<  A  <->  C  .<  B ) )
 
Theoremeqerlem 6160* Lemma for eqer 6161. (Contributed by NM, 17-Mar-2008.) (Proof shortened by Mario Carneiro, 6-Dec-2016.)
 |-  ( x  =  y 
 ->  A  =  B )   &    |-  R  =  { <. x ,  y >.  |  A  =  B }   =>    |-  ( z R w  <->  [_ z  /  x ]_ A  =  [_ w  /  x ]_ A )
 
Theoremeqer 6161* Equivalence relation involving equality of dependent classes  A
( x ) and  B ( y ). (Contributed by NM, 17-Mar-2008.) (Revised by Mario Carneiro, 12-Aug-2015.)
 |-  ( x  =  y 
 ->  A  =  B )   &    |-  R  =  { <. x ,  y >.  |  A  =  B }   =>    |-  R  Er  _V
 
Theoremider 6162 The identity relation is an equivalence relation. (Contributed by NM, 10-May-1998.) (Proof shortened by Andrew Salmon, 22-Oct-2011.) (Proof shortened by Mario Carneiro, 9-Jul-2014.)
 |- 
 _I  Er  _V
 
Theorem0er 6163 The empty set is an equivalence relation on the empty set. (Contributed by Mario Carneiro, 5-Sep-2015.)
 |-  (/)  Er  (/)
 
Theoremeceq1 6164 Equality theorem for equivalence class. (Contributed by NM, 23-Jul-1995.)
 |-  ( A  =  B  ->  [ A ] C  =  [ B ] C )
 
Theoremeceq1d 6165 Equality theorem for equivalence class (deduction form). (Contributed by Jim Kingdon, 31-Dec-2019.)
 |-  ( ph  ->  A  =  B )   =>    |-  ( ph  ->  [ A ] C  =  [ B ] C )
 
Theoremeceq2 6166 Equality theorem for equivalence class. (Contributed by NM, 23-Jul-1995.)
 |-  ( A  =  B  ->  [ C ] A  =  [ C ] B )
 
Theoremelecg 6167 Membership in an equivalence class. Theorem 72 of [Suppes] p. 82. (Contributed by Mario Carneiro, 9-Jul-2014.)
 |-  ( ( A  e.  V  /\  B  e.  W )  ->  ( A  e.  [ B ] R  <->  B R A ) )
 
Theoremelec 6168 Membership in an equivalence class. Theorem 72 of [Suppes] p. 82. (Contributed by NM, 23-Jul-1995.)
 |-  A  e.  _V   &    |-  B  e.  _V   =>    |-  ( A  e.  [ B ] R  <->  B R A )
 
Theoremrelelec 6169 Membership in an equivalence class when  R is a relation. (Contributed by Mario Carneiro, 11-Sep-2015.)
 |-  ( Rel  R  ->  ( A  e.  [ B ] R  <->  B R A ) )
 
Theoremecss 6170 An equivalence class is a subset of the domain. (Contributed by NM, 6-Aug-1995.) (Revised by Mario Carneiro, 12-Aug-2015.)
 |-  ( ph  ->  R  Er  X )   =>    |-  ( ph  ->  [ A ] R  C_  X )
 
Theoremecdmn0m 6171* A representative of an inhabited equivalence class belongs to the domain of the equivalence relation. (Contributed by Jim Kingdon, 21-Aug-2019.)
 |-  ( A  e.  dom  R  <->  E. x  x  e.  [ A ] R )
 
Theoremereldm 6172 Equality of equivalence classes implies equivalence of domain membership. (Contributed by NM, 28-Jan-1996.) (Revised by Mario Carneiro, 12-Aug-2015.)
 |-  ( ph  ->  R  Er  X )   &    |-  ( ph  ->  [ A ] R  =  [ B ] R )   =>    |-  ( ph  ->  ( A  e.  X  <->  B  e.  X ) )
 
Theoremerth 6173 Basic property of equivalence relations. Theorem 73 of [Suppes] p. 82. (Contributed by NM, 23-Jul-1995.) (Revised by Mario Carneiro, 6-Jul-2015.)
 |-  ( ph  ->  R  Er  X )   &    |-  ( ph  ->  A  e.  X )   =>    |-  ( ph  ->  ( A R B  <->  [ A ] R  =  [ B ] R ) )
 
Theoremerth2 6174 Basic property of equivalence relations. Compare Theorem 73 of [Suppes] p. 82. Assumes membership of the second argument in the domain. (Contributed by NM, 30-Jul-1995.) (Revised by Mario Carneiro, 6-Jul-2015.)
 |-  ( ph  ->  R  Er  X )   &    |-  ( ph  ->  B  e.  X )   =>    |-  ( ph  ->  ( A R B  <->  [ A ] R  =  [ B ] R ) )
 
Theoremerthi 6175 Basic property of equivalence relations. Part of Lemma 3N of [Enderton] p. 57. (Contributed by NM, 30-Jul-1995.) (Revised by Mario Carneiro, 9-Jul-2014.)
 |-  ( ph  ->  R  Er  X )   &    |-  ( ph  ->  A R B )   =>    |-  ( ph  ->  [ A ] R  =  [ B ] R )
 
Theoremecidsn 6176 An equivalence class modulo the identity relation is a singleton. (Contributed by NM, 24-Oct-2004.)
 |- 
 [ A ]  _I  =  { A }
 
Theoremqseq1 6177 Equality theorem for quotient set. (Contributed by NM, 23-Jul-1995.)
 |-  ( A  =  B  ->  ( A /. C )  =  ( B /. C ) )
 
Theoremqseq2 6178 Equality theorem for quotient set. (Contributed by NM, 23-Jul-1995.)
 |-  ( A  =  B  ->  ( C /. A )  =  ( C /. B ) )
 
Theoremelqsg 6179* Closed form of elqs 6180. (Contributed by Rodolfo Medina, 12-Oct-2010.)
 |-  ( B  e.  V  ->  ( B  e.  ( A /. R )  <->  E. x  e.  A  B  =  [ x ] R ) )
 
Theoremelqs 6180* Membership in a quotient set. (Contributed by NM, 23-Jul-1995.)
 |-  B  e.  _V   =>    |-  ( B  e.  ( A /. R )  <->  E. x  e.  A  B  =  [ x ] R )
 
Theoremelqsi 6181* Membership in a quotient set. (Contributed by NM, 23-Jul-1995.)
 |-  ( B  e.  ( A /. R )  ->  E. x  e.  A  B  =  [ x ] R )
 
Theoremecelqsg 6182 Membership of an equivalence class in a quotient set. (Contributed by Jeff Madsen, 10-Jun-2010.) (Revised by Mario Carneiro, 9-Jul-2014.)
 |-  ( ( R  e.  V  /\  B  e.  A )  ->  [ B ] R  e.  ( A /. R ) )
 
Theoremecelqsi 6183 Membership of an equivalence class in a quotient set. (Contributed by NM, 25-Jul-1995.) (Revised by Mario Carneiro, 9-Jul-2014.)
 |-  R  e.  _V   =>    |-  ( B  e.  A  ->  [ B ] R  e.  ( A /. R ) )
 
Theoremecopqsi 6184 "Closure" law for equivalence class of ordered pairs. (Contributed by NM, 25-Mar-1996.)
 |-  R  e.  _V   &    |-  S  =  ( ( A  X.  A ) /. R )   =>    |-  ( ( B  e.  A  /\  C  e.  A )  ->  [ <. B ,  C >. ] R  e.  S )
 
Theoremqsexg 6185 A quotient set exists. (Contributed by FL, 19-May-2007.) (Revised by Mario Carneiro, 9-Jul-2014.)
 |-  ( A  e.  V  ->  ( A /. R )  e.  _V )
 
Theoremqsex 6186 A quotient set exists. (Contributed by NM, 14-Aug-1995.)
 |-  A  e.  _V   =>    |-  ( A /. R )  e.  _V
 
Theoremuniqs 6187 The union of a quotient set. (Contributed by NM, 9-Dec-2008.)
 |-  ( R  e.  V  ->  U. ( A /. R )  =  ( R " A ) )
 
Theoremqsss 6188 A quotient set is a set of subsets of the base set. (Contributed by Mario Carneiro, 9-Jul-2014.) (Revised by Mario Carneiro, 12-Aug-2015.)
 |-  ( ph  ->  R  Er  A )   =>    |-  ( ph  ->  ( A /. R )  C_  ~P A )
 
Theoremuniqs2 6189 The union of a quotient set. (Contributed by Mario Carneiro, 11-Jul-2014.)
 |-  ( ph  ->  R  Er  A )   &    |-  ( ph  ->  R  e.  V )   =>    |-  ( ph  ->  U. ( A /. R )  =  A )
 
Theoremsnec 6190 The singleton of an equivalence class. (Contributed by NM, 29-Jan-1999.) (Revised by Mario Carneiro, 9-Jul-2014.)
 |-  A  e.  _V   =>    |-  { [ A ] R }  =  ( { A } /. R )
 
Theoremecqs 6191 Equivalence class in terms of quotient set. (Contributed by NM, 29-Jan-1999.)
 |-  R  e.  _V   =>    |-  [ A ] R  =  U. ( { A } /. R )
 
Theoremecid 6192 A set is equal to its converse epsilon coset. (Note: converse epsilon is not an equivalence relation.) (Contributed by NM, 13-Aug-1995.) (Revised by Mario Carneiro, 9-Jul-2014.)
 |-  A  e.  _V   =>    |-  [ A ] `'  _E  =  A
 
Theoremecidg 6193 A set is equal to its converse epsilon coset. (Note: converse epsilon is not an equivalence relation.) (Contributed by Jim Kingdon, 8-Jan-2020.)
 |-  ( A  e.  V  ->  [ A ] `'  _E  =  A )
 
Theoremqsid 6194 A set is equal to its quotient set mod converse epsilon. (Note: converse epsilon is not an equivalence relation.) (Contributed by NM, 13-Aug-1995.) (Revised by Mario Carneiro, 9-Jul-2014.)
 |-  ( A /. `'  _E  )  =  A
 
Theoremectocld 6195* Implicit substitution of class for equivalence class. (Contributed by Mario Carneiro, 9-Jul-2014.)
 |-  S  =  ( B
 /. R )   &    |-  ( [ x ] R  =  A  ->  ( ph  <->  ps ) )   &    |-  (
 ( ch  /\  x  e.  B )  ->  ph )   =>    |-  (
 ( ch  /\  A  e.  S )  ->  ps )
 
Theoremectocl 6196* Implicit substitution of class for equivalence class. (Contributed by NM, 23-Jul-1995.) (Revised by Mario Carneiro, 9-Jul-2014.)
 |-  S  =  ( B
 /. R )   &    |-  ( [ x ] R  =  A  ->  ( ph  <->  ps ) )   &    |-  ( x  e.  B  ->  ph )   =>    |-  ( A  e.  S  ->  ps )
 
Theoremelqsn0m 6197* An element of a quotient set is inhabited. (Contributed by Jim Kingdon, 21-Aug-2019.)
 |-  ( ( dom  R  =  A  /\  B  e.  ( A /. R ) )  ->  E. x  x  e.  B )
 
Theoremelqsn0 6198 A quotient set doesn't contain the empty set. (Contributed by NM, 24-Aug-1995.)
 |-  ( ( dom  R  =  A  /\  B  e.  ( A /. R ) )  ->  B  =/=  (/) )
 
Theoremecelqsdm 6199 Membership of an equivalence class in a quotient set. (Contributed by NM, 30-Jul-1995.)
 |-  ( ( dom  R  =  A  /\  [ B ] R  e.  ( A /. R ) ) 
 ->  B  e.  A )
 
Theoremxpiderm 6200* A square Cartesian product is an equivalence relation (in general it's not a poset). (Contributed by Jim Kingdon, 22-Aug-2019.)
 |-  ( E. x  x  e.  A  ->  ( A  X.  A )  Er  A )
    < 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-10795
  Copyright terms: Public domain < Previous  Next >