CookBook/Appendix.thy
author Christian Urban <urbanc@in.tum.de>
Mon, 16 Mar 2009 00:12:32 +0100
changeset 178 fb8f22dd8ad0
parent 168 009ca4807baa
child 182 4d0e2edd476d
permissions -rw-r--r--
adapted to latest Attrib.setup changes and more work on the simple induct chapter


theory Appendix
imports Main
begin

text {* \appendix *}


chapter {* Recipes *}

text {*
  Possible further 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

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

end