src/HOL/IMP/Comp_Rev.thy
changeset 45200 1f1897ac7877
parent 45015 fdac1e9880eb
child 45218 f115540543d8
--- a/src/HOL/IMP/Comp_Rev.thy	Wed Oct 19 09:11:21 2011 +0200
+++ b/src/HOL/IMP/Comp_Rev.thy	Wed Oct 19 16:32:12 2011 +0200
@@ -443,7 +443,7 @@
   shows "i = isize(bcomp b c j) + (if c = bval b s then j else 0) \<and>
          s' = s \<and> stk' = stk"
 using assms proof (induction b arbitrary: c j i n s' stk')
-  case B thus ?case 
+  case Bc thus ?case 
     by (simp split: split_if_asm add: exec_n_simps)
 next
   case (Not b)