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

theory Syntax
imports Base
begin

chapter {* Syntax and type-checking *}

text FIXME

end