ProgTutorial/Recipes/USTypes.thy
author Christian Urban <urbanc@in.tum.de>
Tue, 31 Mar 2009 20:31:18 +0100
changeset 218 7ff7325e3b4e
parent 211 d5accbc67e1b
child 346 0fea8b7a14a1
permissions -rw-r--r--
started to adapt the rest of chapter 5 to the simplified version without parameters (they will be described in the extension section)


theory USTypes
imports Main
begin


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



end