src/HOL/Unix/Unix.thy
changeset 36504 7cc639e20cb2
parent 25974 0cb35fa9c6fa
child 36862 952b2b102a0a
equal deleted inserted replaced
36503:bd4e2821482a 36504:7cc639e20cb2
   356 where
   356 where
   357 
   357 
   358   read:
   358   read:
   359     "access root path uid {Readable} = Some (Val (att, text)) \<Longrightarrow>
   359     "access root path uid {Readable} = Some (Val (att, text)) \<Longrightarrow>
   360       root \<midarrow>(Read uid text path)\<rightarrow> root" |
   360       root \<midarrow>(Read uid text path)\<rightarrow> root" |
   361   write:
   361   "write":
   362     "access root path uid {Writable} = Some (Val (att, text')) \<Longrightarrow>
   362     "access root path uid {Writable} = Some (Val (att, text')) \<Longrightarrow>
   363       root \<midarrow>(Write uid text path)\<rightarrow> update path (Some (Val (att, text))) root" |
   363       root \<midarrow>(Write uid text path)\<rightarrow> update path (Some (Val (att, text))) root" |
   364 
   364 
   365   chmod:
   365   chmod:
   366     "access root path uid {} = Some file \<Longrightarrow>
   366     "access root path uid {} = Some file \<Longrightarrow>
   434   using root''
   434   using root''
   435 proof cases
   435 proof cases
   436   case read
   436   case read
   437   with root' show ?thesis by cases auto
   437   with root' show ?thesis by cases auto
   438 next
   438 next
   439   case write
   439   case "write"
   440   with root' show ?thesis by cases auto
   440   with root' show ?thesis by cases auto
   441 next
   441 next
   442   case chmod
   442   case chmod
   443   with root' show ?thesis by cases auto
   443   with root' show ?thesis by cases auto
   444 next
   444 next