aboutsummaryrefslogtreecommitdiffhomepage
path: root/library/loadpath.mli
diff options
context:
space:
mode:
authorGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2014-03-07 16:38:59 +0100
committerGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2014-03-07 16:38:59 +0100
commitd692c5dc034778a1d97ace593c9a3658a44e698b (patch)
tree7b66e9e5056660511a7a3d73efa4eea2fda24eba /library/loadpath.mli
parentb80cf566a39efe65f5ef0b1cc4ff9bb295a67fc7 (diff)
Fix lookup of native files when option -R is missing.
Testcase: mkdir a echo "Definition t := O." > a/a.v coqc -R a a a/a.v echo "Require Import a.a. Definition u := t." > b.v coqc -I . b.v rm -rf a b.*
Diffstat (limited to 'library/loadpath.mli')
-rw-r--r--library/loadpath.mli3
1 files changed, 3 insertions, 0 deletions
diff --git a/library/loadpath.mli b/library/loadpath.mli
index 8928542a6..f755ace9e 100644
--- a/library/loadpath.mli
+++ b/library/loadpath.mli
@@ -30,6 +30,9 @@ val get_load_paths : unit -> t list
val get_paths : unit -> CUnix.physical_path list
(** Same as [get_load_paths] but only get the physical part. *)
+val get_accessible_paths : unit -> CUnix.physical_path list
+(** Same as [get_paths] but also get paths that can be relatively accessed. *)
+
val add_load_path : CUnix.physical_path -> bool -> DirPath.t -> unit
(** [add_load_path root phys log] adds the binding [phys := log] to the current
loadpaths. The [root] flag indicates whether this loadpath has to be treated