src/ZF/AC/first.ML
changeset 1196 d43c1f7a53fe
parent 1123 5dfdc1464966
child 1208 bc3093616ba4
--- a/src/ZF/AC/first.ML	Tue Jul 25 17:03:59 1995 +0200
+++ b/src/ZF/AC/first.ML	Tue Jul 25 17:31:53 1995 +0200
@@ -11,18 +11,6 @@
 by (fast_tac AC_cs 1);
 val first_is_elem = result();
 
-goalw thy [well_ord_def, wf_on_def, wf_def, exists_first_def, first_def]
-	"!!r. well_ord(A,r) ==> ALL B. (B<=A & B~=0) --> exists_first(B,r)";
-by (resolve_tac [allI] 1);
-by (resolve_tac [impI] 1);
-by (REPEAT (eresolve_tac [conjE,allE,disjE] 1));
-by (contr_tac 1);
-by (eresolve_tac [bexE] 1);
-by (resolve_tac [bexI] 1 THEN (atac 2));
-by (rewrite_goals_tac [tot_ord_def, linear_def]);
-by (fast_tac ZF_cs 1);
-val well_ord_imp_ex_first = result();
-
 goalw thy [well_ord_def, wf_on_def, wf_def, 	first_def] 
 	"!!r. [| well_ord(A,r); B<=A; B~=0 |] ==> (EX! b. first(b,B,r))";
 by (REPEAT (eresolve_tac [conjE,allE,disjE] 1));
@@ -35,7 +23,7 @@
 val well_ord_imp_ex1_first = result();
 
 goal thy "!!r. [| well_ord(A,r); B<=A; B~=0 |] ==> (THE b. first(b,B,r)) : B";
-by (dresolve_tac [well_ord_imp_ex1_first] 1 THEN REPEAT (atac 1));
+by (dresolve_tac [well_ord_imp_ex1_first] 1 THEN REPEAT (assume_tac 1));
 by (resolve_tac [first_is_elem] 1);
 by (eresolve_tac [theI] 1);
 val the_first_in = result();