@@ -7,20 +7,19 @@ The |Coq| library
7
7
single: Theories
8
8
9
9
10
- The |Coq | library is structured into two parts:
10
+ The |Coq | library has two parts:
11
11
12
- * **The initial library **: it contains elementary logical notions and
13
- data-types. It constitutes the basic state of the system directly
14
- available when running |Coq |;
12
+ * **The basic library **: definitions and theorems for
13
+ the most commonly used elementary logical notions and
14
+ data types. |Coq | normally loads these files automatically when it starts.
15
15
16
- * **The standard library **: general-purpose libraries containing various
17
- developments of |Coq | axiomatizations about sets, lists, sorting,
18
- arithmetic, etc. This library comes with the system and its modules
19
- are directly accessible through the ``Require `` command (see
20
- Section :ref: `compiled-files `);
16
+ * **The standard library **: general-purpose libraries with
17
+ definitions and theorems for sets, lists, sorting,
18
+ arithmetic, etc. To use these files, users must load them explicitly
19
+ with the ``Require `` command (see Section :ref: `compiled-files `)
21
20
22
- In addition, user-provided libraries or developments are provided by
23
- | Coq | users' community. These libraries and developments are available
21
+ There are also many libraries provided by | Coq | users' community.
22
+ These libraries and developments are available
24
23
for download at http://coq.inria.fr (see
25
24
Section :ref: `userscontributions `).
26
25
@@ -514,8 +513,8 @@ realizability interpretation.
514
513
forall (A B:Prop) (P:Type), (A -> B -> P) -> A /\ B -> P.
515
514
516
515
517
- Basic Arithmetics
518
- ~~~~~~~~~~~~~~~~~
516
+ Basic Arithmetic
517
+ ~~~~~~~~~~~~~~~~
519
518
520
519
The basic library includes a few elementary properties of natural
521
520
numbers, together with the definitions of predecessor, addition and
@@ -804,8 +803,8 @@ Notation Interpretation
804
803
=============== ===================
805
804
806
805
807
- Notations for integer arithmetics
808
- ~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
806
+ Notations for integer arithmetic
807
+ ~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
809
808
810
809
.. index ::
811
810
single: Arithmetical notations
@@ -822,7 +821,7 @@ Notations for integer arithmetics
822
821
823
822
824
823
The following table describes the syntax of expressions
825
- for integer arithmetics . It is provided by requiring and opening the module ``ZArith `` and opening scope ``Z_scope ``.
824
+ for integer arithmetic . It is provided by requiring and opening the module ``ZArith `` and opening scope ``Z_scope ``.
826
825
It specifies how notations are interpreted and, when not
827
826
already reserved, the precedence and associativity.
828
827
@@ -866,7 +865,7 @@ Notations for real numbers
866
865
867
866
This is provided by requiring and opening the module ``Reals `` and
868
867
opening scope ``R_scope ``. This set of notations is very similar to
869
- the notation for integer arithmetics . The inverse function was added.
868
+ the notation for integer arithmetic . The inverse function was added.
870
869
871
870
=============== ===================
872
871
Notation Interpretation
0 commit comments