aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/tacticals.mli
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-03-26 17:05:20 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-03-26 17:51:41 +0100
commitfd2ab327c8d30f129fac3c882b73f4bd4e31a128 (patch)
tree3505b6ddb83c58bee018c850ee37888d645b64b0 /tactics/tacticals.mli
parentaa7c872724e0d9bb79520152d613085c92d67236 (diff)
Removing tactic compatibility layer from Inv.
Diffstat (limited to 'tactics/tacticals.mli')
-rw-r--r--tactics/tacticals.mli4
1 files changed, 4 insertions, 0 deletions
diff --git a/tactics/tacticals.mli b/tactics/tacticals.mli
index 3e6e64ecb..ceaa6f27c 100644
--- a/tactics/tacticals.mli
+++ b/tactics/tacticals.mli
@@ -188,6 +188,7 @@ module New : sig
Ltac error with level more than 0. Otherwise succeeds. *)
val catch_failerror : exn -> unit tactic
+ val tclIDTAC : unit tactic
val tclTHEN : unit tactic -> unit tactic -> unit tactic
(* [tclFAIL n msg] fails with [msg] as an error message at level [n]
(meaning that it will jump over [n] error catching tacticals FROM
@@ -239,6 +240,7 @@ module New : sig
val tclTIMEOUT : int -> unit tactic -> unit tactic
+ val nLastDecls : int -> (named_context -> unit tactic) -> unit tactic
val ifOnHyp : (identifier * types -> bool) ->
(identifier -> unit Proofview.tactic) -> (identifier -> unit Proofview.tactic) ->
@@ -249,6 +251,8 @@ module New : sig
val onLastHyp : (constr -> unit tactic) -> unit tactic
val onLastDecl : (named_declaration -> unit tactic) -> unit tactic
+ val afterHyp : Id.t -> (named_context -> unit tactic) -> unit tactic
+
val tryAllHyps : (identifier -> unit tactic) -> unit tactic
val tryAllHypsAndConcl : (identifier option -> unit tactic) -> unit tactic
val onClause : (identifier option -> unit tactic) -> clause -> unit tactic