diff -r 52a87574bca9 -r 6c6ccf573479 src/HOL/MicroJava/JVM/JVMState.thy --- a/src/HOL/MicroJava/JVM/JVMState.thy Sat Jan 02 18:46:36 2016 +0100 +++ b/src/HOL/MicroJava/JVM/JVMState.thy Sat Jan 02 18:48:45 2016 +0100 @@ -22,11 +22,11 @@ sig \ p_count" - -- "operand stack" - -- "local variables (including this pointer and method parameters)" - -- "name of class where current method is defined" - -- "method name + parameter types" - -- "program counter within frame" + \ "operand stack" + \ "local variables (including this pointer and method parameters)" + \ "name of class where current method is defined" + \ "method name + parameter types" + \ "program counter within frame" subsection \Exceptions\ @@ -35,7 +35,7 @@ subsection \Runtime State\ type_synonym - jvm_state = "val option \ aheap \ frame list" -- "exception flag, heap, frames" + jvm_state = "val option \ aheap \ frame list" \ "exception flag, heap, frames" subsection \Lemmas\