doc-src/TutorialI/Advanced/WFrec.thy
author nipkow
Mon, 06 Nov 2000 11:32:23 +0100
changeset 10396 5ab08609e6c8
parent 10241 e0428c2778f1
child 10522 ed3964d1f1a4
permissions -rw-r--r--
*** empty log message ***
nipkow@10187
     1
(*<*)theory WFrec = Main:(*>*)
nipkow@10187
     2
nipkow@10187
     3
text{*\noindent
nipkow@10187
     4
So far, all recursive definitions where shown to terminate via measure
nipkow@10187
     5
functions. Sometimes this can be quite inconvenient or even
nipkow@10187
     6
impossible. Fortunately, \isacommand{recdef} supports much more
nipkow@10187
     7
general definitions. For example, termination of Ackermann's function
nipkow@10187
     8
can be shown by means of the lexicographic product @{text"<*lex*>"}:
nipkow@10187
     9
*}
nipkow@10187
    10
nipkow@10187
    11
consts ack :: "nat\<times>nat \<Rightarrow> nat";
nipkow@10187
    12
recdef ack "measure(\<lambda>m. m) <*lex*> measure(\<lambda>n. n)"
nipkow@10187
    13
  "ack(0,n)         = Suc n"
nipkow@10187
    14
  "ack(Suc m,0)     = ack(m, 1)"
nipkow@10187
    15
  "ack(Suc m,Suc n) = ack(m,ack(Suc m,n))";
nipkow@10187
    16
nipkow@10187
    17
text{*\noindent
nipkow@10187
    18
The lexicographic product decreases if either its first component
nipkow@10187
    19
decreases (as in the second equation and in the outer call in the
nipkow@10187
    20
third equation) or its first component stays the same and the second
nipkow@10187
    21
component decreases (as in the inner call in the third equation).
nipkow@10187
    22
nipkow@10187
    23
In general, \isacommand{recdef} supports termination proofs based on
nipkow@10396
    24
arbitrary well-founded relations as introduced in \S\ref{sec:Well-founded}.
nipkow@10396
    25
This is called \textbf{well-founded
paulson@10241
    26
recursion}\indexbold{recursion!well-founded}\index{well-founded
nipkow@10396
    27
recursion|see{recursion, well-founded}}. Clearly, a function definition is
nipkow@10396
    28
total iff the set of all pairs $(r,l)$, where $l$ is the argument on the
nipkow@10396
    29
left-hand side of an equation and $r$ the argument of some recursive call on
nipkow@10396
    30
the corresponding right-hand side, induces a well-founded relation.  For a
nipkow@10396
    31
systematic account of termination proofs via well-founded relations see, for
nipkow@10396
    32
example, \cite{Baader-Nipkow}.
nipkow@10187
    33
nipkow@10396
    34
Each \isacommand{recdef} definition should be accompanied (after the name of
nipkow@10396
    35
the function) by a well-founded relation on the argument type of the
nipkow@10396
    36
function.  The HOL library formalizes some of the most important
nipkow@10396
    37
constructions of well-founded relations (see \S\ref{sec:Well-founded}). For
nipkow@10396
    38
example, @{term"measure f"} is always well-founded, and the lexicographic
nipkow@10396
    39
product of two well-founded relations is again well-founded, which we relied
nipkow@10396
    40
on when defining Ackermann's function above.
nipkow@10396
    41
Of course the lexicographic product can also be interated:
nipkow@10189
    42
*}
nipkow@10187
    43
nipkow@10189
    44
consts contrived :: "nat \<times> nat \<times> nat \<Rightarrow> nat"
nipkow@10189
    45
recdef contrived
nipkow@10189
    46
  "measure(\<lambda>i. i) <*lex*> measure(\<lambda>j. j) <*lex*> measure(\<lambda>k. k)"
nipkow@10189
    47
"contrived(i,j,Suc k) = contrived(i,j,k)"
nipkow@10189
    48
"contrived(i,Suc j,0) = contrived(i,j,j)"
nipkow@10189
    49
"contrived(Suc i,0,0) = contrived(i,i,i)"
nipkow@10189
    50
"contrived(0,0,0)     = 0"
nipkow@10189
    51
nipkow@10189
    52
text{*
nipkow@10396
    53
Lexicographic products of measure functions already go a long
nipkow@10396
    54
way. Furthermore you may embedding some type in an
nipkow@10396
    55
existing well-founded relation via the inverse image construction @{term
nipkow@10396
    56
inv_image}. All these constructions are known to \isacommand{recdef}. Thus you
paulson@10241
    57
will never have to prove well-foundedness of any relation composed
nipkow@10189
    58
solely of these building blocks. But of course the proof of
nipkow@10189
    59
termination of your function definition, i.e.\ that the arguments
nipkow@10189
    60
decrease with every recursive call, may still require you to provide
nipkow@10189
    61
additional lemmas.
nipkow@10189
    62
paulson@10241
    63
It is also possible to use your own well-founded relations with \isacommand{recdef}.
nipkow@10189
    64
Here is a simplistic example:
nipkow@10187
    65
*}
nipkow@10189
    66
nipkow@10189
    67
consts f :: "nat \<Rightarrow> nat"
nipkow@10189
    68
recdef f "id(less_than)"
nipkow@10189
    69
"f 0 = 0"
nipkow@10189
    70
"f (Suc n) = f n"
nipkow@10189
    71
nipkow@10396
    72
text{*\noindent
nipkow@10189
    73
Since \isacommand{recdef} is not prepared for @{term id}, the identity
nipkow@10189
    74
function, this leads to the complaint that it could not prove
nipkow@10396
    75
@{prop"wf (id less_than)"}.
nipkow@10396
    76
We should first have proved that @{term id} preserves well-foundedness
nipkow@10189
    77
*}
nipkow@10189
    78
nipkow@10189
    79
lemma wf_id: "wf r \<Longrightarrow> wf(id r)"
nipkow@10189
    80
by simp;
nipkow@10189
    81
nipkow@10189
    82
text{*\noindent
nipkow@10396
    83
and should have appended the following hint to our above definition:
nipkow@10189
    84
*}
nipkow@10189
    85
(*<*)
nipkow@10189
    86
consts g :: "nat \<Rightarrow> nat"
nipkow@10189
    87
recdef g "id(less_than)"
nipkow@10189
    88
"g 0 = 0"
nipkow@10189
    89
"g (Suc n) = g n"
nipkow@10189
    90
(*>*)
nipkow@10189
    91
(hints recdef_wf add: wf_id)
nipkow@10396
    92
(*<*)end(*>*)