1
header {* Plain HOL *}
2
3
theory Plain
4
imports Datatype Record FunDef Extraction
5
begin
6
7
text {*
8
Plain bootstrap of fundamental HOL tools and packages; does not
9
include @{text Hilbert_Choice}.
10
*}
11
12
ML {* path_add "~~/src/HOL/Library" *}
13
14
end