This commit should not have been necessary. For some reason, the previous
authorlcp
Tue, 21 Sep 1993 11:16:19 +0200
changeset 10 e37080f41102
parent 9 c1795fac88c3
child 11 d0e17c42dbb4
This commit should not have been necessary. For some reason, the previous commit did not update genrec.ML. There were still occurrences of SIMP_TAC. Was the commit perhaps interrupted??
src/CCL/genrec.ML
--- a/src/CCL/genrec.ML	Mon Sep 20 18:39:45 1993 +0200
+++ b/src/CCL/genrec.ML	Tue Sep 21 11:16:19 1993 +0200
@@ -43,7 +43,7 @@
 val letrec2T = result();
 
 goal Wfd.thy "SPLIT(<a,<b,c>>,%x xs.SPLIT(xs,%y z.B(x,y,z))) = B(a,b,c)";
-by (SIMP_TAC (ccl_ss addrews [SPLITB]) 1);
+by (simp_tac (ccl_ss addsimps [SPLITB]) 1);
 val lemma = result();
 
 val prems = goalw Wfd.thy [letrec3_def]
@@ -55,7 +55,7 @@
 \    letrec g x y z be h(x,y,z,g) in g(a,b,c) : D(a,b,c)";
 br (lemma RS subst) 1;
 by (REPEAT (ares_tac ([letrecT,pairT,splitT]@prems) 1));
-by (SIMP_TAC (ccl_ss addrews [SPLITB]) 1);
+by (simp_tac (ccl_ss addsimps [SPLITB]) 1);
 by (REPEAT (ares_tac ([ballI,SubtypeI]@prems) 1));
 br (lemma RS subst) 1;
 by (REPEAT (ares_tac ([letrecT,SubtypeI,pairT,splitT]@prems) 1 ORELSE