Theory Plain

Up to index of Isabelle/HOL

theory Plain
imports FunDef Extraction Metis
header {* Plain HOL *}

theory Plain
imports Datatype FunDef Extraction Metis
begin


text {*
Plain bootstrap of fundamental HOL tools and packages; does not
include @{text Hilbert_Choice}.
*}


end