src/ZF/Epsilon.ML
changeset 5116 8eb343ab5748
parent 5067 62b6288e6005
child 5137 60205b0de9b9
--- a/src/ZF/Epsilon.ML	Thu Jul 02 17:56:06 1998 +0200
+++ b/src/ZF/Epsilon.ML	Thu Jul 02 17:58:12 1998 +0200
@@ -305,13 +305,13 @@
 Goal "transrec2(succ(i),a,b) = b(i, transrec2(i,a,b))";
 by (rtac (transrec2_def RS def_transrec RS trans) 1);
 by (simp_tac (simpset() addsimps [succ_not_0, THE_eq, if_P]
-                    setloop split_tac [expand_if]) 1);
+                    addsplits [split_if]) 1);
 by (Blast_tac 1);
 qed "transrec2_succ";
 
 Goal "!!i. Limit(i) ==> transrec2(i,a,b) = (UN j<i. transrec2(j,a,b))";
 by (rtac (transrec2_def RS def_transrec RS trans) 1);
-by (simp_tac (simpset() setloop split_tac [expand_if]) 1);
+by (simp_tac (simpset() addsplits [split_if]) 1);
 by (blast_tac (claset() addSDs [Limit_has_0] addSEs [succ_LimitE]) 1);
 qed "transrec2_Limit";