CookBook/Appendix.thy
author Christian Urban <urbanc@in.tum.de>
Fri, 06 Mar 2009 21:52:17 +0000
changeset 162 3fb9f820a294
parent 131 8db9195bb3e9
child 164 3f617d7a2691
permissions -rw-r--r--
some additions to the simplifier section and general tuning


theory Appendix
imports Main
begin

text {* \appendix *}


chapter {* Recipes *}

text {*
  Possible further topics: 

  translations/print translations

  @{ML "ProofContext.print_syntax"}
  
  user space type systems (in the form that already exists)

  unification and typing algorithms
*}

end