src/CTT/Main.thy
author wenzelm
Sun, 22 May 2005 16:51:13 +0200
changeset 16025 fa2d7364d359
parent 10466 78168ca70469
child 16417 9bc16273c2d4
permissions -rw-r--r--
added find_theorems.ML, ../simplifier.ML;


(*theory Main includes everything*)

theory Main = CTT + Arith + Bool:

end