S2ss_prop.thy
author chunhan
Thu, 29 Aug 2013 10:01:24 +0800
changeset 33 6884b3c9284b
parent 32 705e1e41faf7
child 34 e7f850d1e08e
permissions -rw-r--r--
fix bug of static.thy for the static of recvmsg case

(*<*)
theory S2ss_prop
imports Main Flask Flask_type Static Static_type Init_prop Tainted_prop Valid_prop Alive_prop Co2sobj_prop
begin
(*>*)

context tainting_s begin

(* simpset for s2ss*)

lemma s2ss_execve:
  "valid (Execve p f fds # s) \<Longrightarrow> s2ss (Execve p f fds # s) = s2ss s "