src/HOL/IMP/Compiler.thy
changeset 23746 a455e69c31cc
parent 20217 25b068a99d2b
child 27362 a6dc1769fdda
--- a/src/HOL/IMP/Compiler.thy	Wed Jul 11 11:13:08 2007 +0200
+++ b/src/HOL/IMP/Compiler.thy	Wed Jul 11 11:14:51 2007 +0200
@@ -54,7 +54,7 @@
 
 text {* The other direction! *}
 
-inductive_cases [elim!]: "(([],p,s),next) : stepa1"
+inductive_cases [elim!]: "(([],p,s),(is',p',s')) : stepa1"
 
 lemma [simp]: "(\<langle>[],q,s\<rangle> -n\<rightarrow> \<langle>p',q',t\<rangle>) = (n=0 \<and> p' = [] \<and> q' = q \<and> t = s)"
 apply(rule iffI)