src/HOL/MicroJava/JVM/JVMExec.thy
changeset 62042 6c6ccf573479
parent 61361 8b5f00202e1a
child 67443 3abf6a722518
--- a/src/HOL/MicroJava/JVM/JVMExec.thy	Sat Jan 02 18:46:36 2016 +0100
+++ b/src/HOL/MicroJava/JVM/JVMExec.thy	Sat Jan 02 18:48:45 2016 +0100
@@ -10,7 +10,7 @@
 
 fun
   exec :: "jvm_prog \<times> jvm_state => jvm_state option"
--- "exec is not recursive. fun is just used for pattern matching"
+\<comment> "exec is not recursive. fun is just used for pattern matching"
 where
   "exec (G, xp, hp, []) = None"
 
@@ -30,8 +30,8 @@
 
 text \<open>
   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 
-  @{text this} pointer of the frame is set to @{text Null} to simulate
+  method \<open>m\<close> of class \<open>C\<close> in program \<open>G\<close>. The 
+  \<open>this\<close> pointer of the frame is set to \<open>Null\<close> to simulate
   a static method invokation.
 \<close>
 definition start_state :: "jvm_prog \<Rightarrow> cname \<Rightarrow> mname \<Rightarrow> jvm_state" where