src/CTT/Main.thy
author wenzelm
Mon, 13 Mar 2017 15:25:25 +0100
changeset 65208 91c528cd376a
parent 64980 7dc25cf5793e
permissions -rw-r--r--
more robust Session.stop: idempotent, avoid conflict with startup;

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

theory Main
  imports CTT Bool Arith
begin
end