aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tactics.mli
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-06-12 15:04:06 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-06-12 15:20:36 +0200
commitbda7852cb0896727389935f420eec0e8e3315cf7 (patch)
treedc03858224a7dfbd3b92c0aee016356ab9dda6ce /tactics/tactics.mli
parenta4db087565dd2ecfa3bcc022277bed1a3c868fd3 (diff)
Passing some tactics to the new monad type.
Diffstat (limited to 'tactics/tactics.mli')
-rw-r--r--tactics/tactics.mli6
1 files changed, 3 insertions, 3 deletions
diff --git a/tactics/tactics.mli b/tactics/tactics.mli
index c1911819b..6574d88c5 100644
--- a/tactics/tactics.mli
+++ b/tactics/tactics.mli
@@ -45,8 +45,8 @@ val fix : Id.t option -> int -> tactic
val mutual_cofix : Id.t -> (Id.t * constr) list -> int -> tactic
val cofix : Id.t option -> tactic
-val convert : constr -> constr -> tactic
-val convert_leq : constr -> constr -> tactic
+val convert : constr -> constr -> unit Proofview.tactic
+val convert_leq : constr -> constr -> unit Proofview.tactic
(** {6 Introduction tactics. } *)
@@ -110,7 +110,7 @@ val intros_pattern_bound :
val assumption : unit Proofview.tactic
val exact_no_check : constr -> tactic
val vm_cast_no_check : constr -> tactic
-val exact_check : constr -> tactic
+val exact_check : constr -> unit Proofview.tactic
val exact_proof : Constrexpr.constr_expr -> tactic
(** {6 Reduction tactics. } *)