| author | blanchet |
| Tue, 26 Oct 2010 11:21:08 +0200 | |
| changeset 40159 | bfc716a96e47 |
| parent 40121 | e7a80c6752c9 |
| child 40178 | 00152d17855b |
| permissions | -rw-r--r-- |
| 27368 | 1 |
header {* Plain HOL *}
|
2 |
||
3 |
theory Plain |
|
| 40121 | 4 |
imports Datatype FunDef Extraction Sledgehammer |
| 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 |
||
| 27368 | 12 |
ML {* path_add "~~/src/HOL/Library" *}
|
13 |
||
14 |
end |