diff -r de4bccddcdbd -r 07423b37bc22 src/HOL/IMP/Compiler.thy --- 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 \ (i,s,stk) \ (i',s',stk') \ P' @ P \ (size(P')+i,s,stk) \ (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