CookBook/Appendix.thy
author Christian Urban <urbanc@in.tum.de>
Wed, 11 Mar 2009 17:38:17 +0000
changeset 167 3e30ea95c7aa
parent 164 3f617d7a2691
child 168 009ca4807baa
permissions -rw-r--r--
added temporarily some timing test about conversions and simprocs


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

  useful datastructures:

  discrimination nets

  association lists
*}

end