aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Zeimer <zzaimer@gmail.com>2018-07-19 15:07:12 +0200
committerGravatar Zeimer <zzaimer@gmail.com>2018-07-19 15:48:37 +0200
commit227691b56a396eb274a20168454df7d989b68bf2 (patch)
tree5cf739c255de342ea12a676d040f1f17201446fe
parentbdf65b2516b0dd5f4e1a1c6130fc49ee7712dd07 (diff)
Rewrote section 'Accessing the Type level' in the chapter 'The Coq library' of the Reference Manual.
-rw-r--r--doc/sphinx/language/coq-library.rst21
1 files changed, 16 insertions, 5 deletions
diff --git a/doc/sphinx/language/coq-library.rst b/doc/sphinx/language/coq-library.rst
index 848b3891b..52c56d2bd 100644
--- a/doc/sphinx/language/coq-library.rst
+++ b/doc/sphinx/language/coq-library.rst
@@ -705,9 +705,22 @@ fixpoint equation can be proved.
Accessing the Type level
~~~~~~~~~~~~~~~~~~~~~~~~
-The basic library includes the definitions of the counterparts of some data-types and logical
-quantifiers at the ``Type``: level: negation and properties
-of ``identity``. This is the module ``Logic_Type.v``.
+The standard library includes ``Type`` level definitions of counterparts of some
+logic concepts and basic lemmas about them.
+
+The module ``Datatypes`` defines ``identity``, which is the ``Type`` level counterpart
+of equality:
+
+.. index::
+ single: identity (term)
+
+.. coqtop:: in
+
+ Inductive identity (A:Type) (a:A) : A -> Type :=
+ identity_refl : identity a a.
+
+Some properties of ``identity`` are proved in the module ``Logic_Type``, which also
+provides the definition of ``Type`` level negation:
.. index::
single: notT (term)
@@ -716,8 +729,6 @@ of ``identity``. This is the module ``Logic_Type.v``.
Definition notT (A:Type) := A -> False.
-At the end, it defines data-types at the ``Type`` level.
-
Tactics
~~~~~~~