aboutsummaryrefslogtreecommitdiff
path: root/tactics/hipattern.mli
diff options
context:
space:
mode:
authorherbelin2009-08-04 12:12:50 +0000
committerherbelin2009-08-04 12:12:50 +0000
commita42d753ac38896e58158311b3c384e80c9fd3fd4 (patch)
treee4f2cc05245d61b546956555d64a415ac420605e /tactics/hipattern.mli
parentf9f35dc36f5249a2de18005ab59ae934e0fa7075 (diff)
Fixed subst failing when a truly heterogeneous JMeq hyp is in the
context (problem introduced in r12259) + improved backward compatibility in hippatern.mli (wrt r12259). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12260 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics/hipattern.mli')
-rw-r--r--tactics/hipattern.mli14
1 files changed, 11 insertions, 3 deletions
diff --git a/tactics/hipattern.mli b/tactics/hipattern.mli
index 5be8b20264..3f5411e00f 100644
--- a/tactics/hipattern.mli
+++ b/tactics/hipattern.mli
@@ -123,9 +123,17 @@ val match_with_equation:
(***** Destructing patterns bound to some theory *)
-(* Match terms [(eq A t u)] or [(identity A t u)] *)
-(* Returns associated lemmas and [A,t,u] *)
-val find_eq_data_decompose : constr -> coq_eq_data * equation_kind
+(* 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 : Proof_type.goal sigma -> constr ->
+ coq_eq_data * (types * constr * constr)
+
+(* Idem but fails with an error message instead of PatternMatchingFailure *)
+val find_this_eq_data_decompose : Proof_type.goal sigma -> constr ->
+ coq_eq_data * (types * constr * constr)
+
+(* A variant that returns more informative structure on the equality found *)
+val find_eq_data : constr -> coq_eq_data * equation_kind
(* Match a term of the form [(existT A P t p)] *)
(* Returns associated lemmas and [A,P,t,p] *)