aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc
diff options
context:
space:
mode:
authorGravatar Amin Timany <amintimany@gmail.com>2017-08-02 09:42:37 +0200
committerGravatar Amin Timany <amintimany@gmail.com>2017-08-02 09:42:37 +0200
commit2f0e71c7e25eb193f252b6848dadff771dbc270d (patch)
treebc6c44f91227d581b995c586a3a0cc733368d9f6 /doc
parent819fd4a7a431efb41a080e7aabef2a66a3ca2417 (diff)
Typo in the documentation of cumulativity
Diffstat (limited to 'doc')
-rw-r--r--doc/refman/Universes.tex10
1 files changed, 5 insertions, 5 deletions
diff --git a/doc/refman/Universes.tex b/doc/refman/Universes.tex
index 667fd6698..cd36d1d32 100644
--- a/doc/refman/Universes.tex
+++ b/doc/refman/Universes.tex
@@ -173,17 +173,17 @@ convertible if and only if \texttt{i $=$ j}.
Cumulative inductive types, coninductive types, variants and records
only make sense when they are universe polymorphic. Therefore, an
error is issued whenever the user uses the \texttt{Cumulative} or
-\texttt{NonCumulative} prefix in a monomorphic contexts.
+\texttt{NonCumulative} prefix in a monomorphic context.
Notice that this is not the case for the option \texttt{Set Polymorphic Inductive Cumulativity}.
-That is, this optiotion, when set, makes all subsequent \emph{polymorphic}
-inductive declarations cumulative (unless, of course if the \texttt{NonCumulative} prefix is used)
+That is, this option, when set, makes all subsequent \emph{polymorphic}
+inductive declarations cumulative (unless, of course the \texttt{NonCumulative} prefix is used)
but has no effect on \emph{monomorphic} inductive declarations.
Consider the following examples.
\begin{coq_example}
-Fail Monomorphic Cumulative Inductive Unit := unit.
+Monomorphic Cumulative Inductive Unit := unit.
\end{coq_example}
\begin{coq_example}
-Fail Monomorphic NonCumulative Inductive Unit := unit.
+Monomorphic NonCumulative Inductive Unit := unit.
\end{coq_example}
\begin{coq_example*}
Set Polymorphic Inductive Cumulativity.