aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/refman
diff options
context:
space:
mode:
authorGravatar Matej Kosik <m4tej.kosik@gmail.com>2015-11-06 15:18:35 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-12-10 09:35:17 +0100
commitf7051cd4eb4cefc4b2ec04c8c29369dcaf0062f2 (patch)
treedff6af1b49e6de4b071db84487417cdc06faf17c /doc/refman
parent38fc8566ab59bcf67e6eeaf5860ce97cfab38e74 (diff)
ENH: define the meaning of 'p'
Diffstat (limited to 'doc/refman')
-rw-r--r--doc/refman/RefMan-cic.tex4
1 files changed, 2 insertions, 2 deletions
diff --git a/doc/refman/RefMan-cic.tex b/doc/refman/RefMan-cic.tex
index 87ef046fa..91c141854 100644
--- a/doc/refman/RefMan-cic.tex
+++ b/doc/refman/RefMan-cic.tex
@@ -1571,7 +1571,7 @@ elimination on any sort is allowed.
Let $c$ be a term of type $C$, we assume $C$ is a type of constructor
for an inductive type $I$. Let $P$ be a term that represents the
property to be proved.
-We assume $r$ is the number of parameters.
+We assume $r$ is the number of parameters and $p$ is the number of arguments.
We define a new type \CI{c:C}{P} which represents the type of the
branch corresponding to the $c:C$ constructor.
@@ -1584,7 +1584,7 @@ branch corresponding to the $c:C$ constructor.
We write \CI{c}{P} for \CI{c:C}{P} with $C$ the type of $c$.
\paragraph{Examples.}
-For $\ListA$ the type of $P$ will be $\ListA\ra s$ for $s \in \Sort$. \\
+For $\List \nat$ the type of $P$ will be $\ListA\ra s$ for $s \in \Sort$. \\
$ \CI{(\cons~A)}{P} \equiv
\forall a:A, \forall l:\ListA,(P~(\cons~A~a~l))$.