(* Title: Jinja/JVM/JVMState.thy Author: Cornelia Pusch, Gerwin Klein, Susannah Mansky Copyright 1999 Technische Universitaet Muenchen, 2019-20 UIUC Based on the Jinja theory JVM/JVMState.thy by Cornelia Pusch and Gerwin Klein *) chapter ‹ Jinja Virtual Machine \label{cha:jvm} › section ‹ State of the JVM › theory JVMState imports "../Common/Objects" begin type_synonym pc = nat abbreviation start_sheap :: "sheap" where "start_sheap ≡ (λx. None)(Start ↦ (Map.empty,Done))" definition start_sheap_preloaded :: "'m prog ⇒ sheap" where "start_sheap_preloaded P ≡ fold (λ(C,cl) f. f(C := Some (sblank P C, Prepared))) P (λx. None)" subsection ‹ Frame Stack ›