CookBook/Appendix.thy
author Christian Urban <urbanc@in.tum.de>
Tue, 10 Mar 2009 13:20:46 +0000
changeset 164 3f617d7a2691
parent 162 3fb9f820a294
child 168 009ca4807baa
permissions -rw-r--r--
more work on simple_inductive


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