simplified some internal flags using Config.T instead of full-blown Proof_Data;
header {* Plain HOL *}theory Plainimports Datatype FunDef Extractionbegintext {* Plain bootstrap of fundamental HOL tools and packages; does not include @{text Hilbert_Choice}.*}ML {* path_add "~~/src/HOL/Library" *}end