src/CTT/Main.thy
author wenzelm
Wed, 28 Apr 2010 16:11:13 +0200
changeset 36457 7355af2a7e8a
parent 35762 af3ff2ba4c54
child 58889 5b7a9633cfa8
permissions -rw-r--r--
tuned user-level type abbrevs: explicit warning concerning ignored sort constraints -- sorts never affect formation of types and type abbrevs strip sorts internally;

header {* Main includes everything *}

theory Main
imports CTT Arith Bool
begin
end