author | bulwahn |
Mon, 25 Jul 2011 11:21:45 +0200 | |
changeset 43960 | c2554cc82d34 |
parent 37358 | 74fb4f03bb51 |
child 58329 | a31404ec7414 |
permissions | -rw-r--r-- |
32635 | 1 |
(* Author: Christian Urban TU Muenchen *) |
19495 | 2 |
|
32635 | 3 |
header {* Various examples involving nominal datatypes. *} |
19495 | 4 |
|
32635 | 5 |
theory Nominal_Examples |
6 |
imports |
|
37358 | 7 |
CK_Machine |
32635 | 8 |
CR |
9 |
CR_Takahashi |
|
36277
9be4ab2acc13
split Class.thy into parts to conserve a bit of memory and increase the chance of making it work on Cygwin with only 2 GB available;
wenzelm
parents:
33189
diff
changeset
|
10 |
Class3 |
32635 | 11 |
Compile |
37358 | 12 |
Contexts |
13 |
Crary |
|
32635 | 14 |
Fsub |
15 |
Height |
|
16 |
Lambda_mu |
|
37358 | 17 |
LocalWeakening |
18 |
Pattern |
|
32635 | 19 |
SN |
20 |
SOS |
|
37358 | 21 |
Standardization |
32635 | 22 |
Support |
37358 | 23 |
Type_Preservation |
32635 | 24 |
W |
37358 | 25 |
Weakening |
32635 | 26 |
begin |
24895 | 27 |
|
32635 | 28 |
end |