ProgTutorial/Recipes/USTypes.thy
author Christian Urban <christian dot urban at kcl dot ac dot uk>
Wed, 28 May 2014 12:41:09 +0100
changeset 556 3c214b215f7e
parent 346 0fea8b7a14a1
child 565 cecd7a941885
permissions -rw-r--r--
some small updates for Isabelle and corrections in the Parsing chapter


theory USTypes
imports "../Appendix"
begin


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



end