Theory JVMCFG

Up to index of Isabelle/HOL/Jinja/Slicing

theory JVMCFG
imports BasicDefs BVExample
header {*
\isachapter{A Control Flow Graph for Jinja Byte Code}

This work was done by Denis Lohner (denis.lohner@kit.edu).

\isaheader{Formalizing the CFG}
*}


theory JVMCFG imports "../Basic/BasicDefs" "../../Jinja/BV/BVExample" begin


declare lesub_list_impl_same_size [simp del]
declare listE_length [simp del]

subsection {* Type definitions *}

subsubsection {* Wellformed Programs *}

definition "wf_jvmprog = {(P, Phi). wf_jvm_progPhi P}"

typedef wf_jvmprog = wf_jvmprog
proof
show "(E, Phi) ∈ wf_jvmprog"
unfolding wf_jvmprog_def by (auto intro: wf_prog)
qed

hide_const Phi E

abbreviation rep_jvmprog_jvm_prog :: "wf_jvmprog => jvm_prog"
("_wf")
where "Pwf ≡ fst(Rep_wf_jvmprog(P))"

abbreviation rep_jvmprog_phi :: "wf_jvmprog => tyP"
("_Φ")
where "PΦ ≡ snd(Rep_wf_jvmprog(P))"

lemma wf_jvmprog_is_wf: "wf_jvm_progPΦ (Pwf)"
using Rep_wf_jvmprog [of P]
by (auto simp: wf_jvmprog_def split_beta)

subsubsection {* Basic Types *}

text {*
We consider a program to be a well-formed Jinja program,
together with a given base class and a main method
*}


type_synonym jvmprog = "wf_jvmprog × cname × mname"
type_synonym callstack = "(cname × mname × pc) list"

text {*
The state is modeled as $\textrm{heap} \times \textrm{stack-variables} \times \textrm{local-variables}$

stack and local variables are modeled as pairs of natural numbers. The first number
gives the position in the call stack (i.e. the method in which the variable is used),
the second the position in the method's stack or array of local variables resp.

The stack variables are numbered from bottom up (which is the reverse order of the
array for the stack in Jinja's state representation), whereas local variables are identified
by their position in the array of local variables of Jinja's state representation.
*}


type_synonym state = "heap × ((nat × nat) => val) × ((nat × nat) => val)"


abbreviation heap_of :: "state => heap"
where
"heap_of s ≡ fst(s)"

abbreviation stk_of :: "state => ((nat × nat) => val)"
where
"stk_of s ≡ fst(snd(s))"

abbreviation loc_of :: "state => ((nat × nat) => val)"
where
"loc_of s ≡ snd(snd(s))"


subsection {* Basic Definitions *}

subsubsection {* State update (instruction execution) *}

text {*
This function models instruction execution for our state representation.

Additional parameters are the call depth of the current program point,
the stack length of the current program point,
the length of the stack in the underlying call frame (needed for {\sc Return}),
and (for {\sc Invoke}) the length of the array of local variables of the invoked method.

Exception handling is not covered by this function.
*}


fun exec_instr :: "instr => wf_jvmprog => state => nat => nat => nat => nat => state"
where
exec_instr_Load:
"exec_instr (Load n) P s calldepth stk_length rs ill =
(let (h,stk,loc) = s
in (h, stk((calldepth,stk_length):=loc(calldepth,n)), loc))"


| exec_instr_Store:
"exec_instr (Store n) P s calldepth stk_length rs ill =
(let (h,stk,loc) = s
in (h, stk, loc((calldepth,n):=stk(calldepth,stk_length - 1))))"


| exec_instr_Push:
"exec_instr (Push v) P s calldepth stk_length rs ill =
(let (h,stk,loc) = s
in (h, stk((calldepth,stk_length):=v), loc))"


| exec_instr_New:
"exec_instr (New C) P s calldepth stk_length rs ill =
(let (h,stk,loc) = s;
a = the(new_Addr h)
in (h(a \<mapsto> (blank (Pwf) C)), stk((calldepth,stk_length):=Addr a), loc))"


| exec_instr_Getfield:
"exec_instr (Getfield F C) P s calldepth stk_length rs ill =
(let (h,stk,loc) = s;
a = the_Addr (stk (calldepth,stk_length - 1));
(D,fs) = the(h a)
in (h, stk((calldepth,stk_length - 1) := the(fs(F,C))), loc))"


| exec_instr_Putfield:
"exec_instr (Putfield F C) P s calldepth stk_length rs ill =
(let (h,stk,loc) = s;
v = stk (calldepth,stk_length - 1);
a = the_Addr (stk (calldepth,stk_length - 2));
(D,fs) = the(h a)
in (h(a \<mapsto> (D,fs((F,C) \<mapsto> v))), stk, loc))"


| exec_instr_Checkcast:
"exec_instr (Checkcast C) P s calldepth stk_length rs ill = s"

| exec_instr_Pop:
"exec_instr (Pop) P s calldepth stk_length rs ill = s"

| exec_instr_IAdd:
"exec_instr (IAdd) P s calldepth stk_length rs ill =
(let (h,stk,loc) = s;
i1 = the_Intg (stk (calldepth, stk_length - 1));
i2 = the_Intg (stk (calldepth, stk_length - 2))
in (h, stk((calldepth, stk_length - 2) := Intg (i1 + i2)), loc))"


| exec_instr_IfFalse:
"exec_instr (IfFalse b) P s calldepth stk_length rs ill = s"

| exec_instr_CmpEq:
"exec_instr (CmpEq) P s calldepth stk_length rs ill =
(let (h,stk,loc) = s;
v1 = stk (calldepth, stk_length - 1);
v2 = stk (calldepth, stk_length - 2)
in (h, stk((calldepth, stk_length - 2) := Bool (v1 = v2)), loc))"


| exec_instr_Goto:
"exec_instr (Goto i) P s calldepth stk_length rs ill = s"

| exec_instr_Throw:
"exec_instr (Throw) P s calldepth stk_length rs ill = s"

| exec_instr_Invoke:
"exec_instr (Invoke M n) P s calldepth stk_length rs invoke_loc_length =
(let (h,stk,loc) = s;
loc' = (λ(a,b). if (a ≠ Suc calldepth ∨ b ≥ invoke_loc_length) then loc(a,b) else
(if (b ≤ n) then stk(calldepth, stk_length - (Suc n - b)) else arbitrary))
in (h,stk,loc'))"


| exec_instr_Return:
"exec_instr (Return) P s calldepth stk_length ret_stk_length ill =
(if (calldepth = 0)
then s
else
(let (h,stk,loc) = s;
v = stk(calldepth, stk_length - 1)
in (h,stk((calldepth - 1, ret_stk_length - 1) := v),loc))
)"



subsubsection {* length of stack and local variables *}

text {* The following terms extract the stack length at a given program point
from the well-typing of the given program *}


abbreviation stkLength :: "wf_jvmprog => cname => mname => pc => nat"
where
"stkLength P C M pc ≡ length (fst(the(((PΦ) C M)!pc)))"

abbreviation locLength :: "wf_jvmprog => cname => mname => pc => nat"
where
"locLength P C M pc ≡ length (snd(the(((PΦ) C M)!pc)))"


subsubsection {* Conversion functions *}

text {*
This function takes a natural number n and a function f with domain @{text nat}
and creates the array [f 0, f 1, f 2, ..., f (n - 1)].

This is used for extracting the array of local variables
*}


(*
fun locs :: "nat => (nat => 'a) => 'a list"
where
"locs 0 loc = []"
| "locs (Suc n) loc = (locs n loc)@[loc n]"
*)


abbreviation locs :: "nat => (nat => 'a) => 'a list"
where "locs n loc ≡ map loc [0..<n]"

text {*
This function takes a natural number n and a function f with domain @{text nat}
and creates the array [f (n - 1), ..., f 1, f 0].

This is used for extracting the stack as a list
*}


(*
fun stks :: "nat => (nat => 'a) => 'a list"
where
"stks 0 stk = []"
| "stks (Suc n) stk = (stk n)#(stks n stk)"
*)


abbreviation stks :: "nat => (nat => 'a) => 'a list"
where "stks n stk ≡ map stk (rev [0..<n])"

text {*
This function creates a list of the arrays for local variables from the given state
corresponding to the given callstack
*}


fun locss :: "wf_jvmprog => callstack => ((nat × nat) => 'a) => 'a list list"
where
"locss P [] loc = []"
| "locss P ((C,M,pc)#cs) loc =
(locs (locLength P C M pc) (λa. loc (length cs, a)))#(locss P cs loc)"


text {*
This function creates a list of the (methods') stacks from the given state
corresponding to the given callstack
*}


fun stkss :: "wf_jvmprog => callstack => ((nat × nat) => 'a) => 'a list list"
where
"stkss P [] stk = []"
| "stkss P ((C,M,pc)#cs) stk =
(stks (stkLength P C M pc) (λa. stk (length cs, a)))#(stkss P cs stk)"


text {* Given a callstack and a state, this abbreviation converts the state
to Jinja's state representation
*}


abbreviation state_to_jvm_state :: "wf_jvmprog => callstack => state => jvm_state"
where "state_to_jvm_state P cs s ≡
(None, heap_of s, zip (stkss P cs (stk_of s)) (zip (locss P cs (loc_of s)) cs))"


text {* This function extracts the call stack from a given frame stack (as it is given
by Jinja's state representation)
*}


definition framestack_to_callstack :: "frame list => callstack"
where "framestack_to_callstack frs ≡ map snd (map snd frs)"


subsubsection {* State Conformance *}

text {* Now we lift byte code verifier conformance to our state representation *}

definition bv_conform :: "wf_jvmprog => callstack => state => bool"
("_,_ \<turnstile>BV _ \<surd>")
where "P,cs \<turnstile>BV s \<surd> ≡ correct_state (Pwf) (PΦ) (state_to_jvm_state P cs s)"


subsubsection {* Statically determine catch-block *}

text {* This function is equivalent to Jinja's @{text "find_handler"} function *}
fun find_handler_for :: "wf_jvmprog => cname => callstack => callstack"
where
"find_handler_for P C [] = []"
| "find_handler_for P C (c#cs) = (let (C',M',pc') = c in
(case match_ex_table (Pwf) C pc' (ex_table_of (Pwf) C' M') of
None => find_handler_for P C cs
| Some pc_d => (C', M', fst pc_d)#cs))"



subsection {* Simplification lemmas *}

lemma find_handler_decr [simp]: "find_handler_for P Exc cs ≠ c#cs"
proof
assume "find_handler_for P Exc cs = c#cs"
hence "length cs < length (find_handler_for P Exc cs)" by simp
thus False by (induct cs, auto)
qed

(*
lemma locs_length [simp]: "length (locs n loc) = n"
by (induct n) auto

lemma stks_length [simp]: "length (stks n stk) = n"
by (induct n) auto
*)


lemma stkss_length [simp]: "length (stkss P cs stk) = length cs"
by (induct cs) auto

lemma locss_length [simp]: "length (locss P cs loc) = length cs"
by (induct cs) auto

(*
lemma nth_stks: "b < n ==> stks n stk ! b = stk(n - Suc b)"
by (auto simp: rev_nth)
proof (induct n arbitrary: b)
case (0 b)
thus ?case by simp
next
case (Suc n b)
thus ?case
by (auto simp: nth_Cons' less_Suc_eq)
qed
*)


lemma nth_stkss:
"[| a < length cs; b < length (stkss P cs stk ! (length cs - Suc a)) |]
==> stkss P cs stk ! (length cs - Suc a) !
(length (stkss P cs stk ! (length cs - Suc a)) - Suc b) = stk (a,b)"

proof (induct cs)
case Nil
thus ?case by (simp add: nth_Cons')
next
case (Cons aa cs)
thus ?case
by (cases aa, auto simp add: nth_Cons' rev_nth less_Suc_eq)
qed

(*
lemma nth_locs: "b < n ==> locs n loc ! b = loc b"
proof (induct n)
case 0
thus ?case by simp
next
case (Suc n)
thus ?case
by (auto simp: nth_append less_Suc_eq)
qed
*)


lemma nth_locss:
"[| a < length cs; b < length (locss P cs loc ! (length cs - Suc a)) |]
==> locss P cs loc ! (length cs - Suc a) ! b = loc (a,b)"

proof (induct cs)
case Nil
thus ?case by (simp add: nth_Cons')
next
case (Cons aa cs)
thus ?case
by (cases aa, auto simp: nth_Cons' (* nth_locs *) less_Suc_eq)
qed

lemma hd_stks [simp]: "n ≠ 0 ==> hd (stks n stk) = stk(n - 1)"
by (cases n, simp_all)

lemma hd_tl_stks: "n > 1 ==> hd (tl (stks n stk)) = stk(n - 2)"
by (cases n, auto)

(*
lemma stks_purge:
"d ≥ b ==> stks b (stk(d := e)) = stks b stk"
by (induct b, auto)

lemma stks_purge':
"d ≥ b ==> stks b (λx. if x = d then e else stk x) = stks b stk"
by (fold fun_upd_def, simp only: stks_purge)
*)


lemma stkss_purge:
"length cs ≤ a ==> stkss P cs (stk((a,b) := c)) = stkss P cs stk"
by (induct cs, auto (* simp: stks_purge *))

lemma stkss_purge':
"length cs ≤ a ==> stkss P cs (λs. if s = (a, b) then c else stk s) = stkss P cs stk"
by (fold fun_upd_def, simp only: stkss_purge)

(*
lemma locs_purge:
"d ≥ b ==> locs b (loc(d := e)) = locs b loc"
by (induct b, auto)

lemma locs_purge':
"d ≥ b ==> locs b (λb. if b = d then e else loc b) = locs b loc"
by (fold fun_upd_def, simp only: locs_purge)
*)


lemma locss_purge:
"length cs ≤ a ==> locss P cs (loc((a,b) := c)) = locss P cs loc"
by (induct cs, auto (*simp: locs_purge *))

lemma locss_purge':
"length cs ≤ a ==> locss P cs (λs. if s = (a, b) then c else loc s) = locss P cs loc"
by (fold fun_upd_def, simp only: locss_purge)

lemma locs_pullout [simp]:
"locs b (loc(n := e)) = locs b loc [n := e]"
proof (induct b)
case 0
thus ?case by simp
next
case (Suc b)
thus ?case
by (cases "n - b", auto simp: list_update_append not_less_eq less_Suc_eq)
qed

lemma locs_pullout' [simp]:
"locs b (λa. if a = n then e else loc (c, a)) = locs b (λa. loc (c, a)) [n := e]"
by (fold fun_upd_def) simp

lemma stks_pullout:
"n < b ==> stks b (stk(n := e)) = stks b stk [b - Suc n := e]"
proof (induct b)
case 0
thus ?case by simp
next
case (Suc b)
thus ?case
proof (cases "b = n")
case True
with Suc show ?thesis
by auto
(* by (auto simp: stks_purge') *)
next
case False
with Suc show ?thesis
by (cases "b - n") (auto intro!: nth_equalityI simp: nth_list_update)
qed
qed

lemma nth_tl : "xs ≠ [] ==> tl xs ! n = xs ! (Suc n)"
by (cases xs, simp_all)

lemma f2c_Nil [simp]: "framestack_to_callstack [] = []"
by (simp add: framestack_to_callstack_def)

lemma f2c_Cons [simp]:
"framestack_to_callstack ((stk,loc,C,M,pc)#frs) = (C,M,pc)#(framestack_to_callstack frs)"
by (simp add: framestack_to_callstack_def)

lemma f2c_length [simp]:
"length (framestack_to_callstack frs) = length frs"
by (simp add: framestack_to_callstack_def)

lemma f2c_s2jvm_id [simp]:
"framestack_to_callstack
(snd(snd(state_to_jvm_state P cs s))) =
cs"

by (cases s, simp add: framestack_to_callstack_def)

lemma f2c_s2jvm_id' [simp]:
"framestack_to_callstack
(zip (stkss P cs stk) (zip (locss P cs loc) cs)) = cs"

by (simp add: framestack_to_callstack_def)

lemma f2c_append [simp]:
"framestack_to_callstack (frs @ frs') =
(framestack_to_callstack frs) @ (framestack_to_callstack frs')"

by (simp add: framestack_to_callstack_def)


section {* CFG construction *}

subsection {* Datatypes *}

text {* Nodes are labeled with a callstack and an optional tuple (consisting of
a callstack and a flag).

The first callstack determines the current program point (i.e. the next statement
to execute). If the second parameter is not None, we are at an intermediate state,
where the target of the instruction is determined (the second callstack)
and the flag is set to whether an exception is thrown or not.
*}

datatype j_node =
Entry ("'('_Entry'_')")
| Node "callstack" "(callstack × bool) option" ("'('_ _,_ '_')")

text {* The empty callstack indicates the exit node *}

abbreviation j_node_Exit :: "j_node" ("'('_Exit'_')")
where "j_node_Exit ≡ (_ [],None _)"

text {* An edge is a triple, consisting of two nodes and the edge kind *}

type_synonym j_edge = "(j_node × state edge_kind × j_node)"


subsection {* CFG *}

text {*
The CFG is constructed by a case analysis on the instructions and
their different behavior in different states. E.g. the exceptional behavior of
{\sc New}, if there is no more space in the heap, vs. the normal behavior.

Note: The set of edges defined by this predicate is a first approximation to the
real set of edges in the CFG. We later (theory JVMInterpretation) add some well-formedness
requirements to the nodes.
*}


inductive JVM_CFG :: "jvmprog => j_node => state edge_kind => j_node => bool"
("_ \<turnstile> _ -_-> _")
where
JCFG_EntryExit:
"prog \<turnstile> (_Entry_) -(λs. False)\<surd>-> (_Exit_)"

| JCFG_EntryStart:
"prog = (P, C0, Main) ==> prog \<turnstile> (_Entry_) -(λs. True)\<surd>-> (_ [(C0, Main, 0)],None _)"

| JCFG_ReturnExit:
"[| prog = (P,C0,Main);
(instrs_of (Pwf) C M) ! pc = Return |]
==> prog \<turnstile> (_ [(C, M, pc)],None _) -\<Up>id-> (_Exit_)"


| JCFG_Straight_NoExc:
"[| prog = (P, C0, Main);
instrs_of (Pwf) C M ! pc ∈ {Load idx, Store idx, Push val, Pop, IAdd, CmpEq};
ek = \<Up>(λs. exec_instr ((instrs_of (Pwf) C M) ! pc) P s
(length cs) (stkLength P C M pc) arbitrary arbitrary) |]
==> prog \<turnstile> (_ (C, M, pc)#cs,None _) -ek-> (_ (C, M, Suc pc)#cs,None _)"


| JCFG_New_Normal_Pred:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (New Cl);
ek = (λ(h,stk,loc). new_Addr h ≠ None)\<surd>|]
==> prog \<turnstile> (_ (C, M, pc)#cs,None _) -ek-> (_ (C, M, pc)#cs,⌊((C, M, Suc pc)#cs,False)⌋ _)"


| JCFG_New_Normal_Update:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (New Cl);
ek = \<Up>(λs. exec_instr (New Cl) P s (length cs) (stkLength P C M pc) arbitrary arbitrary) |]
==> prog \<turnstile> (_ (C, M, pc)#cs,⌊((C, M, Suc pc)#cs, False)⌋ _) -ek-> (_ (C, M, Suc pc)#cs,None _)"


| JCFG_New_Exc_Pred:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (New Cl);
find_handler_for P OutOfMemory ((C, M, pc)#cs) = cs';
ek = (λ(h,stk,loc). new_Addr h = None)\<surd> |]
==> prog \<turnstile> (_ (C, M, pc)#cs,None _) -ek-> (_ (C, M, pc)#cs,⌊(cs',True)⌋ _)"


| JCFG_New_Exc_Update:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (New Cl);
find_handler_for P OutOfMemory ((C, M, pc)#cs) = (C', M', pc')#cs';
ek = \<Up>(λ(h,stk,loc).
(h,
stk((length cs',(stkLength P C' M' pc') - 1) := Addr (addr_of_sys_xcpt OutOfMemory)),
loc)
) |]
==> prog \<turnstile> (_ (C, M, pc)#cs,⌊((C', M', pc')#cs', True)⌋ _) -ek-> (_ (C', M', pc')#cs',None _)"


| JCFG_New_Exc_Exit:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (New Cl);
find_handler_for P OutOfMemory ((C, M, pc)#cs) = [] |]
==> prog \<turnstile> (_ (C, M, pc)#cs,⌊([], True)⌋ _) -\<Up>id-> (_Exit_)"


| JCFG_Getfield_Normal_Pred:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Getfield Fd Cl);
ek = (λ(h,stk,loc). stk(length cs, stkLength P C M pc - 1) ≠ Null)\<surd> |]
==> prog \<turnstile> (_ (C, M, pc)#cs,None _) -ek-> (_ (C, M, pc)#cs,⌊((C, M, Suc pc)#cs, False)⌋ _)"


| JCFG_Getfield_Normal_Update:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Getfield Fd Cl);
ek = \<Up>(λs. exec_instr (Getfield Fd Cl) P s (length cs) (stkLength P C M pc)
arbitrary arbitrary) |]
==> prog \<turnstile> (_ (C, M, pc)#cs,⌊((C, M, Suc pc)#cs, False)⌋ _) -ek-> (_ (C, M, Suc pc)#cs,None _)"


| JCFG_Getfield_Exc_Pred:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Getfield Fd Cl);
find_handler_for P NullPointer ((C, M, pc)#cs) = cs';
ek = (λ(h,stk,loc). stk(length cs, stkLength P C M pc - 1) = Null)\<surd> |]
==> prog \<turnstile> (_ (C, M, pc)#cs,None _) -ek-> (_ (C, M, pc)#cs,⌊(cs', True)⌋ _)"


| JCFG_Getfield_Exc_Update:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Getfield Fd Cl);
find_handler_for P NullPointer ((C, M, pc)#cs) = (C', M', pc')#cs';
ek = \<Up>(λ(h,stk,loc).
(h,
stk((length cs',(stkLength P C' M' pc') - 1) := Addr (addr_of_sys_xcpt NullPointer)),
loc)
) |]
==> prog \<turnstile> (_ (C, M, pc)#cs,⌊((C', M', pc')#cs', True)⌋ _) -ek-> (_ (C', M', pc')#cs',None _)"


| JCFG_Getfield_Exc_Exit:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Getfield Fd Cl);
find_handler_for P NullPointer ((C, M, pc)#cs) = [] |]
==> prog \<turnstile> (_ (C, M, pc)#cs,⌊([], True)⌋ _) -\<Up>id-> (_Exit_)"


| JCFG_Putfield_Normal_Pred:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Putfield Fd Cl);
ek = (λ(h,stk,loc). stk(length cs, stkLength P C M pc - 2) ≠ Null)\<surd> |]
==> prog \<turnstile> (_ (C, M, pc)#cs,None _) -ek-> (_ (C, M, pc)#cs,⌊((C, M, Suc pc)#cs, False)⌋ _)"


| JCFG_Putfield_Normal_Update:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Putfield Fd Cl);
ek = \<Up>(λs. exec_instr (Putfield Fd Cl) P s (length cs) (stkLength P C M pc)
arbitrary arbitrary) |]
==> prog \<turnstile> (_ (C, M, pc)#cs,⌊((C, M, Suc pc)#cs, False)⌋ _) -ek-> (_ (C, M, Suc pc)#cs,None _)"


| JCFG_Putfield_Exc_Pred:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Putfield Fd Cl);
find_handler_for P NullPointer ((C, M, pc)#cs) = cs';
ek = (λ(h,stk,loc). stk(length cs, stkLength P C M pc - 2) = Null)\<surd> |]
==> prog \<turnstile> (_ (C, M, pc)#cs,None _) -ek-> (_ (C, M, pc)#cs,⌊(cs', True)⌋ _)"


| JCFG_Putfield_Exc_Update:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Putfield Fd Cl);
find_handler_for P NullPointer ((C, M, pc)#cs) = (C', M', pc')#cs';
ek = \<Up>(λ(h,stk,loc).
(h,
stk((length cs',(stkLength P C' M' pc') - 1) := Addr (addr_of_sys_xcpt NullPointer)),
loc)
) |]
==> prog \<turnstile> (_ (C, M, pc)#cs,⌊((C', M', pc')#cs', True)⌋ _) -ek-> (_ (C', M', pc')#cs',None _)"


| JCFG_Putfield_Exc_Exit:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Putfield Fd Cl);
find_handler_for P NullPointer ((C, M, pc)#cs) = [] |]
==> prog \<turnstile> (_ (C, M, pc)#cs,⌊([], True)⌋ _) -\<Up>id-> (_Exit_)"


| JCFG_Checkcast_Normal_Pred:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Checkcast Cl);
ek = (λ(h,stk,loc). cast_ok (Pwf) Cl h (stk(length cs, stkLength P C M pc - Suc 0)))\<surd> |]
==> prog \<turnstile> (_ (C, M, pc)#cs,None _) -ek-> (_ (C, M, Suc pc)#cs,None _)"


| JCFG_Checkcast_Exc_Pred:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Checkcast Cl);
find_handler_for P ClassCast ((C, M, pc)#cs) = cs';
ek = (λ(h,stk,loc). ¬ cast_ok (Pwf) Cl h (stk(length cs, stkLength P C M pc - Suc 0)))\<surd> |]
==> prog \<turnstile> (_ (C, M, pc)#cs,None _) -ek-> (_ (C, M, pc)#cs,⌊(cs', True)⌋ _)"


| JCFG_Checkcast_Exc_Update:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Checkcast Cl);
find_handler_for P ClassCast ((C, M, pc)#cs) = (C', M', pc')#cs';
ek = \<Up>(λ(h,stk,loc).
(h,
stk((length cs',(stkLength P C' M' pc') - 1) := Addr (addr_of_sys_xcpt ClassCast)),
loc)
) |]
==> prog \<turnstile> (_ (C, M, pc)#cs,⌊((C', M', pc')#cs', True)⌋ _) -ek-> (_ (C', M', pc')#cs',None _)"


| JCFG_Checkcast_Exc_Exit:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Checkcast Cl);
find_handler_for P ClassCast ((C, M, pc)#cs) = [] |]
==> prog \<turnstile> (_ (C, M, pc)#cs,⌊([], True)⌋ _) -\<Up>id-> (_Exit_)"


| JCFG_Invoke_Normal_Pred:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Invoke M2 n);
cd = length cs;
stk_length = stkLength P C M pc;
ek = (λ(h,stk,loc).
stk(cd, stk_length - Suc n) ≠ Null ∧
fst(method (Pwf) (cname_of h (the_Addr(stk(cd, stk_length - Suc n)))) M2) = D
)\<surd> |]
==>
prog \<turnstile> (_ (C, M, pc)#cs,None _) -ek-> (_ (C, M, pc)#cs,⌊((D, M2, 0)#(C, M, pc)#cs, False)⌋ _)"


| JCFG_Invoke_Normal_Update:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Invoke M2 n);
stk_length = stkLength P C M pc;
loc_length = locLength P D M2 0;
ek = \<Up>(λs. exec_instr (Invoke M2 n) P s (length cs) stk_length arbitrary loc_length)
|]
==> prog \<turnstile> (_ (C, M, pc)#cs,⌊((D, M2, 0)#(C, M, pc)#cs, False)⌋ _) -ek->
(_ (D, M2, 0)#(C, M, pc)#cs,None _)"


| JCFG_Invoke_Exc_Pred:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Invoke m2 n);
find_handler_for P NullPointer ((C, M, pc)#cs) = cs';
ek = (λ(h,stk,loc). stk(length cs, stkLength P C M pc - Suc n) = Null)\<surd> |]
==> prog \<turnstile> (_ (C, M, pc)#cs,None _) -ek-> (_ (C, M, pc)#cs,⌊(cs', True)⌋ _)"


| JCFG_Invoke_Exc_Update:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Invoke M2 n);
find_handler_for P NullPointer ((C, M, pc)#cs) = (C', M', pc')#cs';
ek = \<Up>(λ(h,stk,loc).
(h,
stk((length cs',(stkLength P C' M' pc') - 1) := Addr (addr_of_sys_xcpt NullPointer)),
loc)
)
|]
==> prog \<turnstile> (_ (C, M, pc)#cs,⌊((C', M', pc')#cs', True)⌋ _) -ek-> (_ (C', M', pc')#cs',None _)"


| JCFG_Invoke_Exc_Exit:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (Invoke M2 n);
find_handler_for P NullPointer ((C, M, pc)#cs) = [] |]
==> prog \<turnstile> (_ (C, M, pc)#cs,⌊([], True)⌋ _) -\<Up>id-> (_Exit_)"


| JCFG_Return_Update:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = Return;
stk_length = stkLength P C M pc;
r_stk_length = stkLength P C' M' (Suc pc');
ek = \<Up>(λs. exec_instr Return P s (Suc (length cs)) stk_length r_stk_length arbitrary) |]
==> prog \<turnstile> (_ (C, M, pc)#(C', M', pc')#cs,None _) -ek-> (_ (C', M', Suc pc')#cs,None _)"


| JCFG_Goto_Update:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = Goto idx |]
==> prog \<turnstile> (_ (C, M, pc)#cs,None _) -\<Up>id-> (_ (C, M, nat (int pc + idx))#cs,None _)"


| JCFG_IfFalse_False:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (IfFalse b);
b ≠ 1;
ek = (λ(h,stk,loc). stk(length cs, stkLength P C M pc - 1) = Bool False)\<surd> |]
==> prog \<turnstile> (_ (C, M, pc)#cs,None _) -ek-> (_ (C, M, nat (int pc + b))#cs,None _)"


| JCFG_IfFalse_Next:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = (IfFalse b);
ek = (λ(h,stk,loc). stk(length cs, stkLength P C M pc - 1) ≠ Bool False ∨ b = 1)\<surd> |]
==> prog \<turnstile> (_ (C, M, pc)#cs,None _) -ek-> (_ (C, M, Suc pc)#cs,None _)"


| JCFG_Throw_Pred:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = Throw;
cd = length cs;
stk_length = stkLength P C M pc;
∃Exc. find_handler_for P Exc ((C, M, pc)#cs) = cs';
ek = (λ(h,stk,loc).
(stk(length cs, stkLength P C M pc - 1) = Null ∧
find_handler_for P NullPointer ((C, M, pc)#cs) = cs') ∨
(stk(length cs, stkLength P C M pc - 1) ≠ Null ∧
find_handler_for P (cname_of h (the_Addr(stk(cd, stk_length - 1)))) ((C, M, pc)#cs) = cs')
)\<surd> |]
==> prog \<turnstile> (_ (C, M, pc)#cs,None _) -ek-> (_ (C, M, pc)#cs,⌊(cs', True)⌋ _)"


| JCFG_Throw_Update:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = Throw;
ek = \<Up>(λ(h,stk,loc).
(h,
stk((length cs',(stkLength P C' M' pc') - 1) :=
if (stk(length cs, stkLength P C M pc - 1) = Null) then
Addr (addr_of_sys_xcpt NullPointer)
else (stk(length cs, stkLength P C M pc - 1))),
loc)
) |]
==> prog \<turnstile> (_ (C, M, pc)#cs,⌊((C', M', pc')#cs', True)⌋ _) -ek-> (_ (C', M', pc')#cs',None _)"


| JCFG_Throw_Exit:
"[| prog = (P, C0, Main);
(instrs_of (Pwf) C M) ! pc = Throw |]
==> prog \<turnstile> (_ (C, M, pc)#cs,⌊([],True)⌋ _) -\<Up>id-> (_Exit_)"



subsection {* CFG properties *}

lemma JVMCFG_Exit_no_sourcenode [dest]:
assumes edge:"prog \<turnstile> (_Exit_) -et-> n'"
shows "False"
proof -
{ fix n
have "[|prog \<turnstile> n -et-> n'; n = (_Exit_)|] ==> False"
by (auto elim!: JVM_CFG.cases)
}
with edge show ?thesis by fastforce
qed

lemma JVMCFG_Entry_no_targetnode [dest]:
assumes edge:"prog \<turnstile> n -et-> (_Entry_)"
shows "False"
proof -
{ fix n' have "[|prog \<turnstile> n -et-> n'; n' = (_Entry_)|] ==> False"
by (auto elim!: JVM_CFG.cases)
}
with edge show ?thesis by fastforce
qed

lemma JVMCFG_EntryD:
"[|(P,C,M) \<turnstile> n -et-> n'; n = (_Entry_)|]
==> (n' = (_Exit_) ∧ et = (λs. False)\<surd>) ∨ (n' = (_ [(C,M,0)],None _) ∧ et = (λs. True)\<surd>)"

by (erule JVM_CFG.cases) simp_all

declare split_def [simp add]
declare find_handler_for.simps [simp del]

(* The following lemma explores many cases, it takes a little to prove *)
lemma JVMCFG_edge_det:
"[|prog \<turnstile> n -et-> n'; prog \<turnstile> n -et'-> n'|] ==> et = et'"
by (erule JVM_CFG.cases, (erule JVM_CFG.cases, fastforce+)+)

declare split_def [simp del]
declare find_handler_for.simps [simp add]

end