aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/context.ml
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 /kernel/context.ml
parent16ecabd99d66b3068e17fae486ba4ed77954e813 (diff)
CLEANUP: functions "Context.{Rel,Named}.Context.fold" were renamed to "Context.{Rel,Named}.fold_constr"
Diffstat (limited to 'kernel/context.ml')
-rw-r--r--kernel/context.ml4
1 files changed, 2 insertions, 2 deletions
diff --git a/kernel/context.ml b/kernel/context.ml
index 43be9fc4f..4c88283ca 100644
--- a/kernel/context.ml
+++ b/kernel/context.ml
@@ -138,7 +138,7 @@ struct
| LocalDef (_,v,ty) -> f v; f ty
(** Reduce all terms in a given declaration to a single value. *)
- let fold f decl acc =
+ let fold_constr f decl acc =
match decl with
| LocalAssum (n,ty) -> f ty acc
| LocalDef (n,v,ty) -> f ty (f v acc)
@@ -333,7 +333,7 @@ struct
| LocalDef (_, v, ty) -> f v; f ty
(** Reduce all terms in a given declaration to a single value. *)
- let fold f decl a =
+ let fold_constr f decl a =
match decl with
| LocalAssum (_, ty) -> f ty a
| LocalDef (_, v, ty) -> a |> f v |> f ty