src/ZF/Cardinal.ML
changeset 5325 f7a5e06adea1
parent 5284 c77e9dd9bafc
child 6068 2d8f3e1f1151
--- a/src/ZF/Cardinal.ML	Mon Aug 17 13:06:29 1998 +0200
+++ b/src/ZF/Cardinal.ML	Mon Aug 17 13:09:08 1998 +0200
@@ -29,16 +29,15 @@
                              gfun RS fun_is_rel RS image_subset]) 1);
 qed "Banach_last_equation";
 
-val prems = goal Cardinal.thy
-    "[| f: X->Y;  g: Y->X |] ==>   \
-\    EX XA XB YA YB. (XA Int XB = 0) & (XA Un XB = X) &    \
-\                    (YA Int YB = 0) & (YA Un YB = Y) &    \
-\                    f``XA=YA & g``YB=XB";
+Goal "[| f: X->Y;  g: Y->X |] ==>   \
+\     EX XA XB YA YB. (XA Int XB = 0) & (XA Un XB = X) &    \
+\                     (YA Int YB = 0) & (YA Un YB = Y) &    \
+\                     f``XA=YA & g``YB=XB";
 by (REPEAT 
     (FIRSTGOAL
      (resolve_tac [refl, exI, conjI, Diff_disjoint, Diff_partition])));
 by (rtac Banach_last_equation 3);
-by (REPEAT (resolve_tac (prems@[fun_is_rel, image_subset, lfp_subset]) 1));
+by (REPEAT (ares_tac [fun_is_rel, image_subset, lfp_subset] 1));
 qed "decomposition";
 
 val prems = goal Cardinal.thy
@@ -740,7 +739,7 @@
 (*Krzysztof Grabczewski's proof that the converse of a finite, well-ordered
   set is well-ordered.  Proofs simplified by lcp. *)
 
-goal Nat.thy "!!n. n:nat ==> wf[n](converse(Memrel(n)))";
+Goal "n:nat ==> wf[n](converse(Memrel(n)))";
 by (etac nat_induct 1);
 by (blast_tac (claset() addIs [wf_onI]) 1);
 by (rtac wf_onI 1);