get rid of all "optimizations" regarding "unit" and other cardinality-1 types
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