aboutsummaryrefslogtreecommitdiffhomepage
path: root/library/library.mli
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 /library/library.mli
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 'library/library.mli')
-rw-r--r--library/library.mli1
1 files changed, 0 insertions, 1 deletions
diff --git a/library/library.mli b/library/library.mli
index 3d96f9a75..d5e610dd6 100644
--- a/library/library.mli
+++ b/library/library.mli
@@ -22,7 +22,6 @@ open Libnames
(** Require = load in the environment + open (if the optional boolean
is not [None]); mark also for export if the boolean is [Some true] *)
val require_library_from_dirpath : (DirPath.t * string) list -> bool option -> unit
-val require_library_from_file : CUnix.physical_path -> bool option -> unit
(** {6 Start the compilation of a library } *)