aboutsummaryrefslogtreecommitdiff
path: root/interp/constrintern.mli
diff options
context:
space:
mode:
authorppedrot2013-08-03 18:35:03 +0000
committerppedrot2013-08-03 18:35:03 +0000
commit2b8ad61822111fad93176b54800cb43e347df292 (patch)
tree9a4668cc5533d355a69c3f6583658ee9e342c66b /interp/constrintern.mli
parenteb4bdf9317ad53f464a87219c1625b9118d4660a (diff)
Replacing uses of association lists by maps in notations.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@16655 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'interp/constrintern.mli')
-rw-r--r--interp/constrintern.mli14
1 files changed, 6 insertions, 8 deletions
diff --git a/interp/constrintern.mli b/interp/constrintern.mli
index 2a80856827..5535b6c84e 100644
--- a/interp/constrintern.mli
+++ b/interp/constrintern.mli
@@ -68,7 +68,7 @@ val compute_internalization_env : env -> var_internalization_type ->
Id.t list -> types list -> Impargs.manual_explicitation list list ->
internalization_env
-type ltac_sign = Id.t list * Id.Set.t
+type ltac_sign = Id.Set.t * Id.Set.t
type glob_binder = (Name.t * binding_kind * glob_constr option * glob_constr)
@@ -163,14 +163,12 @@ val construct_reference : named_context -> Id.t -> constr
val global_reference : Id.t -> constr
val global_reference_in_absolute_module : DirPath.t -> Id.t -> constr
-(** Interprets a term as the left-hand side of a notation; the boolean
- list is a set and this set is [true] for a variable occurring in
- term position, [false] for a variable occurring in binding
- position; [true;false] if in both kinds of position *)
+(** Interprets a term as the left-hand side of a notation. The returned map is
+ guaranteed to have the same domain as the input one. *)
val interp_notation_constr : ?impls:internalization_env ->
- (Id.t * notation_var_internalization_type) list ->
- (Id.t * Id.t) list -> constr_expr ->
- (Id.t * (subscopes * notation_var_internalization_type)) list *
+ notation_var_internalization_type Id.Map.t ->
+ Id.t Id.Map.t -> constr_expr ->
+ (subscopes * notation_var_internalization_type) Id.Map.t *
notation_constr
(** Globalization options *)