Tainted_prop.thy
author chunhan
Tue, 04 Jun 2013 15:51:02 +0800
changeset 18 9b42765ce554
child 19 ced0fcfbcf8e
permissions -rw-r--r--
info_flow did NOT guarantee in current_procs

theory Tainted_prop 
imports Main Flask Flask_type Init_prop Current_files_prop Current_sockets_prop Delete_prop Proc_fd_of_file_prop
begin

context tainting begin

lemma tainted_in_current:
  "\<lbrakk>obj \<in> tainted s; valid s\<rbrakk> \<Longrightarrow> alive s obj"
apply (erule tainted.induct, auto dest:vt_grant_os simp:is_file_simps)




end

end