src/HOL/IMP/Compiler2.thy
changeset 63540 f8652d0534fa
parent 62390 842917225d56
child 67019 7a3724078363
--- a/src/HOL/IMP/Compiler2.thy	Fri Jul 22 08:02:37 2016 +0200
+++ b/src/HOL/IMP/Compiler2.thy	Fri Jul 22 11:00:43 2016 +0200
@@ -366,9 +366,8 @@
     rest: "P @ P' \<turnstile> (i', s'', stk'') \<rightarrow>^k (n, s', stk')"
     by auto
   from step `size P \<le> i`
-  have "P' \<turnstile> (i - size P, s, stk) \<rightarrow> (i' - size P, s'', stk'')" 
+  have *: "P' \<turnstile> (i - size P, s, stk) \<rightarrow> (i' - size P, s'', stk'')" 
     by (rule exec1_drop_left)
-  moreover
   then have "i' - size P \<in> succs P' 0"
     by (fastforce dest!: succs_iexec1 simp: exec1_def simp del: iexec.simps)
   with `exits P' \<subseteq> {0..}`
@@ -376,8 +375,7 @@
   from rest this `exits P' \<subseteq> {0..}`     
   have "P' \<turnstile> (i' - size P, s'', stk'') \<rightarrow>^k (n - size P, s', stk')"
     by (rule Suc.IH)
-  ultimately
-  show ?case by auto
+  with * show ?case by auto
 qed
 
 lemmas exec_n_drop_Cons =