aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/equality.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/equality.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/equality.mli')
-rw-r--r--tactics/equality.mli3
1 files changed, 0 insertions, 3 deletions
diff --git a/tactics/equality.mli b/tactics/equality.mli
index 9008af77b..5ac4fccb8 100644
--- a/tactics/equality.mli
+++ b/tactics/equality.mli
@@ -60,9 +60,6 @@ val general_rewrite_in :
val general_rewrite_clause :
orientation -> evars_flag -> ?tac:(unit Proofview.tactic * conditions) -> constr with_bindings -> clause -> unit Proofview.tactic
-type delayed_open_constr_with_bindings =
- env -> evar_map -> evar_map * constr with_bindings
-
val general_multi_rewrite :
evars_flag -> (bool * multi * clear_flag * delayed_open_constr_with_bindings) list ->
clause -> (unit Proofview.tactic * conditions) option -> unit Proofview.tactic