aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tactics.mli
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2018-03-05 13:15:15 +0100
committerGravatar Maxime Dénès <mail@maximedenes.fr>2018-03-05 13:15:15 +0100
commit736e86e06b5831a0dd4b6a655708b4ffd2b4ee64 (patch)
treef1f572e011f0e5e476256d58517258774bdf149e /tactics/tactics.mli
parenta46a04577e34c69b42c2728ec1e0babb5be23e31 (diff)
parent7267e31fa4456aee62a1e39dfdb7e38a8832f93f (diff)
Merge PR #6700: [ssr] rewrite Ssripats and Ssrview in the tactic monad
Diffstat (limited to 'tactics/tactics.mli')
-rw-r--r--tactics/tactics.mli4
1 files changed, 3 insertions, 1 deletions
diff --git a/tactics/tactics.mli b/tactics/tactics.mli
index 100ddf17f..5a29ff694 100644
--- a/tactics/tactics.mli
+++ b/tactics/tactics.mli
@@ -130,7 +130,8 @@ val exact_proof : Constrexpr.constr_expr -> unit Proofview.tactic
(** {6 Reduction tactics. } *)
-type tactic_reduction = env -> evar_map -> constr -> constr
+type tactic_reduction = Reductionops.reduction_function
+type e_tactic_reduction = Reductionops.e_reduction_function
type change_arg = patvar_map -> evar_map -> evar_map * constr
@@ -138,6 +139,7 @@ val make_change_arg : constr -> change_arg
val reduct_in_hyp : ?check:bool -> tactic_reduction -> hyp_location -> unit Proofview.tactic
val reduct_option : ?check:bool -> tactic_reduction * cast_kind -> goal_location -> unit Proofview.tactic
val reduct_in_concl : tactic_reduction * cast_kind -> unit Proofview.tactic
+val e_reduct_in_concl : check:bool -> e_tactic_reduction * cast_kind -> unit Proofview.tactic
val change_in_concl : (occurrences * constr_pattern) option -> change_arg -> unit Proofview.tactic
val change_concl : constr -> unit Proofview.tactic
val change_in_hyp : (occurrences * constr_pattern) option -> change_arg ->