src/HOL/Main.thy
author wenzelm
Mon, 01 May 2017 13:03:56 +0200
changeset 65666 45d0692bb019
parent 65553 006a274cdbc2
child 65813 bdd17b18e103
permissions -rw-r--r--
incremental download of Jenkins log files, which are also added to database;

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