doc-src/IsarImplementation/Thy/Syntax.thy
changeset 30124 b956bf0dc87c
child 30270 61811c9224a6
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/doc-src/IsarImplementation/Thy/Syntax.thy	Thu Feb 26 21:16:53 2009 +0100
@@ -0,0 +1,9 @@
+theory Syntax
+imports Base
+begin
+
+chapter {* Syntax and type-checking *}
+
+text FIXME
+
+end