aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics/hipattern.mli
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-11-29 16:30:00 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-02-14 17:30:44 +0100
commitd549d9d3d169fbfc5f555e3e4f22f46301161d53 (patch)
tree4cb4052135639414c1f46e3f61a2064ed74d94eb /tactics/hipattern.mli
parent4e9cebb0641927f11a21cbb50828974f910cfe47 (diff)
Do not ask for a normalized goal to get hypotheses and conclusions.
This is now useless as this returns evar-constrs, so that all functions acting on them should be insensitive to evar-normalization.
Diffstat (limited to 'tactics/hipattern.mli')
-rw-r--r--tactics/hipattern.mli6
1 files changed, 3 insertions, 3 deletions
diff --git a/tactics/hipattern.mli b/tactics/hipattern.mli
index 65ba0aad0..c46817f50 100644
--- a/tactics/hipattern.mli
+++ b/tactics/hipattern.mli
@@ -121,11 +121,11 @@ val match_with_equation:
(** Match terms [eq A t u], [identity A t u] or [JMeq A t A u]
Returns associated lemmas and [A,t,u] or fails PatternMatchingFailure *)
-val find_eq_data_decompose : ([ `NF ], 'r) Proofview.Goal.t -> constr ->
+val find_eq_data_decompose : ('a, 'r) Proofview.Goal.t -> constr ->
coq_eq_data * Univ.universe_instance * (types * constr * constr)
(** Idem but fails with an error message instead of PatternMatchingFailure *)
-val find_this_eq_data_decompose : ([ `NF ], 'r) Proofview.Goal.t -> constr ->
+val find_this_eq_data_decompose : ('a, 'r) Proofview.Goal.t -> constr ->
coq_eq_data * Univ.universe_instance * (types * constr * constr)
(** A variant that returns more informative structure on the equality found *)
@@ -146,7 +146,7 @@ val is_matching_sigma : evar_map -> constr -> bool
val match_eqdec : evar_map -> constr -> bool * constr * constr * constr * constr
(** Match an equality up to conversion; returns [(eq,t1,t2)] in normal form *)
-val dest_nf_eq : ([ `NF ], 'r) Proofview.Goal.t -> constr -> (constr * constr * constr)
+val dest_nf_eq : ('a, 'r) Proofview.Goal.t -> constr -> (constr * constr * constr)
(** Match a negation *)
val is_matching_not : evar_map -> constr -> bool