doc-src/TutorialI/Recdef/Nested1.thy
changeset 10186 499637e8f2c6
parent 10171 59d6633835fa
child 10242 028f54cd2cc9
equal deleted inserted replaced
10185:c452fea3ce74 10186:499637e8f2c6
     1 (*<*)
     1 (*<*)
     2 theory Nested1 = Nested0:;
     2 theory Nested1 = Nested0:;
     3 (*>*)
     3 (*>*)
     4 consts trev  :: "('a,'b)term \<Rightarrow> ('a,'b)term";
       
     5 
     4 
     6 text{*\noindent
     5 text{*\noindent
     7 Although the definition of @{term trev} is quite natural, we will have
     6 Although the definition of @{term trev} is quite natural, we will have
     8 overcome a minor difficulty in convincing Isabelle of is termination.
     7 overcome a minor difficulty in convincing Isabelle of is termination.
     9 It is precisely this difficulty that is the \textit{raison d'\^etre} of
     8 It is precisely this difficulty that is the \textit{raison d'\^etre} of