src/HOL/IMP/Comp_Rev.thy
changeset 45218 f115540543d8
parent 45200 1f1897ac7877
child 45322 654cc47f6115
--- a/src/HOL/IMP/Comp_Rev.thy	Thu Oct 20 10:44:00 2011 +0200
+++ b/src/HOL/IMP/Comp_Rev.thy	Thu Oct 20 12:30:43 2011 -0400
@@ -39,7 +39,7 @@
 
 lemma exec_0 [intro!]: "P \<turnstile> c \<rightarrow>^0 c" by simp
 
-lemma exec_Suc [trans]:
+lemma exec_Suc:
   "\<lbrakk> P \<turnstile> c \<rightarrow> c'; P \<turnstile> c' \<rightarrow>^n c'' \<rbrakk> \<Longrightarrow> P \<turnstile> c \<rightarrow>^(Suc n) c''" 
   by (fastforce simp del: split_paired_Ex)
 
@@ -350,7 +350,7 @@
   from step `isize P \<le> i`
   have "P' \<turnstile> (i - isize P, s, stk) \<rightarrow> (i' - isize P, s'', stk'')" 
     by (rule exec1_drop_left)
-  also
+  moreover
   then have "i' - isize P \<in> succs P' 0"
     by (fastforce dest!: succs_iexec1)
   with `exits P' \<subseteq> {0..}`
@@ -358,8 +358,8 @@
   from rest this `exits P' \<subseteq> {0..}`     
   have "P' \<turnstile> (i' - isize P, s'', stk'') \<rightarrow>^k (n - isize P, s', stk')"
     by (rule Suc.IH)
-  finally
-  show ?case .
+  ultimately
+  show ?case by auto
 qed
 
 lemmas exec_n_drop_Cons =