tidied
authorpaulson
Thu, 10 Sep 1998 17:40:03 +0200
changeset 5468 079d8eb6db19
parent 5467 f864dbcda5f1
child 5469 024d887eae50
tidied
src/ZF/upair.ML
--- a/src/ZF/upair.ML	Thu Sep 10 17:38:36 1998 +0200
+++ b/src/ZF/upair.ML	Thu Sep 10 17:40:03 1998 +0200
@@ -16,14 +16,13 @@
 
 val Pow_bottom = empty_subsetI RS PowI;         (* 0 : Pow(B) *)
 val Pow_top = subset_refl RS PowI;              (* A : Pow(A) *)
-val Pow_neq_0 = Pow_top RSN (2,equals0E);       (* Pow(a)=0 ==> P *) 
 
 
 (*** Unordered pairs - Upair ***)
 
 qed_goalw "Upair_iff" thy [Upair_def]
     "c : Upair(a,b) <-> (c=a | c=b)"
- (fn _ => [ (blast_tac (claset() addEs [Pow_neq_0, sym RS Pow_neq_0]) 1) ]);
+ (fn _ => [ (Blast_tac 1) ]);
 
 Addsimps [Upair_iff];