aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/refman/RefMan-cic.tex
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-10-04 08:47:15 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-12-10 09:35:05 +0100
commit75896eaaf60ce947e1fbc5a795ca5969bb1e4fae (patch)
treec9b000ca8676a1f2906890ce3db947334bf2a923 /doc/refman/RefMan-cic.tex
parentcd31e372c6fb25769c26879f2f65f1937d098b87 (diff)
RefMan, ch. 4: Dropping the "Co" which noone uses in "(Co)Inductive".
Diffstat (limited to 'doc/refman/RefMan-cic.tex')
-rw-r--r--doc/refman/RefMan-cic.tex16
1 files changed, 9 insertions, 7 deletions
diff --git a/doc/refman/RefMan-cic.tex b/doc/refman/RefMan-cic.tex
index 3b8a8fee1..2bf5bb357 100644
--- a/doc/refman/RefMan-cic.tex
+++ b/doc/refman/RefMan-cic.tex
@@ -2,20 +2,22 @@
\label{Cic}
\index{Cic@\textsc{CIC}}
\index{pCic@p\textsc{CIC}}
-\index{Calculus of (Co)Inductive Constructions}}
+\index{Calculus of Inductive Constructions}}
The underlying formal language of {\Coq} is a {\em Calculus of
- Constructions} with {\em Inductive Definitions}. It is presented in
-this chapter.
+ Constructions} with {\em Inductive Definitions}, also featuring a
+universe hierarchy and coinductive types. Its inference rules are
+presented in this chapter.
+
For {\Coq} version V7, this Calculus was known as the
-{\em Calculus of (Co)Inductive Constructions}\index{Calculus of
- (Co)Inductive Constructions} (\iCIC\ in short).
+{\em Calculus of Inductive Constructions}\index{Calculus of
+ Inductive Constructions} (\iCIC\ in short).
The underlying calculus of {\Coq} version V8.0 and up is a weaker
calculus where the sort \Set{} satisfies predicative rules.
We call this calculus the
-{\em Predicative Calculus of (Co)Inductive
+{\em Predicative Calculus of Inductive
Constructions}\index{Predicative Calculus of
- (Co)Inductive Constructions} (\pCIC\ in short).
+ Inductive Constructions} (\pCIC\ in short).
In Section~\ref{impredicativity} we give the extra-rules for \iCIC. A
compiling option of \Coq{} allows type-checking theories in this
extended system.