src/HOL/MicroJava/JVM/JVMExecInstr.thy
changeset 67443 3abf6a722518
parent 62390 842917225d56
--- a/src/HOL/MicroJava/JVM/JVMExecInstr.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/HOL/MicroJava/JVM/JVMExecInstr.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -67,8 +67,8 @@
               else []
    in 
       (xp', hp, frs'@(stk, vars, Cl, sig, pc)#frs))" |
-  \<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)."
+  \<comment> \<open>Because exception handling needs the pc of the Invoke instruction,\<close>
+  \<comment> \<open>Invoke doesn't change stk and pc yet (\<open>Return\<close> does that).\<close>
 
  "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))"
-  \<comment> "Return drops arguments from the caller's stack and increases"
-  \<comment> "the program counter in the caller" |
+  \<comment> \<open>Return drops arguments from the caller's stack and increases\<close>
+  \<comment> \<open>the program counter in the caller\<close> |
 
  "exec_instr Pop G hp stk vars Cl sig pc frs = 
       (None, hp, (tl stk, vars, Cl, sig, pc+1)#frs)" |