diff -r f127e949389f -r e0968e1f6fe9 src/HOL/MicroJava/JVM/JVMDefensive.thy --- a/src/HOL/MicroJava/JVM/JVMDefensive.thy Tue Aug 13 22:25:24 2013 +0200 +++ b/src/HOL/MicroJava/JVM/JVMDefensive.thy Tue Aug 13 22:37:58 2013 +0200 @@ -119,14 +119,11 @@ definition exec_all_d :: "jvm_prog \ jvm_state type_error \ jvm_state type_error \ bool" - ("_ |- _ -jvmd-> _" [61,61,61]60) where - "G |- s -jvmd-> t \ + ("_ \ _ \jvmd\ _" [61,61,61]60) where + "G \ s \jvmd\ t \ (s,t) \ ({(s,t). exec_d G s = TypeError \ t = TypeError} \ {(s,t). \t'. exec_d G s = Normal (Some t') \ t = Normal t'})\<^sup>*" -notation (xsymbols) - exec_all_d ("_ \ _ -jvmd\ _" [61,61,61]60) - declare split_paired_All [simp del] declare split_paired_Ex [simp del] @@ -146,9 +143,9 @@ lemma defensive_imp_aggressive: - "G \ (Normal s) -jvmd\ (Normal t) \ G \ s -jvm\ t" + "G \ (Normal s) \jvmd\ (Normal t) \ G \ s \jvm\ t" proof - - have "\x y. G \ x -jvmd\ y \ \s t. x = Normal s \ y = Normal t \ G \ s -jvm\ t" + have "\x y. G \ x \jvmd\ y \ \s t. x = Normal s \ y = Normal t \ G \ s \jvm\ t" apply (unfold exec_all_d_def) apply (erule rtrancl_induct) apply (simp add: exec_all_def) @@ -163,9 +160,9 @@ apply blast done moreover - assume "G \ (Normal s) -jvmd\ (Normal t)" + assume "G \ (Normal s) \jvmd\ (Normal t)" ultimately - show "G \ s -jvm\ t" by blast + show "G \ s \jvm\ t" by blast qed end \ No newline at end of file