src/ZF/AC/AC16_WO4.ML
changeset 6176 707b6f9859d2
parent 6112 5e4871c5136b
child 7499 23e090051cb8
--- a/src/ZF/AC/AC16_WO4.ML	Wed Feb 03 15:49:24 1999 +0100
+++ b/src/ZF/AC/AC16_WO4.ML	Wed Feb 03 15:50:37 1999 +0100
@@ -76,10 +76,7 @@
 Goal "[| ~(EX x:A. f`x=y); f : inj(A, B); y:B |]  \
 \     ==> (lam a:succ(A). if(a=A, y, f`a)) : inj(succ(A), B)";
 by (res_inst_tac [("d","%z. if(z=y, A, converse(f)`z)")] lam_injective 1);
-by (ALLGOALS
-    (asm_simp_tac 
-     (simpset() addsimps [inj_is_fun RS apply_type, left_inverse] 
-      setloop (split_tac [split_if] ORELSE' Step_tac))));
+by (auto_tac (claset(), simpset() addsimps [inj_is_fun RS apply_type]));
 qed "succ_not_lepoll_lemma";
 
 Goalw [lepoll_def, eqpoll_def, bij_def, surj_def]