aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-09-01 21:47:37 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-09-01 21:47:37 +0000
commit6e58d190a40f27b8e2039c4063523f9f3e62215b (patch)
treeb6974c81c6cdbe4ec4e31718f8c01c0e8afc2044 /doc
parentaae13cd8c4d76a0c1d7db42e4451c63587a1ab56 (diff)
A word on the measure and wf modifiers
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10110 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc')
-rw-r--r--doc/refman/Program.tex8
1 files changed, 6 insertions, 2 deletions
diff --git a/doc/refman/Program.tex b/doc/refman/Program.tex
index 4357f57e8..d5c8ec5e4 100644
--- a/doc/refman/Program.tex
+++ b/doc/refman/Program.tex
@@ -161,7 +161,11 @@ Program Fixpoint div2 (n : nat) {measure id n} : { x : nat | n = 2 * x \/ n = 2
end.
\end{coq_example}
-\emph{Caution:} When defining structurally recursive functions, the
+The \verb|measure| keyword expects a measure function into the naturals, whereas
+\verb|wf| expects a relation.
+
+\paragraph{Caution}
+When defining structurally recursive functions, the
generated obligations should have the prototype of the currently defined functional
in their context. In this case, the obligations should be transparent
(e.g. using Defined) so that the guardedness condition on
@@ -174,7 +178,7 @@ context, the proof of the obligation is \emph{required} to be declared transpare
No such problems arise when using measures or well-founded recursion.
-An important point about wellfounded and measure-based functions is the following:
+An important point about well-founded and measure-based functions is the following:
The recursive prototype of a function of type
{\binder$_1$}\ldots{\binder$_n$} \{ {\tt measure m \binder$_i$} \}:{\type$_1$},
inside the body is