aboutsummaryrefslogtreecommitdiffhomepage
path: root/library
diff options
context:
space:
mode:
authorGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-12-18 18:52:54 +0000
committerGravatar ppedrot <ppedrot@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-12-18 18:52:54 +0000
commitc3ca134628ad4d9ef70a13b65c48ff17c737238f (patch)
tree136b4efbc3aefe76dcd2fa772141c774343f46df /library
parent6946bbbf2390024b3ded7654814104e709cce755 (diff)
Modulification of name
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16099 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'library')
-rw-r--r--library/impargs.mli2
-rw-r--r--library/nameops.mli14
2 files changed, 8 insertions, 8 deletions
diff --git a/library/impargs.mli b/library/impargs.mli
index 66d72abbb..de8d89166 100644
--- a/library/impargs.mli
+++ b/library/impargs.mli
@@ -95,7 +95,7 @@ type manual_implicits = manual_explicitation list
val compute_implicits_with_manual : env -> types -> bool ->
manual_implicits -> implicit_status list
-val compute_implicits_names : env -> types -> name list
+val compute_implicits_names : env -> types -> Name.t list
(** {6 Computation of implicits (done using the global environment). } *)
diff --git a/library/nameops.mli b/library/nameops.mli
index 0f71d28a1..1d3275d30 100644
--- a/library/nameops.mli
+++ b/library/nameops.mli
@@ -10,7 +10,7 @@ open Names
(** Identifiers and names *)
val pr_id : Id.t -> Pp.std_ppcmds
-val pr_name : name -> Pp.std_ppcmds
+val pr_name : Name.t -> Pp.std_ppcmds
val make_ident : string -> int option -> Id.t
val repr_ident : Id.t -> string * int option
@@ -25,15 +25,15 @@ val has_subscript : Id.t -> bool
val lift_subscript : Id.t -> Id.t
val forget_subscript : Id.t -> Id.t
-val out_name : name -> Id.t
+val out_name : Name.t -> Id.t
(** [out_name] associates [id] to [Name id]. Raises [Failure "Nameops.out_name"]
otherwise. *)
-val name_fold : (Id.t -> 'a -> 'a) -> name -> 'a -> 'a
-val name_iter : (Id.t -> unit) -> name -> unit
-val name_cons : name -> Id.t list -> Id.t list
-val name_app : (Id.t -> Id.t) -> name -> name
-val name_fold_map : ('a -> Id.t -> 'a * Id.t) -> 'a -> name -> 'a * name
+val name_fold : (Id.t -> 'a -> 'a) -> Name.t -> 'a -> 'a
+val name_iter : (Id.t -> unit) -> Name.t -> unit
+val name_cons : Name.t -> Id.t list -> Id.t list
+val name_app : (Id.t -> Id.t) -> Name.t -> Name.t
+val name_fold_map : ('a -> Id.t -> 'a * Id.t) -> 'a -> Name.t -> 'a * Name.t
val pr_lab : Label.t -> Pp.std_ppcmds