aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-10-18 15:49:24 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-10-18 15:49:24 +0000
commit4decf9451f8fad147e884f244b9472d539ac6ee6 (patch)
tree71260c9b2dec46f6ece78f1aebc73883c84d25a8 /test-suite/success
parent862a01d7cfc5c3073a81d38557f9861877e61cca (diff)
- Merge modifs coq_makefile.ml4 de la 8.1 vers le trunk (commit 11429)
- Makefile: typo apparente avec .ml4.preprocessed - test-suite: ajout d'un test sur eta qui trainait dans le coin git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11465 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success')
-rw-r--r--test-suite/success/apply.v13
1 files changed, 13 insertions, 0 deletions
diff --git a/test-suite/success/apply.v b/test-suite/success/apply.v
index fcce68b91..8c9712e97 100644
--- a/test-suite/success/apply.v
+++ b/test-suite/success/apply.v
@@ -201,3 +201,16 @@ Axiom silly_axiom : forall v : exp, v = v -> False.
Lemma silly_lemma : forall x : atom, False.
intros x.
apply silly_axiom with (v := x). (* fails *)
+reflexivity.
+Qed.
+
+(* Check that unification does not commit too early to a representative
+ of an eta-equivalence class that would be incompatible with other
+ unification constraints *)
+
+Lemma eta : forall f : (forall P, P 1),
+ (forall P, f P = f P) ->
+ forall Q, f (fun x => Q x) = f (fun x => Q x).
+intros.
+apply H.
+Qed.