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