src/CTT/Main.thy
author blanchet
Fri, 26 Feb 2010 18:38:23 +0100
changeset 35388 42d39948cace
parent 17441 5b5feca0344a
child 35762 af3ff2ba4c54
permissions -rw-r--r--
use SAT4J for "Tests_Nits.thy" for safety (this should solve the Isatest failures) + minor changes


(* $Id$ *)

header {* Main includes everything *}

theory Main
imports CTT Arith Bool
begin
end