aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/refman/RefMan-coi.tex
diff options
context:
space:
mode:
Diffstat (limited to 'doc/refman/RefMan-coi.tex')
-rw-r--r--doc/refman/RefMan-coi.tex2
1 files changed, 1 insertions, 1 deletions
diff --git a/doc/refman/RefMan-coi.tex b/doc/refman/RefMan-coi.tex
index 7de837436..2c0396642 100644
--- a/doc/refman/RefMan-coi.tex
+++ b/doc/refman/RefMan-coi.tex
@@ -157,7 +157,7 @@ CoFixpoint zeros : Stream nat := cons nat 0%N zeros.
CoFixpoint from (n:nat) : Stream nat := cons nat n (from (S n)).
\end{coq_example}
-As in the \verb!Fixpoint! command (cf. section~\ref{Fixpoint}), it is possible
+As in the \verb!Fixpoint! command (see Section~\ref{Fixpoint}), it is possible
to introduce a block of mutually dependent methods. The general syntax
for this case is :