aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/find_subterm.mli
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-11-10 17:26:36 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-11-10 17:27:07 +0100
commitd57e30cfe8f68987ed216415079f4dab42065408 (patch)
treec95b7b789fa20ca464b69ceccddd6047ba1e4505 /pretyping/find_subterm.mli
parent07620386b3c1b535ee7e43306a6345f015a318f0 (diff)
Revert "Fixing #1225: we now skip the canonically built binding contexts of"
This reverts commit 07620386b3c1b535ee7e43306a6345f015a318f0. Very sorry not ready.
Diffstat (limited to 'pretyping/find_subterm.mli')
-rw-r--r--pretyping/find_subterm.mli5
1 files changed, 2 insertions, 3 deletions
diff --git a/pretyping/find_subterm.mli b/pretyping/find_subterm.mli
index 23d7ed949..47d9654e5 100644
--- a/pretyping/find_subterm.mli
+++ b/pretyping/find_subterm.mli
@@ -29,7 +29,6 @@ exception SubtermUnificationError of subterm_unification_error
type 'a testing_function = {
match_fun : 'a -> constr -> 'a;
merge_fun : 'a -> 'a -> 'a;
- get_evars : 'a -> evar_map;
mutable testing_state : 'a;
mutable last_found : position_reporting option
}
@@ -44,14 +43,14 @@ val make_eq_univs_test : env -> evar_map -> constr -> evar_map testing_function
()]; it turns a NotUnifiable exception raised by the testing
function into a SubtermUnificationError. *)
val replace_term_occ_modulo : occurrences or_like_first ->
- 'a testing_function -> (unit -> constr) -> env -> constr -> constr
+ 'a testing_function -> (unit -> constr) -> constr -> constr
(** [replace_term_occ_decl_modulo] is similar to
[replace_term_occ_modulo] but for a named_declaration. *)
val replace_term_occ_decl_modulo :
(occurrences * hyp_location_flag) or_like_first ->
'a testing_function -> (unit -> constr) ->
- env -> named_declaration -> named_declaration
+ named_declaration -> named_declaration
(** [subst_closed_term_occ occl c d] replaces occurrences of
closed [c] at positions [occl] by [Rel 1] in [d] (see also Note OCC),