--- a/ex/Qsort.ML Fri Dec 02 11:43:20 1994 +0100
+++ b/ex/Qsort.ML Fri Dec 02 16:09:49 1994 +0100
@@ -15,13 +15,13 @@
goal Qsort.thy "(Alls x:[x:xs.P(x)].Q(x)) = (Alls x:xs. P(x)-->Q(x))";
-by(list_ind_tac "xs" 1);
+by(list.induct_tac "xs" 1);
by(ALLGOALS(asm_simp_tac (ss setloop (split_tac [expand_if]))));
val ss = ss addsimps [result()];
goal Qsort.thy
"((Alls x:xs.P(x)) & (Alls x:xs.Q(x))) = (Alls x:xs. P(x)&Q(x))";
-by(list_ind_tac "xs" 1);
+by(list.induct_tac "xs" 1);
by(ALLGOALS(asm_simp_tac ss));
val ss = ss addsimps [result()];
@@ -37,7 +37,7 @@
goal Qsort.thy
"sorted(le,xs@ys) = (sorted(le,xs) & sorted(le,ys) & \
\ (Alls x:xs. Alls y:ys. le(x,y)))";
-by(list_ind_tac "xs" 1);
+by(list.induct_tac "xs" 1);
by(ALLGOALS(asm_simp_tac ss));
val ss = ss addsimps [result()];
@@ -69,7 +69,7 @@
goal Qsort.thy
"sorted(le,xs@ys) = (sorted(le,xs) & sorted(le,ys) & \
\ (!x. x mem xs --> (!y. y mem ys --> le(x,y))))";
-by(list_ind_tac "xs" 1);
+by(list.induct_tac "xs" 1);
by(ALLGOALS(asm_simp_tac (ss setloop (split_tac [expand_if]))));
by(fast_tac HOL_cs 1);
val ss = ss addsimps [result()];