src/HOL/Unix/Unix.thy
changeset 58310 91ea607a34d8
parent 58249 180f1b3508ed
child 58613 4a16f8e41879
equal deleted inserted replaced
58309:a09ec6daaa19 58310:91ea607a34d8
    71   is member of a single global group.\footnote{A general HOL model of
    71   is member of a single global group.\footnote{A general HOL model of
    72   user group structures and related issues is given in
    72   user group structures and related issues is given in
    73   \cite{Naraschewski:2001}.}
    73   \cite{Naraschewski:2001}.}
    74 *}
    74 *}
    75 
    75 
    76 datatype_new perm =
    76 datatype perm =
    77     Readable
    77     Readable
    78   | Writable
    78   | Writable
    79   | Executable    -- "(ignored)"
    79   | Executable    -- "(ignored)"
    80 
    80 
    81 type_synonym perms = "perm set"
    81 type_synonym perms = "perm set"
   282   operation} for the syntax of system-calls, together with an
   282   operation} for the syntax of system-calls, together with an
   283   inductive definition of file-system state transitions of the form
   283   inductive definition of file-system state transitions of the form
   284   @{text "root \<midarrow>x\<rightarrow> root'"} for the operational semantics.
   284   @{text "root \<midarrow>x\<rightarrow> root'"} for the operational semantics.
   285 *}
   285 *}
   286 
   286 
   287 datatype_new operation =
   287 datatype operation =
   288     Read uid string path
   288     Read uid string path
   289   | Write uid string path
   289   | Write uid string path
   290   | Chmod uid perms path
   290   | Chmod uid perms path
   291   | Creat uid perms path
   291   | Creat uid perms path
   292   | Unlink uid path
   292   | Unlink uid path