aboutsummaryrefslogtreecommitdiffhomepage
path: root/interp/implicit_quantifiers.mli
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 /interp/implicit_quantifiers.mli
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 'interp/implicit_quantifiers.mli')
-rw-r--r--interp/implicit_quantifiers.mli14
1 files changed, 7 insertions, 7 deletions
diff --git a/interp/implicit_quantifiers.mli b/interp/implicit_quantifiers.mli
index 2c5ad7408..66be2ae5a 100644
--- a/interp/implicit_quantifiers.mli
+++ b/interp/implicit_quantifiers.mli
@@ -34,23 +34,23 @@ val free_vars_of_constr_expr : constr_expr -> ?bound:Id.Set.t ->
Id.t list -> Id.t list
val free_vars_of_binders :
- ?bound:Id.Set.t -> Names.Id.t list -> local_binder list -> Id.Set.t * Names.Id.t list
+ ?bound:Id.Set.t -> Id.t list -> local_binder list -> Id.Set.t * Id.t list
(** Returns the generalizable free ids in left-to-right
order with the location of their first occurence *)
val generalizable_vars_of_glob_constr : ?bound:Id.Set.t -> ?allowed:Id.Set.t ->
- glob_constr -> (Names.Id.t * Loc.t) list
+ glob_constr -> (Id.t * Loc.t) list
-val make_fresh : Names.Id.Set.t -> Environ.env -> Id.t -> Id.t
+val make_fresh : Id.Set.t -> Environ.env -> Id.t -> Id.t
val implicits_of_glob_constr : ?with_products:bool -> Glob_term.glob_constr -> Impargs.manual_implicits
val combine_params_freevar :
- Names.Id.Set.t -> (global_reference * bool) option * (Names.name * Term.constr option * Term.types) ->
- Constrexpr.constr_expr * Names.Id.Set.t
+ Id.Set.t -> (global_reference * bool) option * (Name.t * Term.constr option * Term.types) ->
+ Constrexpr.constr_expr * Id.Set.t
val implicit_application : Id.Set.t -> ?allow_partial:bool ->
- (Names.Id.Set.t -> (global_reference * bool) option * (Names.name * Term.constr option * Term.types) ->
- Constrexpr.constr_expr * Names.Id.Set.t) ->
+ (Id.Set.t -> (global_reference * bool) option * (Name.t * Term.constr option * Term.types) ->
+ Constrexpr.constr_expr * Id.Set.t) ->
constr_expr -> constr_expr * Id.Set.t