author | kleing |
Sat, 10 Aug 2013 10:15:30 +0200 | |
changeset 52952 | 07423b37bc22 |
parent 52951 | de4bccddcdbd |
child 52953 | 2c927b7501c5 |
--- a/src/HOL/IMP/Compiler.thy Sat Aug 10 09:06:42 2013 +0200 +++ b/src/HOL/IMP/Compiler.thy Sat Aug 10 10:15:30 2013 +0200 @@ -107,7 +107,7 @@ "P \<turnstile> (i,s,stk) \<rightarrow> (i',s',stk') \<Longrightarrow> P' @ P \<turnstile> (size(P')+i,s,stk) \<rightarrow> (size(P')+i',s',stk')" unfolding exec1_def - by (auto split: instr.split) + by (auto simp del: iexec.simps) lemma exec_appendL: fixes i i' :: int