doc-src/TutorialI/Datatype/unfoldnested.thy
changeset 8751 9ed0548177fb
child 10971 6852682eaf16
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/doc-src/TutorialI/Datatype/unfoldnested.thy	Wed Apr 19 13:40:42 2000 +0200
@@ -0,0 +1,8 @@
+(*<*)
+theory unfoldnested = Main:;
+(*>*)
+datatype ('a,'b)"term" = Var 'a | App 'b "('a,'b)term_list"
+and ('a,'b)term_list = Nil | Cons "('a,'b)term" "('a,'b)term_list"
+(*<*)
+end
+(*>*)