ProgTutorial/Appendix.thy
author Christian Urban <christian dot urban at kcl dot ac dot uk>
Sat, 01 Dec 2012 16:50:46 +0000
changeset 540 d144fc51fe04
parent 517 d8c376662bb4
child 565 cecd7a941885
permissions -rw-r--r--
removed versions


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