src/HOL/MicroJava/JVM/JVMExecInstr.thy
changeset 62042 6c6ccf573479
parent 61361 8b5f00202e1a
child 62390 842917225d56
--- a/src/HOL/MicroJava/JVM/JVMExecInstr.thy	Sat Jan 02 18:46:36 2016 +0100
+++ b/src/HOL/MicroJava/JVM/JVMExecInstr.thy	Sat Jan 02 18:48:45 2016 +0100
@@ -67,8 +67,8 @@
               else []
    in 
       (xp', hp, frs'@(stk, vars, Cl, sig, pc)#frs))" |
-  -- "Because exception handling needs the pc of the Invoke instruction,"
-  -- "Invoke doesn't change stk and pc yet (@{text Return} does that)."
+  \<comment> "Because exception handling needs the pc of the Invoke instruction,"
+  \<comment> "Invoke doesn't change stk and pc yet (\<open>Return\<close> does that)."
 
  "exec_instr Return G hp stk0 vars Cl sig0 pc frs =
   (if frs=[] then 
@@ -78,8 +78,8 @@
          (mn,pt) = sig0; n = length pt
    in 
       (None, hp, (val#(drop (n+1) stk),loc,C,sig,pc+1)#tl frs))"
-  -- "Return drops arguments from the caller's stack and increases"
-  -- "the program counter in the caller" |
+  \<comment> "Return drops arguments from the caller's stack and increases"
+  \<comment> "the program counter in the caller" |
 
  "exec_instr Pop G hp stk vars Cl sig pc frs = 
       (None, hp, (tl stk, vars, Cl, sig, pc+1)#frs)" |