src/CTT/Main.thy
author krauss
Thu, 25 Aug 2011 14:06:34 +0200
changeset 44490 e3e8d20a6ebc
parent 35762 af3ff2ba4c54
child 58889 5b7a9633cfa8
permissions -rw-r--r--
lemma Compl_insert: "- insert x A = (-A) - {x}"

header {* Main includes everything *}

theory Main
imports CTT Arith Bool
begin
end