src/ZF/Cardinal.thy
changeset 13357 6f54e992777e
parent 13356 c9cfe1638bf2
child 13524 604d0f3622d6
--- a/src/ZF/Cardinal.thy	Sun Jul 14 15:14:43 2002 +0200
+++ b/src/ZF/Cardinal.thy	Sun Jul 14 19:59:55 2002 +0200
@@ -9,11 +9,6 @@
 
 theory Cardinal = OrderType + Finite + Nat + Sum:
 
-(*** The following really belong in upair ***)
-
-lemma eq_imp_not_mem: "a=A ==> a ~: A"
-by (blast intro: elim: mem_irrefl)
-
 constdefs
 
   (*least ordinal operator*)
@@ -44,7 +39,8 @@
   "lesspoll"    :: "[i,i] => o"       (infixl "\<prec>" 50)
   "LEAST "         :: "[pttrn, o] => i"  ("(3\<mu>_./ _)" [0, 10] 10)
 
-subsection{*The Schroeder-Bernstein Theorem -- see Davey & Priestly, page 106 *}
+subsection{*The Schroeder-Bernstein Theorem*}
+text{*See Davey and Priestly, page 106*}
 
 (** Lemma: Banach's Decomposition Theorem **)