aboutsummaryrefslogtreecommitdiffhomepage
path: root/engine
diff options
context:
space:
mode:
authorGravatar Matej Kosik <matej.kosik@inria.fr>2016-08-14 18:36:30 +0200
committerGravatar Matej Kosik <matej.kosik@inria.fr>2016-08-25 07:53:02 +0200
commit4688a3b9750827eb0f5f61066ca617efcd97bc8c (patch)
tree33289dff2847f51ef99f7711bee7624ca80a9341 /engine
parent16ecabd99d66b3068e17fae486ba4ed77954e813 (diff)
CLEANUP: functions "Context.{Rel,Named}.Context.fold" were renamed to "Context.{Rel,Named}.fold_constr"
Diffstat (limited to 'engine')
-rw-r--r--engine/evarutil.ml2
-rw-r--r--engine/evd.ml8
2 files changed, 5 insertions, 5 deletions
diff --git a/engine/evarutil.ml b/engine/evarutil.ml
index fcb429aef..326cd25fc 100644
--- a/engine/evarutil.ml
+++ b/engine/evarutil.ml
@@ -689,7 +689,7 @@ let undefined_evars_of_term evd t =
let undefined_evars_of_named_context evd nc =
Context.Named.fold_outside
- (NamedDecl.fold (fun c s -> Evar.Set.union s (undefined_evars_of_term evd c)))
+ (NamedDecl.fold_constr (fun c s -> Evar.Set.union s (undefined_evars_of_term evd c)))
nc
~init:Evar.Set.empty
diff --git a/engine/evd.ml b/engine/evd.ml
index 036abbdeb..d573a9f05 100644
--- a/engine/evd.ml
+++ b/engine/evd.ml
@@ -287,7 +287,7 @@ let metavars_of c =
let rec collrec acc c =
match kind_of_term c with
| Meta mv -> Int.Set.add mv acc
- | _ -> fold_constr collrec acc c
+ | _ -> Term.fold_constr collrec acc c
in
collrec Int.Set.empty c
@@ -734,20 +734,20 @@ let evar_list c =
let rec evrec acc c =
match kind_of_term c with
| Evar (evk, _ as ev) -> ev :: acc
- | _ -> fold_constr evrec acc c in
+ | _ -> Term.fold_constr evrec acc c in
evrec [] c
let evars_of_term c =
let rec evrec acc c =
match kind_of_term c with
| Evar (n, l) -> Evar.Set.add n (Array.fold_left evrec acc l)
- | _ -> fold_constr evrec acc c
+ | _ -> Term.fold_constr evrec acc c
in
evrec Evar.Set.empty c
let evars_of_named_context nc =
Context.Named.fold_outside
- (NamedDecl.fold (fun constr s -> Evar.Set.union s (evars_of_term constr)))
+ (NamedDecl.fold_constr (fun constr s -> Evar.Set.union s (evars_of_term constr)))
nc
~init:Evar.Set.empty