aboutsummaryrefslogtreecommitdiff
path: root/man
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2019-01-29 00:44:34 +0100
committerEmilio Jesus Gallego Arias2019-01-30 13:41:08 +0100
commitd9fb8db86d5b4ddc79a207c5f0ac32eb98215e78 (patch)
tree12c39326849f9491b5bf34f20a1aa4cb165e3933 /man
parent469032d0274812cbf00823f86fc3db3a1204647e (diff)
[toplevel] Deprecate the `-compile` flag in favor of `coqc`.
This PR deprecates the use of `coqtop` as a compiler. There is no point on having two binaries with the same purpose; after the experiment in #8690, IMHO we have a lot to gain in terms of code organization by splitting the compiler and the interactive binary. We adapt the documentation and adapt the test-suite. Note that we don't make `coqc` a true binary yet, but here we take care only of the user-facing part. The conversion of the binary will take place in #8690 and will bring code simplification, including a unified handling of arguments.
Diffstat (limited to 'man')
-rw-r--r--man/coqtop.118
1 files changed, 0 insertions, 18 deletions
diff --git a/man/coqtop.1 b/man/coqtop.1
index 084adfe453..addfb54672 100644
--- a/man/coqtop.1
+++ b/man/coqtop.1
@@ -85,22 +85,6 @@ load Coq library
and import it (Require Import path.)
.TP
-.BI \-compile \ filename.v
-compile Coq file
-.I filename.v
-(implies
-.B \-batch
-)
-
-.TP
-.BI \-compile\-verbose \ filename.v
-verbosely compile Coq file
-.I filename.v
-(implies
-.B \-batch
-)
-
-.TP
.B \-where
print Coq's standard library location and exit
@@ -125,8 +109,6 @@ batch mode (exits just after arguments parsing)
.B \-boot
boot mode (implies
.B \-q
-and
-.B \-batch
)
.TP