ProgTutorial/Recipes/USTypes.thy
author griff
Tue, 21 Jul 2009 11:53:41 +0200
changeset 267 83abec907072
parent 211 d5accbc67e1b
child 346 0fea8b7a14a1
permissions -rw-r--r--
if n would be 0, rev_sum would be missing an argument


theory USTypes
imports Main
begin


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



end