src/HOL/MicroJava/JVM/JVMExec.thy
changeset 16417 9bc16273c2d4
parent 13056 4fd18d409fd7
child 28524 644b62cf678f
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     4     Copyright   1999 Technische Universitaet Muenchen
     4     Copyright   1999 Technische Universitaet Muenchen
     5 *)
     5 *)
     6 
     6 
     7 header {* \isaheader{Program Execution in the JVM} *}
     7 header {* \isaheader{Program Execution in the JVM} *}
     8 
     8 
     9 theory JVMExec = JVMExecInstr + JVMExceptions:
     9 theory JVMExec imports JVMExecInstr JVMExceptions begin
    10 
    10 
    11 
    11 
    12 consts
    12 consts
    13   exec :: "jvm_prog \<times> jvm_state => jvm_state option"
    13   exec :: "jvm_prog \<times> jvm_state => jvm_state option"
    14 
    14