ProgTutorial/Appendix.thy
author Christian Urban <urbanc@in.tum.de>
Mon, 30 Apr 2012 14:43:52 +0100
changeset 517 d8c376662bb4
parent 475 25371f74c768
child 565 cecd7a941885
permissions -rw-r--r--
removed special ML-setup and replaced it by explicit markups (i.e., %grayML)


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