aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/refine.mli
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-12-06 12:12:48 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-05-03 20:05:57 +0200
commit3b57395029447119eea1fd399636cd9cfe3e673e (patch)
tree29ce6a8ddde295015124f69dcb26559969732d75 /proofs/refine.mli
parent9262f440e8d8b8559c5488b1333c023f7305d811 (diff)
Generalizing the refine primitive so as to accept tactic arguments.
Diffstat (limited to 'proofs/refine.mli')
-rw-r--r--proofs/refine.mli7
1 files changed, 6 insertions, 1 deletions
diff --git a/proofs/refine.mli b/proofs/refine.mli
index 1a254d578..1dcee3188 100644
--- a/proofs/refine.mli
+++ b/proofs/refine.mli
@@ -12,6 +12,7 @@
in Ltac which is actually based on the one below. *)
open Proofview
+open Proofview.Notations
(** {6 The refine tactic} *)
@@ -31,7 +32,11 @@ val refine : ?unsafe:bool -> EConstr.t Sigma.run -> unit tactic
type-checked beforehand. *)
val refine_one : ?unsafe:bool -> ('a * EConstr.t) Sigma.run -> 'a tactic
-(** A generalization of [refine] which assumes exactly one goal under focus *)
+(** A variant of [refine] which assumes exactly one goal under focus *)
+
+val generic_refine : ?unsafe:bool -> ('a * EConstr.t) tactic ->
+ ([ `NF ], 'r) Proofview.Goal.t -> 'a tactic
+(** The general version of refine. *)
(** {7 Helper functions} *)