doc-src/TutorialI/Datatype/unfoldnested.thy
changeset 48985 5386df44a037
parent 48984 f51d4a302962
child 48986 037d32448e29
--- a/doc-src/TutorialI/Datatype/unfoldnested.thy	Tue Aug 28 18:46:15 2012 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,8 +0,0 @@
-(*<*)
-theory unfoldnested imports Main begin;
-(*>*)
-datatype ('v,'f)"term" = Var 'v | App 'f "('v,'f)term_list"
-and ('v,'f)term_list = Nil | Cons "('v,'f)term" "('v,'f)term_list"
-(*<*)
-end
-(*>*)