ProgTutorial/Recipes/USTypes.thy
author Christian Urban <urbanc@in.tum.de>
Tue, 17 Nov 2009 23:59:19 +0100
changeset 392 47e5b71c7f6c
parent 346 0fea8b7a14a1
child 565 cecd7a941885
permissions -rw-r--r--
modified the typ-pretty-printer and added parser exercise


theory USTypes
imports "../Appendix"
begin


section {* User Space Type-Systems (TBD) *}



end