src/CTT/Main.thy
author wenzelm
Sun, 03 May 2015 17:36:46 +0200
changeset 60243 5901cb4db0ae
parent 58889 5b7a9633cfa8
child 60770 240563fbf41d
permissions -rw-r--r--
tuned output;

section {* Main includes everything *}

theory Main
imports CTT Arith Bool
begin
end