aboutsummaryrefslogtreecommitdiffhomepage
path: root/intf/glob_term.mli
diff options
context:
space:
mode:
Diffstat (limited to 'intf/glob_term.mli')
-rw-r--r--intf/glob_term.mli38
1 files changed, 19 insertions, 19 deletions
diff --git a/intf/glob_term.mli b/intf/glob_term.mli
index 7ee0320f0..5cb369562 100644
--- a/intf/glob_term.mli
+++ b/intf/glob_term.mli
@@ -27,31 +27,31 @@ open Misctypes
locs here refers to the ident's location, not whole pat *)
type cases_pattern =
- | PatVar of loc * name
- | PatCstr of loc * constructor * cases_pattern list * name
+ | PatVar of Loc.t * name
+ | PatCstr of Loc.t * constructor * cases_pattern list * name
(** [PatCstr(p,C,l,x)] = "|'C' 'l' as 'x'" *)
type glob_constr =
- | GRef of (loc * global_reference)
- | GVar of (loc * identifier)
- | GEvar of loc * existential_key * glob_constr list option
- | GPatVar of loc * (bool * patvar) (** Used for patterns only *)
- | GApp of loc * glob_constr * glob_constr list
- | GLambda of loc * name * binding_kind * glob_constr * glob_constr
- | GProd of loc * name * binding_kind * glob_constr * glob_constr
- | GLetIn of loc * name * glob_constr * glob_constr
- | GCases of loc * case_style * glob_constr option * tomatch_tuples * cases_clauses
+ | GRef of (Loc.t * global_reference)
+ | GVar of (Loc.t * identifier)
+ | GEvar of Loc.t * existential_key * glob_constr list option
+ | GPatVar of Loc.t * (bool * patvar) (** Used for patterns only *)
+ | GApp of Loc.t * glob_constr * glob_constr list
+ | GLambda of Loc.t * name * binding_kind * glob_constr * glob_constr
+ | GProd of Loc.t * name * binding_kind * glob_constr * glob_constr
+ | GLetIn of Loc.t * name * glob_constr * glob_constr
+ | GCases of Loc.t * case_style * glob_constr option * tomatch_tuples * cases_clauses
(** [GCases(l,style,r,tur,cc)] = "match 'tur' return 'r' with 'cc'" (in
[MatchStyle]) *)
- | GLetTuple of loc * name list * (name * glob_constr option) *
+ | GLetTuple of Loc.t * name list * (name * glob_constr option) *
glob_constr * glob_constr
- | GIf of loc * glob_constr * (name * glob_constr option) * glob_constr * glob_constr
- | GRec of loc * fix_kind * identifier array * glob_decl list array *
+ | GIf of Loc.t * glob_constr * (name * glob_constr option) * glob_constr * glob_constr
+ | GRec of Loc.t * fix_kind * identifier array * glob_decl list array *
glob_constr array * glob_constr array
- | GSort of loc * glob_sort
- | GHole of (loc * Evar_kinds.t)
- | GCast of loc * glob_constr * glob_constr cast_type
+ | GSort of Loc.t * glob_sort
+ | GHole of (Loc.t * Evar_kinds.t)
+ | GCast of Loc.t * glob_constr * glob_constr cast_type
and glob_decl = name * binding_kind * glob_constr option * glob_constr
@@ -65,14 +65,14 @@ and fix_kind =
| GCoFix of int
and predicate_pattern =
- name * (loc * inductive * name list) option
+ name * (Loc.t * inductive * name list) option
(** [(na,id)] = "as 'na' in 'id'" where if [id] is [Some(l,I,k,args)]. *)
and tomatch_tuple = (glob_constr * predicate_pattern)
and tomatch_tuples = tomatch_tuple list
-and cases_clause = (loc * identifier list * cases_pattern list * glob_constr)
+and cases_clause = (Loc.t * identifier list * cases_pattern list * glob_constr)
(** [(p,il,cl,t)] = "|'cl' as 'il' => 't'" *)
and cases_clauses = cases_clause list