aboutsummaryrefslogtreecommitdiffhomepage
path: root/man
diff options
context:
space:
mode:
authorGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2015-09-28 11:04:59 +0200
committerGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2015-09-28 11:04:59 +0200
commit2cf609c41f7af83d9eaf43308a368fcb7307e6fa (patch)
treecdc9a1459d4b753309d7ad729bf41c7f50522adb /man
parentb6d5a9f47634371aa18c6e3159c6bc24203d229f (diff)
Make -load-vernac-object respect the loadpath.
This command-line option was behaving like the old -require, except that it did not do Import. In other words, it was loading files without respecting the loadpath. Now it behaves exactly like Require, while -require now behaves like Require Import. This patch also removes Library.require_library_from_file and all its dependencies, since they are no longer used inside Coq.
Diffstat (limited to 'man')
-rw-r--r--man/coqide.18
-rw-r--r--man/coqtop.17
2 files changed, 9 insertions, 6 deletions
diff --git a/man/coqide.1 b/man/coqide.1
index cfd9c3b4a..6a3e67ad5 100644
--- a/man/coqide.1
+++ b/man/coqide.1
@@ -63,9 +63,11 @@ Load Coq file
(Load Verbose
.IR f .).
.TP
-.BI \-load\-vernac\-object\ f
-Load Coq object file
-.IR f .vo.
+.BI \-load\-vernac\-object\ path
+Load Coq library
+.IR path
+(Require
+.IR path .).
.TP
.BI \-require\ path
Load Coq library
diff --git a/man/coqtop.1 b/man/coqtop.1
index e079bee39..62d17aa67 100644
--- a/man/coqtop.1
+++ b/man/coqtop.1
@@ -73,9 +73,10 @@ load verbosely Coq file
(Load Verbose filename.)
.TP
-.BI \-load\-vernac\-object \ filename
-load Coq object file
-.I filename.vo
+.BI \-load\-vernac\-object \ path
+load Coq library
+.I path
+(Require path.)
.TP
.BI \-require \ path