Skip to content

Commit

Permalink
Apply suggestions from code review
Browse files Browse the repository at this point in the history
Co-authored-by: Théo Zimmermann <[email protected]>
  • Loading branch information
SkySkimmer and Zimmi48 authored Dec 13, 2024
1 parent 6d358b1 commit 0e7dcf7
Show file tree
Hide file tree
Showing 2 changed files with 9 additions and 10 deletions.
4 changes: 2 additions & 2 deletions doc/sphinx/language/cic.rst
Original file line number Diff line number Diff line change
Expand Up @@ -443,8 +443,8 @@ command, the following is rejected,

Fail Definition id: Set := forall X:Set,X->X.

while it will type check, if one uses instead the `rocq repl`
``-impredicative-set`` option..
while it will type check, if one uses instead the
``-impredicative-set`` command-line flag.

The major change in the theory concerns the rule for product formation
in the sort :math:`\Set`, which is extended to a domain in any sort:
Expand Down
15 changes: 7 additions & 8 deletions doc/sphinx/practical-tools/coq-commands.rst
Original file line number Diff line number Diff line change
Expand Up @@ -9,7 +9,7 @@ There are several Rocq commands:
:ref:`here <coqintegrateddevelopmentenvironment>`. In addition, there are
several other IDEs such as Proof General, vsCoq and Coqtail that are not
included with the Coq installation.
+ ``rocq``: the main entry point for Rocq
+ ``rocq``: the main entry point for the Rocq prover
+ ``rocqchk``: the Rocq checker (validation of compiled libraries) (also available through ``rocq check``)

Many of the parameters to start these tools are shared and are described below.
Expand All @@ -22,13 +22,12 @@ but they are probably less current than `-help` or this document).
Interactive use (rocq repl)
---------------------------

In the interactive mode, also known as the Coq toplevel, users can
develop their theories and proofs step by step. The Coq toplevel is run
The Rocq toplevel (or read-eval-print-loop) is run
by the command ``rocq repl`` (equivalently, `rocq top`).

There is also a byte-code toplevel `rocq repl-with-drop` based on an OCaml toplevel.
You can switch to the OCaml toplevel with the command ``Drop.``,
and come back to the Coq toplevel with the command ``#go;;``.
and come back to the Rocq toplevel with the command ``#go;;``.

.. flag:: Coqtop Exit On Error

Expand All @@ -39,9 +38,9 @@ Batch compilation (rocq compile)
--------------------------------

The ``rocq compile`` (equivalently, `rocq c`) command compiles
a Coq proof script file with a ".v" suffix
a Rocq proof script file with a ".v" suffix
to create a compiled file with a ".vo" suffix. (See :ref:`compiled-files`.)
The last component of the filename must be a valid Coq identifier as described in
The last component of the filename must be a valid Rocq identifier as described in
:ref:`lexical-conventions`; it should contain only letters, digits or
underscores (_) with a ".v" suffix on the final component.
For example ``/bar/foo/toto.v`` is valid, but ``/bar/foo/to-to.v`` is not.
Expand All @@ -66,7 +65,7 @@ See :ref:`rocq_makefile` and :ref:`building_dune`.
`_CoqProject` file (see :ref:`rocq_makefile`) in the directory from which you
start `CoqIDE` or give it as an argument to the ``coqide`` command.
*<PATH>* is the pathname of the directory containing the module,
which can be an absolute path or relative to Coq's current directory. For now,
which can be an absolute path or relative to Rocq's current directory. For now,
you must close and reload a named script file for `CoqIDE` to pick up the change,
or restart `CoqIDE`.
The project file name is configurable in `Edit / Preferences / Project`.
Expand All @@ -91,7 +90,7 @@ In order of importance they are:
~~~~~~~~~~~~~~~~~~~~~~~

When Rocq is launched, it can implicitly prepend a startup script to any document
read by Rocq, whether it is an interactive session or a file to compile.
it reads, whether it is an interactive session or a file to compile.
The startup script can come from a configuration directory or it can be
specified on the command line.

Expand Down

0 comments on commit 0e7dcf7

Please sign in to comment.