src/HOL/Main.thy
author wenzelm
Sun, 23 Apr 2017 14:15:09 +0200
changeset 65553 006a274cdbc2
child 65813 bdd17b18e103
permissions -rw-r--r--
added missing file (amending f533820e7248);

section \<open>Main HOL\<close>

text \<open>
  Classical Higher-order Logic -- only ``Main'', excluding real and
  complex numbers etc.
\<close>

theory Main
imports Pre_Main GCD Binomial
begin

end