author | haftmann |
Wed, 21 Jan 2009 23:40:23 +0100 | |
changeset 29609 | a010aab5bed0 |
parent 29304 | 5c71a6da989d |
child 29820 | 07f53494cf20 |
permissions | -rw-r--r-- |
27368 | 1 |
header {* Plain HOL *} |
2 |
||
3 |
theory Plain |
|
29609 | 4 |
imports Datatype FunDef Record SAT Extraction Divides |
27368 | 5 |
begin |
6 |
||
29304 | 7 |
text {* |
8 |
Plain bootstrap of fundamental HOL tools and packages; does not |
|
9 |
include @{text Hilbert_Choice}. |
|
10 |
*} |
|
11 |
||
29609 | 12 |
instance option :: (finite) finite |
13 |
by default (simp add: insert_None_conv_UNIV [symmetric]) |
|
14 |
||
27368 | 15 |
ML {* path_add "~~/src/HOL/Library" *} |
16 |
||
17 |
end |