src/HOL/List.thy
changeset 15251 bb6f072c8d10
parent 15246 0984a2c2868b
child 15281 bd4611956c7b
--- a/src/HOL/List.thy	Mon Oct 18 13:40:45 2004 +0200
+++ b/src/HOL/List.thy	Tue Oct 19 18:18:45 2004 +0200
@@ -838,7 +838,7 @@
 done
 
 lemma set_conv_nth: "set xs = {xs!i | i. i < length xs}"
-apply (induct_tac xs, simp, simp)
+apply (induct xs, simp, simp)
 apply safe
 apply (rule_tac x = 0 in exI, simp)
  apply (rule_tac x = "Suc i" in exI, simp)
@@ -1503,10 +1503,10 @@
 by (induct xs) auto
 
 lemma remdups_eq_nil_iff [simp]: "(remdups x = []) = (x = [])"
-  by (induct_tac x, auto) 
+  by (induct x, auto) 
 
 lemma remdups_eq_nil_right_iff [simp]: "([] = remdups x) = (x = [])"
-  by (induct_tac x, auto)
+  by (induct x, auto)
 
 lemma length_remdups_leq[iff]: "length(remdups xs) <= length xs"
 by (induct xs) auto
@@ -1528,7 +1528,7 @@
 it is useful. *}
 lemma distinct_conv_nth:
 "distinct xs = (\<forall>i j. i < size xs \<and> j < size xs \<and> i \<noteq> j --> xs!i \<noteq> xs!j)"
-apply (induct_tac xs, simp, simp)
+apply (induct xs, simp, simp)
 apply (rule iffI, clarsimp)
  apply (case_tac i)
 apply (case_tac j, simp)
@@ -1653,7 +1653,7 @@
 subsection {* Lexicographic orderings on lists *}
 
 lemma wf_lexn: "wf r ==> wf (lexn r n)"
-apply (induct_tac n, simp, simp)
+apply (induct n, simp, simp)
 apply(rule wf_subset)
  prefer 2 apply (rule Int_lower1)
 apply(rule wf_prod_fun_image)
@@ -1678,7 +1678,7 @@
 "lexn r n =
 {(xs,ys). length xs = n \<and> length ys = n \<and>
 (\<exists>xys x y xs' ys'. xs= xys @ x#xs' \<and> ys= xys @ y # ys' \<and> (x, y):r)}"
-apply (induct_tac n, simp, blast)
+apply (induct n, simp, blast)
 apply (simp add: image_Collect lex_prod_def, safe, blast)
  apply (rule_tac x = "ab # xys" in exI, simp)
 apply (case_tac xys, simp_all, blast)