Theory JVMInstructions

Up to index of Isabelle/HOL/Jinja

theory JVMInstructions
imports JVMState
(*  Title:      HOL/MicroJava/JVM/JVMInstructions.thy

Author: Gerwin Klein
Copyright 2000 Technische Universitaet Muenchen
*)


header {* \isaheader{Instructions of the JVM} *}


theory JVMInstructions imports JVMState begin


datatype
instr = Load nat -- "load from local variable"
| Store nat -- "store into local variable"
| Push val -- "push a value (constant)"
| New cname -- "create object"
| Getfield vname cname -- "Fetch field from object"
| Putfield vname cname -- "Set field in object "
| Checkcast cname -- "Check whether object is of given type"
| Invoke mname nat -- "inv. instance meth of an object"
| Return -- "return from method"
| Pop -- "pop top element from opstack"
| IAdd -- "integer addition"
| Goto int -- "goto relative address"
| CmpEq -- "equality comparison"
| IfFalse int -- "branch if top of stack false"
| Throw -- "throw top of stack as exception"

type_synonym
bytecode = "instr list"

type_synonym
ex_entry = "pc × pc × cname × pc × nat"
-- "start-pc, end-pc, exception type, handler-pc, remaining stack depth"

type_synonym
ex_table = "ex_entry list"

type_synonym
jvm_method = "nat × nat × bytecode × ex_table"
-- "max stacksize"
-- "number of local variables. Add 1 + no. of parameters to get no. of registers"
-- "instruction sequence"
-- "exception handler table"

type_synonym
jvm_prog = "jvm_method prog"

end