Skip to content

Commit 18c079d

Browse files
committed
Review changes #2
1 parent dbf029a commit 18c079d

File tree

3 files changed

+26
-23
lines changed

3 files changed

+26
-23
lines changed

doc/sphinx/language/coq-library.rst

+16-17
Original file line numberDiff line numberDiff line change
@@ -7,20 +7,19 @@ The |Coq| library
77
single: Theories
88

99

10-
The |Coq| library is structured into two parts:
10+
The |Coq| library has two parts:
1111

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.
1515

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`)
2120

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
2423
for download at http://coq.inria.fr (see
2524
Section :ref:`userscontributions`).
2625

@@ -514,8 +513,8 @@ realizability interpretation.
514513
forall (A B:Prop) (P:Type), (A -> B -> P) -> A /\ B -> P.
515514

516515

517-
Basic Arithmetics
518-
~~~~~~~~~~~~~~~~~
516+
Basic Arithmetic
517+
~~~~~~~~~~~~~~~~
519518

520519
The basic library includes a few elementary properties of natural
521520
numbers, together with the definitions of predecessor, addition and
@@ -804,8 +803,8 @@ Notation Interpretation
804803
=============== ===================
805804

806805

807-
Notations for integer arithmetics
808-
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
806+
Notations for integer arithmetic
807+
~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~~
809808

810809
.. index::
811810
single: Arithmetical notations
@@ -822,7 +821,7 @@ Notations for integer arithmetics
822821

823822

824823
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``.
826825
It specifies how notations are interpreted and, when not
827826
already reserved, the precedence and associativity.
828827

@@ -866,7 +865,7 @@ Notations for real numbers
866865

867866
This is provided by requiring and opening the module ``Reals`` and
868867
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.
870869

871870
=============== ===================
872871
Notation Interpretation

doc/sphinx/language/gallina-specification-language.rst

+9-5
Original file line numberDiff line numberDiff line change
@@ -106,20 +106,24 @@ Keywords
106106

107107
Note that plugins may define additional keywords when they are loaded.
108108

109-
Special tokens
110-
The set of special
109+
Other tokens
110+
The set of
111111
tokens defined at any given time can vary because the :cmd:`Notation`
112112
command can define new tokens. A :cmd:`Require` command may load more notation definitions,
113-
while the end of a :cmd:`Section` may remove notations.
113+
while the end of a :cmd:`Section` may remove notations. Some notations
114+
are defined in the basic library (see :ref:`thecoqlibrary`) and are normallly
115+
loaded automatically at startup time.
114116

115-
Here are some of the character sequences that are special tokens::
117+
118+
Here are the character sequences that Coq directly defines as tokens
119+
without using :cmd:`Notation` (omitting 25 specialized tokens that begin with
120+
``#int63_``)::
116121

117122
! #[ % & ' ( () (bfs) (dfs) ) * ** + , - ->
118123
. .( .. ... / : ::= := :> :>> ; < <+ <- <:
119124
<<: <= = => > >-> >= ? @ @{ [ [= ] _ _eqn
120125
`( `{ { {| | |- || }
121126

122-
123127
When multiple tokens match the beginning of a sequence of characters,
124128
the longest matching token is used.
125129
Occasionally you may need to insert spaces to separate tokens. For example,

doc/sphinx/proof-engine/ltac.rst

+1-1
Original file line numberDiff line numberDiff line change
@@ -34,7 +34,7 @@ in these grammar rules. Various already defined entries will be used in this
3434
chapter: entries :token:`num`, :token:`int`, :token:`ident`
3535
:token:`qualid`, :token:`term`, :token:`cpattern` and :token:`tactic`
3636
represent respectively natural and integer numbers,
37-
identifiers, qualified names, terms, patterns and the atomic
37+
identifiers, qualified names, Coq terms, patterns and the atomic
3838
tactics described in Chapter :ref:`tactics`.
3939

4040
The syntax of :production:`cpattern` is

0 commit comments

Comments
 (0)