aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tactics.mli
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-11-15 22:13:28 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-11-16 13:31:49 +0100
commit4c576db3ed40328caa37144eb228365f497293e5 (patch)
treec83ff5a281e6918682510d33a28bf6412189adec /tactics/tactics.mli
parent346df3d1336bfa01bc6e58ea08245b67d3127a00 (diff)
Fixing side bug in db37c9f3f32ae7 delaying interpretation of the
right-hand side of a "change with": the rhs lives in the toplevel environment.
Diffstat (limited to 'tactics/tactics.mli')
-rw-r--r--tactics/tactics.mli2
1 files changed, 1 insertions, 1 deletions
diff --git a/tactics/tactics.mli b/tactics/tactics.mli
index 556a5a351..75b1fe704 100644
--- a/tactics/tactics.mli
+++ b/tactics/tactics.mli
@@ -125,7 +125,7 @@ val exact_proof : Constrexpr.constr_expr -> tactic
type tactic_reduction = env -> evar_map -> constr -> constr
-type change_arg = env -> evar_map -> evar_map * constr
+type change_arg = evar_map -> evar_map * constr
val reduct_in_hyp : ?check:bool -> tactic_reduction -> hyp_location -> tactic
val reduct_option : ?check:bool -> tactic_reduction * cast_kind -> goal_location -> tactic