aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/inv.mli
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-08-15 17:43:35 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-08-18 18:56:39 +0200
commit5dcafa956e49eefc451dd021a0fe8ad2e2338088 (patch)
treec851c0f1cb32815bae652309c39f6d4a681fd2cc /tactics/inv.mli
parent72498d6d68ac12ba4db0db7d54f0ac6fdaaf0c61 (diff)
Lazy interpretation of patterns so that expressions such as "intros H H'/H"
can be given with second H bound by the first one. Not very satisfied by passing closure to tactics.ml, but otherwise tactics would have to be aware of glob_constr.
Diffstat (limited to 'tactics/inv.mli')
-rw-r--r--tactics/inv.mli6
1 files changed, 3 insertions, 3 deletions
diff --git a/tactics/inv.mli b/tactics/inv.mli
index a71b5eeb3..c730716d8 100644
--- a/tactics/inv.mli
+++ b/tactics/inv.mli
@@ -15,14 +15,14 @@ open Tacexpr
type inversion_status = Dep of constr option | NoDep
val inv_clause :
- inversion_kind -> constr or_and_intro_pattern_expr located option -> Id.t list ->
+ inversion_kind -> or_and_intro_pattern option -> Id.t list ->
quantified_hypothesis -> unit Proofview.tactic
-val inv : inversion_kind -> constr or_and_intro_pattern_expr located option ->
+val inv : inversion_kind -> or_and_intro_pattern option ->
quantified_hypothesis -> unit Proofview.tactic
val dinv : inversion_kind -> constr option ->
- constr or_and_intro_pattern_expr located option -> quantified_hypothesis -> unit Proofview.tactic
+ or_and_intro_pattern option -> quantified_hypothesis -> unit Proofview.tactic
val inv_tac : Id.t -> unit Proofview.tactic
val inv_clear_tac : Id.t -> unit Proofview.tactic