diff -r a273bdac0934 -r 8b5f00202e1a src/HOL/MicroJava/JVM/JVMState.thy --- a/src/HOL/MicroJava/JVM/JVMState.thy Wed Oct 07 19:45:00 2015 +0200 +++ b/src/HOL/MicroJava/JVM/JVMState.thy Wed Oct 07 23:28:49 2015 +0200 @@ -2,15 +2,15 @@ Author: Cornelia Pusch, Gerwin Klein, Technische Universitaet Muenchen *) -chapter {* Java Virtual Machine \label{cha:jvm} *} +chapter \Java Virtual Machine \label{cha:jvm}\ -section {* State of the JVM *} +section \State of the JVM\ theory JVMState imports "../J/Conform" begin -subsection {* Frame Stack *} +subsection \Frame Stack\ type_synonym opstack = "val list" type_synonym locvars = "val list" type_synonym p_count = nat @@ -29,16 +29,16 @@ -- "program counter within frame" -subsection {* Exceptions *} +subsection \Exceptions\ definition raise_system_xcpt :: "bool \ xcpt \ val option" where "raise_system_xcpt b x \ raise_if b x None" -subsection {* Runtime State *} +subsection \Runtime State\ type_synonym jvm_state = "val option \ aheap \ frame list" -- "exception flag, heap, frames" -subsection {* Lemmas *} +subsection \Lemmas\ lemma new_Addr_OutOfMemory: "snd (new_Addr hp) = Some xcp \ xcp = Addr (XcptRef OutOfMemory)"