Tainted_prop.thy
changeset 34 e7f850d1e08e
parent 31 aa1375b6c0eb
child 43 137358bd4921
equal deleted inserted replaced
33:6884b3c9284b 34:e7f850d1e08e
     1 theory Tainted_prop 
     1 theory Tainted_prop 
     2 imports Main Flask Flask_type Init_prop Current_files_prop Current_sockets_prop Delete_prop Proc_fd_of_file_prop Current_prop Alive_prop
     2 imports Main Flask Flask_type Init_prop Current_files_prop Current_sockets_prop Delete_prop Proc_fd_of_file_prop Current_prop Alive_prop
     3 begin
     3 begin
       
     4 
       
     5 ML {*quick_and_dirty := true*}
     4 
     6 
     5 context tainting begin
     7 context tainting begin
     6 
     8 
     7 fun Tainted :: "t_state \<Rightarrow> t_object set"
     9 fun Tainted :: "t_state \<Rightarrow> t_object set"
     8 where
    10 where