src/CTT/Main.thy
author wenzelm
Thu, 15 Feb 2001 17:18:54 +0100
changeset 11145 3e47692e3a3e
parent 10466 78168ca70469
child 16417 9bc16273c2d4
permissions -rw-r--r--
eliminate get_def;


(*theory Main includes everything*)

theory Main = CTT + Arith + Bool:

end