src/Doc/Tutorial/Datatype/unfoldnested.thy
author wenzelm
Wed, 29 Nov 2023 19:45:54 +0100
changeset 79081 9d6359b71264
parent 58860 fee7cfa69c50
permissions -rw-r--r--
more compact representation of theory_id -- via consecutive thread-local ids;

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