src/HOL/MicroJava/Comp/AuxLemmas.thy
changeset 52866 438f578ef1d9
parent 44890 22f665a2e91c
child 55466 786edc984c98
--- a/src/HOL/MicroJava/Comp/AuxLemmas.thy	Mon Aug 05 17:14:02 2013 +0200
+++ b/src/HOL/MicroJava/Comp/AuxLemmas.thy	Mon Aug 05 17:52:07 2013 +0200
@@ -15,20 +15,20 @@
 
 
 
-lemma app_nth_greater_len [rule_format (no_asm), simp]:
- "\<forall> ind. length pre \<le> ind \<longrightarrow> (pre @ a # post) ! (Suc ind) = (pre @ post) ! ind"
-apply (induct "pre")
+lemma app_nth_greater_len [simp]:
+ "length pre \<le> ind \<Longrightarrow> (pre @ a # post) ! (Suc ind) = (pre @ post) ! ind"
+apply (induct pre arbitrary: ind)
 apply auto
 apply (case_tac ind)
 apply auto
 done
 
 lemma length_takeWhile: "v \<in> set xs \<Longrightarrow> length (takeWhile (%z. z~=v) xs) < length xs"
-by (induct xs, auto)
+by (induct xs) auto
 
 lemma nth_length_takeWhile [simp]: 
   "v \<in> set xs \<Longrightarrow> xs ! (length (takeWhile (%z. z~=v) xs)) = v"
-by (induct xs, auto)
+by (induct xs) auto
 
 
 lemma map_list_update [simp]: