doc-src/IsarImplementation/Thy/Base.thy
author wenzelm
Thu, 26 Feb 2009 21:16:53 +0100
changeset 30124 b956bf0dc87c
parent 29755 d66b34e46bdf
child 30270 61811c9224a6
permissions -rw-r--r--
basic setup for chapter "Syntax and type-checking";

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

end