doc-src/TutorialI/Datatype/unfoldnested.thy
changeset 8751 9ed0548177fb
child 10971 6852682eaf16
equal deleted inserted replaced
8750:36b165788421 8751:9ed0548177fb
       
     1 (*<*)
       
     2 theory unfoldnested = Main:;
       
     3 (*>*)
       
     4 datatype ('a,'b)"term" = Var 'a | App 'b "('a,'b)term_list"
       
     5 and ('a,'b)term_list = Nil | Cons "('a,'b)term" "('a,'b)term_list"
       
     6 (*<*)
       
     7 end
       
     8 (*>*)