doc-src/TutorialI/Datatype/unfoldnested.thy
author wenzelm
Sun, 15 Oct 2000 19:50:35 +0200
changeset 10220 2a726de6e124
parent 8751 9ed0548177fb
child 10971 6852682eaf16
permissions -rw-r--r--
proper symbol markup with \isamath, \isatext; support sub/super scripts:

(*<*)
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
(*>*)