src/HOL/MicroJava/JVM/JVMExecInstr.thy
changeset 16417 9bc16273c2d4
parent 13677 5fad004bd9df
child 28524 644b62cf678f
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     6 
     6 
     7 
     7 
     8 header {* \isaheader{JVM Instruction Semantics} *}
     8 header {* \isaheader{JVM Instruction Semantics} *}
     9 
     9 
    10 
    10 
    11 theory JVMExecInstr = JVMInstructions + JVMState:
    11 theory JVMExecInstr imports JVMInstructions JVMState begin
    12 
    12 
    13 
    13 
    14 consts
    14 consts
    15   exec_instr :: "[instr, jvm_prog, aheap, opstack, locvars, 
    15   exec_instr :: "[instr, jvm_prog, aheap, opstack, locvars, 
    16                   cname, sig, p_count, frame list] => jvm_state"
    16                   cname, sig, p_count, frame list] => jvm_state"