Theory JVMControlDependences

Up to index of Isabelle/HOL/Jinja/Slicing

theory JVMControlDependences
imports JVMPostdomination JVMCFG_wf DynPDG CDepInstantiations
header {* \isaheader{Instantiating the control dependences} *}

theory JVMControlDependences imports
JVMPostdomination
JVMCFG_wf
"../Dynamic/DynPDG"
"../StaticIntra/CDepInstantiations"
begin

subsection {* Dynamic dependences *}

interpretation JVMDynStandardControlDependence:
DynStandardControlDependencePDG "sourcenode" "targetnode" "kind"
"valid_edgeCFG prog" "(_Entry_)" "Def (fstCFG prog)" "Use (fstCFG prog)"
"state_val" "(_Exit_)" ..

interpretation JVMDynWeakControlDependence:
DynWeakControlDependencePDG "sourcenode" "targetnode" "kind"
"valid_edgeCFG prog" "(_Entry_)" "Def (fstCFG prog)" "Use (fstCFG prog)"
"state_val" "(_Exit_)" ..

subsection {* Static dependences *}

interpretation JVMStandardControlDependence:
StandardControlDependencePDG "sourcenode" "targetnode" "kind"
"valid_edgeCFG prog" "(_Entry_)" "Def (fstCFG prog)" "Use (fstCFG prog)"
"state_val" "(_Exit_)" ..

interpretation JVMWeakControlDependence:
WeakControlDependencePDG "sourcenode" "targetnode" "kind"
"valid_edgeCFG prog" "(_Entry_)" "Def (fstCFG prog)" "Use (fstCFG prog)"
"state_val" "(_Exit_)" ..

end