| author | wenzelm |
| Mon, 18 Oct 2010 21:37:26 +0100 | |
| changeset 39867 | a8363532cd4d |
| parent 39865 | a724b90f951e |
| child 39876 | 1ff9bce085bd |
| permissions | -rw-r--r-- |
| 30124 | 1 |
theory Syntax |
2 |
imports Base |
|
3 |
begin |
|
4 |
||
| 34924 | 5 |
chapter {* Concrete syntax and type-checking *}
|
| 30124 | 6 |
|
7 |
text FIXME |
|
| 30272 | 8 |
|
| 39852 | 9 |
|
| 39865 | 10 |
section {* Parsing and printing \label{sec:parse-print} *}
|
| 34924 | 11 |
|
12 |
text FIXME |
|
13 |
||
| 39852 | 14 |
|
| 34924 | 15 |
section {* Checking and unchecking \label{sec:term-check} *}
|
16 |
||
| 39852 | 17 |
text FIXME |
18 |
||
| 30124 | 19 |
end |