author | Christian Urban <urbanc@in.tum.de> |
Tue, 19 Jun 2012 05:17:46 +0100 | |
changeset 524 | 25f544b077f9 |
parent 517 | d8c376662bb4 |
child 565 | cecd7a941885 |
permissions | -rw-r--r-- |
theory Appendix imports Base begin text {* \appendix *} chapter {* Recipes *} text {* Possible topics: \begin{itemize} \item translations/print translations; @{ML "Proof_Context.print_syntax"} \item user space type systems (in the form that already exists) \item useful datastructures: discrimination nets, graphs, association lists \item Brief history of Isabelle \end{itemize} *} end