diff -r f127e949389f -r e0968e1f6fe9 src/HOL/MicroJava/Comp/CorrComp.thy --- a/src/HOL/MicroJava/Comp/CorrComp.thy Tue Aug 13 22:25:24 2013 +0200 +++ b/src/HOL/MicroJava/Comp/CorrComp.thy Tue Aug 13 22:37:58 2013 +0200 @@ -59,7 +59,7 @@ theorem exec_instr_in_exec_all: "\ exec_instr i G hp stk lvars C S pc frs = (None, hp', frs'); gis (gmb G C S) ! pc = i\ \ - G \ (None, hp, (stk, lvars, C, S, pc) # frs) -jvm\ (None, hp', frs')" + G \ (None, hp, (stk, lvars, C, S, pc) # frs) \jvm\ (None, hp', frs')" apply (simp only: exec_all_def) apply (rule rtrancl_refl [THEN rtrancl_into_rtrancl]) apply (simp add: gis_def gmb_def) @@ -71,7 +71,7 @@ (exec_instr i G hp0 stk0 lvars0 C S pc0 frs) = (None, hp1, (stk1,lvars1,C,S, Suc pc0)#frs) \ \ - G \ (None, hp0, (stk0,lvars0,C,S, pc0)#frs) -jvm\ + G \ (None, hp0, (stk0,lvars0,C,S, pc0)#frs) \jvm\ (None, hp1, (stk1,lvars1,C,S, Suc pc0)#frs)" apply (unfold exec_all_def) apply (rule r_into_rtrancl) @@ -90,7 +90,7 @@ "{G,C,S} \ {hp0, os0, lvars0} >- instrs \ {hp1, os1, lvars1} == \ pre post frs. (gis (gmb G C S) = pre @ instrs @ post) \ - G \ (None,hp0,(os0,lvars0,C,S,length pre)#frs) -jvm\ + G \ (None,hp0,(os0,lvars0,C,S,length pre)#frs) \jvm\ (None,hp1,(os1,lvars1,C,S,(length pre) + (length instrs))#frs)"