ProgTutorial/Recipes/USTypes.thy
author griff
Mon, 23 Mar 2009 12:13:21 +0100
changeset 196 840b49bfb1cf
parent 189 069d525f8f1d
child 211 d5accbc67e1b
permissions -rw-r--r--
fixed `str_of_thms' output in example + small changes


theory USTypes
imports Main
begin


section {* User Space Type-Systems *}



end