author | Christian Urban <urbanc@in.tum.de> |
Fri, 01 Jan 2010 00:19:11 +0100 | |
changeset 413 | 95461cf6fd07 |
parent 407 | aee4abd02db1 |
child 475 | 25371f74c768 |
permissions | -rw-r--r-- |
theory Appendix imports Base begin (*<*) setup{* open_file_with_prelude "Recipes_Code.thy" ["theory Recipes", "imports Main", "begin"] *} (*>*) text {* \appendix *} chapter {* Recipes *} text {* Possible topics: \begin{itemize} \item translations/print translations; @{ML "ProofContext.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