src/CTT/Main.thy
author wenzelm
Fri, 15 Jan 2016 19:50:37 +0100
changeset 62185 155d30f721dd
parent 60770 240563fbf41d
child 63505 42e1dece537a
permissions -rw-r--r--
misc updates and tuning; more on "Output" versus "Proof state";

section \<open>Main includes everything\<close>

theory Main
imports CTT Arith Bool
begin
end