src/HOL/MicroJava/BV/Typing_Framework_JVM.thy
changeset 16417 9bc16273c2d4
parent 14045 a34d89ce6097
child 17090 603f23d71ada
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     4     Copyright   2000 TUM
     4     Copyright   2000 TUM
     5 *)
     5 *)
     6 
     6 
     7 header {* \isaheader{The Typing Framework for the JVM}\label{sec:JVM} *}
     7 header {* \isaheader{The Typing Framework for the JVM}\label{sec:JVM} *}
     8 
     8 
     9 theory Typing_Framework_JVM = Typing_Framework_err + JVMType + EffectMono + BVSpec:
     9 theory Typing_Framework_JVM imports Typing_Framework_err JVMType EffectMono BVSpec begin
    10 
    10 
    11 
    11 
    12 constdefs
    12 constdefs
    13   exec :: "jvm_prog \<Rightarrow> nat \<Rightarrow> ty \<Rightarrow> exception_table \<Rightarrow> instr list \<Rightarrow> state step_type"
    13   exec :: "jvm_prog \<Rightarrow> nat \<Rightarrow> ty \<Rightarrow> exception_table \<Rightarrow> instr list \<Rightarrow> state step_type"
    14   "exec G maxs rT et bs == 
    14   "exec G maxs rT et bs ==