aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tactics.mli
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2018-02-20 15:13:26 +0100
committerGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2018-03-04 17:55:50 +0100
commit9efd7ac0311f2b55756d7aa2790b0adb75c69579 (patch)
tree1ccea63a490b02a6e6da3dfcf2077cf74df274be /tactics/tactics.mli
parent6b7139b0963523fc6d1c3bf95db4dd081b59105d (diff)
tactics: export e_reduct_in_concl
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 ->