ProgTutorial/Appendix.thy
author Christian Urban <urbanc@in.tum.de>
Fri, 20 Nov 2009 03:03:04 +0100
changeset 398 7f7080ce7c2b
parent 356 43df2d59fb98
child 407 aee4abd02db1
permissions -rw-r--r--
started something about sorts


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

  \item useful datastructures: discrimination nets, association lists

  \item Brief history of Isabelle
  \end{itemize}
*}

end