src/CTT/Main.thy
author ballarin
Tue, 29 Sep 2009 22:15:54 +0200
changeset 32804 ca430e6aee1c
parent 17441 5b5feca0344a
child 35762 af3ff2ba4c54
permissions -rw-r--r--
Propagation of mixins for interpretation; reactivated diagnostic command print_interps.


(* $Id$ *)

header {* Main includes everything *}

theory Main
imports CTT Arith Bool
begin
end