ProgTutorial/Appendix.thy
author Christian Urban <urbanc@in.tum.de>
Thu, 23 May 2019 00:56:39 +0100
changeset 576 b78c4fab81a9
parent 569 f875a25aa72d
permissions -rw-r--r--
small typo


theory Appendix
imports Base
begin

text \<open>\appendix\<close>


chapter \<open>Recipes\<close>

text \<open>
  Possible topics: 

  \begin{itemize}
  \item translations/print translations; 
  @{ML \<open>Proof_Context.print_syntax\<close>}
  
  \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}
\<close>

end