aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/refman
diff options
context:
space:
mode:
authorGravatar glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-29 13:35:00 +0000
committerGravatar glondu <glondu@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-29 13:35:00 +0000
commit8ffad6dc0ea972bd7354be76be9e4c6a633e3692 (patch)
treec9fe4fed2a46862d363a2ac6cfb6f8461408af27 /doc/refman
parente14100f74f50b68dded694953bebf097e0ffff0c (diff)
Typo in doc
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11292 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc/refman')
-rw-r--r--doc/refman/Cases.tex29
1 files changed, 14 insertions, 15 deletions
diff --git a/doc/refman/Cases.tex b/doc/refman/Cases.tex
index a0f483ab0..6f58269f5 100644
--- a/doc/refman/Cases.tex
+++ b/doc/refman/Cases.tex
@@ -407,7 +407,7 @@ In general if $m$ has type $(I~q_1\ldots q_r~t_1\ldots t_s)$ where
$q_1\ldots q_r$ are parameters, the elimination predicate should be of
the form~:
{\tt fun $y_1$\ldots $y_s$ $x$:($I$~$q_1$\ldots $q_r$~$y_1$\ldots
- $y_s$) => P}.
+ $y_s$) => Q}.
In the concrete syntax, it should be written~:
\[ \kw{match}~m~\kw{as}~x~\kw{in}~(I~\_\ldots \_~y_1\ldots y_s)~\kw{return}~Q~\kw{with}~\ldots~\kw{end}\]
@@ -472,7 +472,7 @@ In all the previous examples the elimination predicate does not depend
on the object(s) matched. But it may depend and the typical case
is when we write a proof by induction or a function that yields an
object of dependent type. An example of proof using \texttt{match} in
-given in Section~\ref{refine-example}
+given in Section~\ref{refine-example}.
For example, we can write
the function \texttt{buildlist} that given a natural number
@@ -619,28 +619,28 @@ Here is a summary of the error messages corresponding to each situation:
\begin{ErrMsgs}
\item \sverb{The constructor } {\sl
- ident} \sverb{expects } {\sl num} \sverb{arguments}
+ ident} \sverb{ expects } {\sl num} \sverb{ arguments}
- \sverb{The variable } {\sl ident} \sverb{is bound several times
+ \sverb{The variable } {\sl ident} \sverb{ is bound several times
in pattern } {\sl term}
- \sverb{Found a constructor of inductive type} {\term}
- \sverb{while a constructor of} {\term} \sverb{is expected}
+ \sverb{Found a constructor of inductive type } {\term}
+ \sverb{ while a constructor of } {\term} \sverb{ is expected}
Patterns are incorrect (because constructors are not applied to
the correct number of the arguments, because they are not linear or
- they are wrongly typed)
+ they are wrongly typed).
\item \errindex{Non exhaustive pattern-matching}
-the pattern matching is not exhaustive
+The pattern matching is not exhaustive.
-\item \sverb{The elimination predicate } {\sl term} \sverb{should be
- of arity } {\sl num} \sverb{(for non dependent case) or } {\sl
- num} \sverb{(for dependent case)}
+\item \sverb{The elimination predicate } {\sl term} \sverb{ should be
+ of arity } {\sl num} \sverb{ (for non dependent case) or } {\sl
+ num} \sverb{ (for dependent case)}
The elimination predicate provided to \texttt{match} has not the
- expected arity
+ expected arity.
%\item the whole expression is wrongly typed
@@ -662,9 +662,8 @@ The elimination predicate provided to \texttt{match} has not the
Either there is a type incompatiblity or the problem involves\\
dependencies}
- There is a type mismatch between the different branches
-
- Then the user should provide an elimination predicate.
+ There is a type mismatch between the different branches.
+ The user should provide an elimination predicate.
% Obsolete ?
% \item because of nested patterns, it may happen that even though all