src/HOL/UNITY/GenPrefix.ML
changeset 8442 96023903c2df
parent 8423 3c19160b6432
child 9111 33b32680669a
--- a/src/HOL/UNITY/GenPrefix.ML	Mon Mar 13 15:42:19 2000 +0100
+++ b/src/HOL/UNITY/GenPrefix.ML	Mon Mar 13 16:23:34 2000 +0100
@@ -129,7 +129,7 @@
 
 Goal "((xs, y#ys) : genPrefix r) = \
 \     (xs=[] | (EX z zs. xs=z#zs & (z,y) : r & (zs,ys) : genPrefix r))";
-by (cases_tac "xs" 1);
+by (case_tac "xs" 1);
 by Auto_tac;
 qed "genPrefix_Cons";
 
@@ -183,7 +183,7 @@
 \               --> (xs, ys) : genPrefix r --> (xs ! i, ys ! i) : r";
 by (induct_tac "xs" 1);
 by Auto_tac;
-by (cases_tac "i" 1);
+by (case_tac "i" 1);
 by Auto_tac;
 qed_spec_mp "genPrefix_imp_nth";
 
@@ -194,7 +194,7 @@
 by (ALLGOALS (asm_simp_tac (simpset() addsimps [less_Suc_eq_0_disj, 
 						all_conj_distrib])));
 by (Clarify_tac 1);
-by (cases_tac "ys" 1);
+by (case_tac "ys" 1);
 by (ALLGOALS Force_tac);
 qed_spec_mp "nth_imp_genPrefix";