src/HOL/MicroJava/JVM/JVMInstructions.thy
changeset 13674 f4c64597fb02
parent 12911 704713ca07ea
child 13676 b1915d3e571d
equal deleted inserted replaced
13673:2950128b8206 13674:f4c64597fb02
    34   bytecode = "instr list"
    34   bytecode = "instr list"
    35   exception_entry = "p_count \<times> p_count \<times> p_count \<times> cname" 
    35   exception_entry = "p_count \<times> p_count \<times> p_count \<times> cname" 
    36                   -- "start-pc, end-pc, handler-pc, exception type"
    36                   -- "start-pc, end-pc, handler-pc, exception type"
    37   exception_table = "exception_entry list"
    37   exception_table = "exception_entry list"
    38   jvm_method = "nat \<times> nat \<times> bytecode \<times> exception_table"
    38   jvm_method = "nat \<times> nat \<times> bytecode \<times> exception_table"
       
    39              -- "max stacksize, length of local var array, \<dots>"
    39   jvm_prog = "jvm_method prog" 
    40   jvm_prog = "jvm_method prog" 
    40 
    41 
    41 end
    42 end