doc-src/TutorialI/Datatype/unfoldnested.thy
author blanchet
Mon, 19 Apr 2010 11:54:07 +0200
changeset 36222 0e3e49bd658d
parent 16417 9bc16273c2d4
permissions -rw-r--r--
don't use readable names if proof reconstruction is needed, because it uses the structure of names

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