aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/unification.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-06-13 22:21:33 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-06-13 22:21:33 +0000
commit981ece2836d6366f3dad790c21350feb24b036af (patch)
treec3045de235e39a7d5e9a90d291b643c03e601ab4 /test-suite/success/unification.v
parentd5b1c83d0f0a60f9658c45ae902035f2fdef0c41 (diff)
Added full pattern-unification on Meta for tactic unification.
No way to control it yet; maybe flag use_evars_pattern_unification should be generalized for that purpose. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14199 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/unification.v')
-rw-r--r--test-suite/success/unification.v7
1 files changed, 7 insertions, 0 deletions
diff --git a/test-suite/success/unification.v b/test-suite/success/unification.v
index 18ba0fc87..fdc7c7222 100644
--- a/test-suite/success/unification.v
+++ b/test-suite/success/unification.v
@@ -21,6 +21,12 @@ Proof.
intros; apply H.
Qed.
+ (* Feature introduced June 2011 *)
+
+Lemma l7 : forall x (P:nat->Prop), (forall f, P (f x)) -> P (x+x).
+Proof.
+intros x P H; apply H.
+Qed.
(* Example submitted for Zenon *)
@@ -138,3 +144,4 @@ Goal (forall (A B : Set) (f : A -> B), (fun x => f x) = f) ->
Proof.
intros.
rewrite H with (f:=f0).
+Abort.