ProgTutorial/Appendix.thy
author Christian Urban <urbanc@in.tum.de>
Tue, 24 Mar 2009 09:34:03 +0100
changeset 206 096776f180fc
parent 189 069d525f8f1d
child 346 0fea8b7a14a1
permissions -rw-r--r--
added a keyword file, but needs to re-generated whenever something changes with keywords in Isabelle


theory Appendix
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 unification and typing algorithms 
  (@{ML_file "Pure/pattern.ML"} implements HOPU)

  \item useful datastructures: discrimination nets, association lists
  \end{itemize}
*}

end