equal
deleted
inserted
replaced
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 *} |