replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)
header {* Plain HOL *}theory Plainimports Datatype Record FunDef Extractionbegintext {* Plain bootstrap of fundamental HOL tools and packages; does not include @{text Hilbert_Choice}.*}ML {* path_add "~~/src/HOL/Library" *}end