doc-src/IsarImplementation/Thy/Base.thy
author wenzelm
Wed, 06 Apr 2011 22:25:44 +0200
changeset 42263 49b1b8d0782f
parent 40110 93e7935d4cb5
child 43564 9864182c6bad
permissions -rw-r--r--
type syntax as regular mixfix specification (type_ext for bootstrapping has been obsolete for many years);

theory Base
imports Main
uses "../../antiquote_setup.ML"
begin

end