doc-src/IsarImplementation/Thy/Syntax.thy
author wenzelm
Thu, 05 Mar 2009 02:20:06 +0100
changeset 30270 61811c9224a6
parent 30124 b956bf0dc87c
child 30272 2d612824e642
permissions -rw-r--r--
dummy changes to produce a new changeset of these files;

theory Syntax
imports Base
begin

chapter {* Syntax and type-checking *}

text FIXME
 
end