CookBook/Recipes/USTypes.thy
author Christian Urban <urbanc@in.tum.de>
Wed, 18 Mar 2009 18:27:48 +0100
changeset 186 371e4375c994
parent 127 74846cb0fff9
permissions -rw-r--r--
made the Ackermann function example safer and included suggestions from MW


theory USTypes
imports Main
begin


section {* User Space Type-Systems *}



end