equal
deleted
inserted
replaced
4 |
4 |
5 header {* Unix file-systems \label{sec:unix-file-system} *} |
5 header {* Unix file-systems \label{sec:unix-file-system} *} |
6 |
6 |
7 theory Unix |
7 theory Unix |
8 imports |
8 imports |
9 Main |
9 Nested_Environment |
10 "~~/src/HOL/Library/Nested_Environment" |
|
11 "~~/src/HOL/Library/List_Prefix" |
10 "~~/src/HOL/Library/List_Prefix" |
12 begin |
11 begin |
13 |
12 |
14 text {* |
13 text {* |
15 We give a simple mathematical model of the basic structures |
14 We give a simple mathematical model of the basic structures |