| author | chaieb |
| Mon, 09 Feb 2009 11:07:17 +0000 | |
| changeset 29835 | 62da280e5d0b |
| parent 29820 | 07f53494cf20 |
| child 29837 | eb7e62c0f53c |
| permissions | -rw-r--r-- |
| 27368 | 1 |
header {* Plain HOL *}
|
2 |
||
3 |
theory Plain |
|
|
29820
07f53494cf20
Rearrange Refute/SAT theory dependencies so as to use even more antiquotations in refute.ML +
blanchet
parents:
29609
diff
changeset
|
4 |
imports Datatype FunDef Record 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 |