src/HOL/Main.thy
author huffman
Sun, 28 Aug 2011 20:56:49 -0700
changeset 44571 bd91b77c4cd6
parent 44324 d972b91ed09d
child 44860 56101fa00193
permissions -rw-r--r--
move class perfect_space into RealVector.thy; use not_open_singleton as perfect_space class axiom; generalize some lemmas to class perfect_space;

header {* Main HOL *}

theory Main
imports Plain Predicate_Compile Nitpick
begin

text {*
  Classical Higher-order Logic -- only ``Main'', excluding real and
  complex numbers etc.
*}

text {* See further \cite{Nipkow-et-al:2002:tutorial} *}

text {* Compatibility layer -- to be dropped *}

lemma Inf_bool_def:
  "Inf A \<longleftrightarrow> (\<forall>x\<in>A. x)"
  by (auto intro: bool_induct)

lemma Sup_bool_def:
  "Sup A \<longleftrightarrow> (\<exists>x\<in>A. x)"
  by auto

declare Complete_Lattice.Inf_bool_def [simp del]
declare Complete_Lattice.Sup_bool_def [simp del]

end