doc-src/TutorialI/Advanced/WFrec.thy
changeset 11161 166f7d87b37f
parent 10885 90695f46440b
child 11196 bb4ede27fcb7
equal deleted inserted replaced
11160:e0ab13bec5c8 11161:166f7d87b37f
     1 (*<*)theory WFrec = Main:(*>*)
     1 (*<*)theory WFrec = Main:(*>*)
     2 
     2 
     3 text{*\noindent
     3 text{*\noindent
     4 So far, all recursive definitions where shown to terminate via measure
     4 So far, all recursive definitions were shown to terminate via measure
     5 functions. Sometimes this can be quite inconvenient or even
     5 functions. Sometimes this can be quite inconvenient or even
     6 impossible. Fortunately, \isacommand{recdef} supports much more
     6 impossible. Fortunately, \isacommand{recdef} supports much more
     7 general definitions. For example, termination of Ackermann's function
     7 general definitions. For example, termination of Ackermann's function
     8 can be shown by means of the \rmindex{lexicographic product} @{text"<*lex*>"}:
     8 can be shown by means of the \rmindex{lexicographic product} @{text"<*lex*>"}:
     9 *}
     9 *}