doc-src/TutorialI/Datatype/unfoldnested.thy
author Walther Neuper <neuper@ist.tugraz.at>
Thu, 12 Aug 2010 15:03:34 +0200
branchisac-from-Isabelle2009-2
changeset 37913 20e3616b2d9c
parent 16417 9bc16273c2d4
permissions -rw-r--r--
prepare reactivation of isac-update-Isa09-2
nipkow@8751
     1
(*<*)
haftmann@16417
     2
theory unfoldnested imports Main begin;
nipkow@8751
     3
(*>*)
nipkow@10971
     4
datatype ('v,'f)"term" = Var 'v | App 'f "('v,'f)term_list"
nipkow@10971
     5
and ('v,'f)term_list = Nil | Cons "('v,'f)term" "('v,'f)term_list"
nipkow@8751
     6
(*<*)
nipkow@8751
     7
end
nipkow@8751
     8
(*>*)