src/CTT/Main.thy
author blanchet
Thu, 14 Apr 2011 11:24:05 +0200
changeset 42353 7797efa897a1
parent 35762 af3ff2ba4c54
child 58889 5b7a9633cfa8
permissions -rw-r--r--
correctly handle TFrees that occur in (local) facts -- Metis did the right thing here but Sledgehammer was incorrectly generating spurious preconditions such as "dense_linorder(t_a)"

header {* Main includes everything *}

theory Main
imports CTT Arith Bool
begin
end