aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tactics.mli
diff options
context:
space:
mode:
Diffstat (limited to 'tactics/tactics.mli')
-rw-r--r--tactics/tactics.mli9
1 files changed, 4 insertions, 5 deletions
diff --git a/tactics/tactics.mli b/tactics/tactics.mli
index ce31a4dcc..2e35c1761 100644
--- a/tactics/tactics.mli
+++ b/tactics/tactics.mli
@@ -96,7 +96,7 @@ val try_intros_until :
val assumption : tactic
val exact_no_check : constr -> tactic
val exact_check : constr -> tactic
-val exact_proof : Coqast.t -> tactic
+val exact_proof : Topconstr.constr_expr -> tactic
(*s Reduction tactics. *)
@@ -121,12 +121,11 @@ val simpl_option : hyp_location option -> tactic
val normalise_in_concl: tactic
val normalise_in_hyp : hyp_location -> tactic
val normalise_option : hyp_location option -> tactic
-val unfold_in_concl : (int list * Closure.evaluable_global_reference) list
- -> tactic
+val unfold_in_concl : (int list * evaluable_global_reference) list -> tactic
val unfold_in_hyp :
- (int list * Closure.evaluable_global_reference) list -> hyp_location -> tactic
+ (int list * evaluable_global_reference) list -> hyp_location -> tactic
val unfold_option :
- (int list * Closure.evaluable_global_reference) list -> hyp_location option
+ (int list * evaluable_global_reference) list -> hyp_location option
-> tactic
val reduce : red_expr -> hyp_location list -> tactic
val change : constr -> hyp_location list -> tactic