src/HOL/Plain.thy
author blanchet
Tue, 09 Aug 2011 09:33:50 +0200
changeset 44092 bf489e54d7f8
parent 41886 aa8dce9ab8a9
child 46691 72d81e789106
permissions -rw-r--r--
renamed E wrappers for consistency with CASC conventions

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