Mercurial
Mercurial
>
repos
>
isabelle
/ file revision
summary
|
shortlog
|
changelog
|
graph
|
tags
|
bookmarks
|
branches
|
files
|
changeset
| file |
latest
|
revisions
|
annotate
|
diff
|
comparison
|
raw
|
help
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
doc-src/IsarImplementation/Thy/Syntax.thy
author
nipkow
Mon, 14 Sep 2009 19:30:48 +0200
changeset 32571
d4bb776874b8
parent 30272
2d612824e642
child 34924
520727474bbe
permissions
-rw-r--r--
count number of iterations required for minimization (and fixed bug: minimization was always called)
theory Syntax
imports Base
begin
chapter {* Syntax and type-checking *}
text FIXME
end