src/HOL/Unix/Unix.thy
changeset 25706 45d090186bbe
parent 25592 e8ddaf6bf5df
child 25974 0cb35fa9c6fa
equal deleted inserted replaced
25705:45a2ffc5911e 25706:45d090186bbe
   364 
   364 
   365   chmod:
   365   chmod:
   366     "access root path uid {} = Some file \<Longrightarrow>
   366     "access root path uid {} = Some file \<Longrightarrow>
   367       uid = 0 \<or> uid = owner (attributes file) \<Longrightarrow>
   367       uid = 0 \<or> uid = owner (attributes file) \<Longrightarrow>
   368       root \<midarrow>(Chmod uid perms path)\<rightarrow> update path
   368       root \<midarrow>(Chmod uid perms path)\<rightarrow> update path
   369         (Some (map_attributes (others_update (K_record perms)) file)) root" |
   369         (Some (map_attributes (others_update (\<lambda>_. perms)) file)) root" |
   370 
   370 
   371   creat:
   371   creat:
   372     "path = parent_path @ [name] \<Longrightarrow>
   372     "path = parent_path @ [name] \<Longrightarrow>
   373       access root parent_path uid {Writable} = Some (Env att parent) \<Longrightarrow>
   373       access root parent_path uid {Writable} = Some (Env att parent) \<Longrightarrow>
   374       access root path uid {} = None \<Longrightarrow>
   374       access root path uid {} = None \<Longrightarrow>