src/HOL/Main.thy
author haftmann
Fri, 12 May 2017 20:03:50 +0200
changeset 65813 bdd17b18e103
parent 65553 006a274cdbc2
child 65814 3039d4aa7143
permissions -rw-r--r--
relaxed theory dependencies

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
begin

end