aboutsummaryrefslogtreecommitdiffhomepage
path: root/doc/refman
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 /doc/refman
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 'doc/refman')
-rw-r--r--doc/refman/RefMan-com.tex4
1 files changed, 2 insertions, 2 deletions
diff --git a/doc/refman/RefMan-com.tex b/doc/refman/RefMan-com.tex
index 0f1823a02..9862abb53 100644
--- a/doc/refman/RefMan-com.tex
+++ b/doc/refman/RefMan-com.tex
@@ -153,9 +153,9 @@ Add physical path {\em directory} to the {\ocaml} loadpath.
Load \Coq~file {\em file}{\tt .v} optionally with copy it contents on the
standard input.
-\item[{\tt -load-vernac-object} {\em file}]\
+\item[{\tt -load-vernac-object} {\em path}]\
- Load \Coq~compiled file {\em file}{\tt .vo}
+ Load \Coq~compiled library {\em path} (equivalent to {\tt Require} {\em path}).
\item[{\tt -require} {\em path}]\