1
section \<open>Main HOL\<close>
2
3
text \<open>
4
Classical Higher-order Logic -- only ``Main'', excluding real and
5
complex numbers etc.
6
\<close>
7
8
theory Main
9
imports Pre_Main GCD Binomial
10
begin
11
12
end