diff -r f127e949389f -r e0968e1f6fe9 src/HOL/MicroJava/JVM/JVMExec.thy --- a/src/HOL/MicroJava/JVM/JVMExec.thy Tue Aug 13 22:25:24 2013 +0200 +++ b/src/HOL/MicroJava/JVM/JVMExec.thy Tue Aug 13 22:37:58 2013 +0200 @@ -24,13 +24,10 @@ definition exec_all :: "[jvm_prog,jvm_state,jvm_state] => bool" - ("_ |- _ -jvm-> _" [61,61,61]60) where - "G |- s -jvm-> t == (s,t) \ {(s,t). exec(G,s) = Some t}^*" + ("_ \ _ \jvm\ _" [61,61,61]60) where + "G \ s \jvm\ t == (s,t) \ {(s,t). exec(G,s) = Some t}^*" -notation (xsymbols) - exec_all ("_ \ _ -jvm\ _" [61,61,61]60) - text {* The start configuration of the JVM: in the start heap, we call a method @{text m} of class @{text C} in program @{text G}. The