diff -r 1e31ddcab458 -r 4c275405faae src/HOL/Unix/Unix.thy --- a/src/HOL/Unix/Unix.thy Sun Jan 15 16:28:03 2023 +0100 +++ b/src/HOL/Unix/Unix.thy Sun Jan 15 18:30:18 2023 +0100 @@ -67,7 +67,7 @@ simplification as we just do not intend to discuss a model of multiple groups and group membership, but pretend that everyone is member of a single global group.\<^footnote>\A general HOL model of user group structures and related - issues is given in @{cite "Naraschewski:2001"}.\ + issues is given in \<^cite>\"Naraschewski:2001"\.\ \ datatype perm = @@ -104,7 +104,7 @@ text \ In order to model the general tree structure of a Unix file-system we use the arbitrarily branching datatype \<^typ>\('a, 'b, 'c) env\ from the - standard library of Isabelle/HOL @{cite "Bauer-et-al:2002:HOL-Library"}. + standard library of Isabelle/HOL \<^cite>\"Bauer-et-al:2002:HOL-Library"\. This type provides constructors \<^term>\Val\ and \<^term>\Env\ as follows: \<^medskip> @@ -142,15 +142,14 @@ @{thm [display, indent = 2, eta_contract = false] lookup_eq [no_vars]} @{thm [display, indent = 2, eta_contract = false] update_eq [no_vars]} - Several further properties of these operations are proven in @{cite - "Bauer-et-al:2002:HOL-Library"}. These will be routinely used later on + Several further properties of these operations are proven in \<^cite>\"Bauer-et-al:2002:HOL-Library"\. These will be routinely used later on without further notice. \<^bigskip> Apparently, the elements of type \<^typ>\file\ contain an \<^typ>\att\ component in either case. We now define a few auxiliary operations to manipulate this field uniformly, following the conventions for record types - in Isabelle/HOL @{cite "Nipkow-et-al:2000:HOL"}. + in Isabelle/HOL \<^cite>\"Nipkow-et-al:2000:HOL"\. \ definition @@ -208,8 +207,7 @@ access was granted according to the permissions recorded within the file-system. - Note that by the rules of Unix file-system security (e.g.\ @{cite - "Tanenbaum:1992"}) both the super-user and owner may always access a file + Note that by the rules of Unix file-system security (e.g.\ \<^cite>\"Tanenbaum:1992"\) both the super-user and owner may always access a file unconditionally (in our simplified model). \ @@ -264,8 +262,7 @@ subsection \Unix system calls \label{sec:unix-syscall}\ text \ - According to established operating system design (cf.\ @{cite - "Tanenbaum:1992"}) user space processes may only initiate system operations + According to established operating system design (cf.\ \<^cite>\"Tanenbaum:1992"\) user space processes may only initiate system operations by a fixed set of \<^emph>\system-calls\. This enables the kernel to enforce certain security policies in the first place.\<^footnote>\Incidently, this is the very same principle employed by any ``LCF-style'' theorem proving system @@ -388,7 +385,7 @@ If in doubt, one may consider to compare our definition with the informal specifications given the corresponding Unix man pages, or even peek at an - actual implementation such as @{cite "Torvalds-et-al:Linux"}. Another common + actual implementation such as \<^cite>\"Torvalds-et-al:Linux"\. Another common way to gain confidence into the formal model is to run simple simulations (see \secref{sec:unix-examples}), and check the results with that of experiments performed on a real Unix system.