ProgTutorial/Recipes/USTypes.thy
author Christian Urban <urbanc@in.tum.de>
Tue, 04 Aug 2009 16:18:39 +0200
changeset 303 05e6a33edef6
parent 211 d5accbc67e1b
child 346 0fea8b7a14a1
permissions -rw-r--r--
added an antiquotation for printing the raw proof state; polished the example about proof state


theory USTypes
imports Main
begin


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



end