doc-src/TutorialI/Recdef/Nested0.thy
changeset 11494 23a118849801
parent 11196 bb4ede27fcb7
child 16417 9bc16273c2d4
equal deleted inserted replaced
11493:f3ff2549cdc8 11494:23a118849801
     1 (*<*)
     1 (*<*)
     2 theory Nested0 = Main:
     2 theory Nested0 = Main:
     3 (*>*)
     3 (*>*)
     4 
     4 
     5 text{*
     5 text{*
       
     6 \index{datatypes!nested}%
     6 In \S\ref{sec:nested-datatype} we defined the datatype of terms
     7 In \S\ref{sec:nested-datatype} we defined the datatype of terms
     7 *}
     8 *}
     8 
     9 
     9 datatype ('a,'b)"term" = Var 'a | App 'b "('a,'b)term list"
    10 datatype ('a,'b)"term" = Var 'a | App 'b "('a,'b)term list"
    10 
    11