aboutsummaryrefslogtreecommitdiff
diff options
context:
space:
mode:
-rw-r--r--library/libnames.ml5
-rw-r--r--library/libnames.mli2
-rw-r--r--tactics/declare.ml4
3 files changed, 2 insertions, 9 deletions
diff --git a/library/libnames.ml b/library/libnames.ml
index 18af216e46..485f8837e8 100644
--- a/library/libnames.ml
+++ b/library/libnames.ml
@@ -128,11 +128,6 @@ let path_of_string s =
let pr_path sp = str (string_of_path sp)
-let restrict_path n sp =
- let dir, s = repr_path sp in
- let dir' = List.firstn n (DirPath.repr dir) in
- make_path (DirPath.make dir') s
-
(*s qualified names *)
type qualid_r = full_path
type qualid = qualid_r CAst.t
diff --git a/library/libnames.mli b/library/libnames.mli
index 4455e29818..ffd7032fff 100644
--- a/library/libnames.mli
+++ b/library/libnames.mli
@@ -57,8 +57,6 @@ val pr_path : full_path -> Pp.t
module Spmap : CSig.MapS with type key = full_path
-val restrict_path : int -> full_path -> full_path
-
(** {6 ... } *)
(** A [qualid] is a partially qualified ident; it includes fully
qualified names (= absolute names) and all intermediate partial
diff --git a/tactics/declare.ml b/tactics/declare.ml
index e550e06471..dbf570eaad 100644
--- a/tactics/declare.ml
+++ b/tactics/declare.ml
@@ -301,7 +301,7 @@ type section_variable_entry =
type variable_declaration = DirPath.t * section_variable_entry
-let cache_variable ((sp,_),o) =
+let cache_variable (_,o) =
match o with
| Inl ctx -> Global.push_context_set false ctx
| Inr (id,(path,d),kind) ->
@@ -339,7 +339,7 @@ let cache_variable ((sp,_),o) =
let () = Global.push_named_def (id, se) in
Decl_kinds.Explicit, de.proof_entry_opaque,
poly, univs in
- Nametab.push (Nametab.Until 1) (Libnames.restrict_path 0 sp) (GlobRef.VarRef id);
+ Nametab.push (Nametab.Until 1) (Libnames.make_path DirPath.empty id) (GlobRef.VarRef id);
add_section_variable ~name:id ~kind:impl ~poly univs;
Decls.(add_variable_data id {path;opaque;univs;poly;kind})