src/HOL/Unix/Unix.thy
changeset 25592 e8ddaf6bf5df
parent 23769 7bc32680a495
child 25706 45d090186bbe
equal deleted inserted replaced
25591:0792e02973cc 25592:e8ddaf6bf5df
     4 *)
     4 *)
     5 
     5 
     6 header {* Unix file-systems \label{sec:unix-file-system} *}
     6 header {* Unix file-systems \label{sec:unix-file-system} *}
     7 
     7 
     8 theory Unix
     8 theory Unix
     9 imports Nested_Environment List_Prefix
     9 imports Main Nested_Environment List_Prefix
    10 begin
    10 begin
    11 
    11 
    12 text {*
    12 text {*
    13   We give a simple mathematical model of the basic structures
    13   We give a simple mathematical model of the basic structures
    14   underlying the Unix file-system, together with a few fundamental
    14   underlying the Unix file-system, together with a few fundamental