doc-src/TutorialI/Advanced/WFrec.thy
changeset 17914 99ead7a7eb42
parent 13111 2d6782e71702
child 20217 25b068a99d2b
equal deleted inserted replaced
17913:4159e1523ad8 17914:99ead7a7eb42
     1 (*<*)theory WFrec = Main:(*>*)
     1 (*<*)theory WFrec imports Main begin(*>*)
     2 
     2 
     3 text{*\noindent
     3 text{*\noindent
     4 So far, all recursive definitions were shown to terminate via measure
     4 So far, all recursive definitions were shown to terminate via measure
     5 functions. Sometimes this can be inconvenient or
     5 functions. Sometimes this can be inconvenient or
     6 impossible. Fortunately, \isacommand{recdef} supports much more
     6 impossible. Fortunately, \isacommand{recdef} supports much more