diff options
author | Matthieu Sozeau <matthieu.sozeau@inria.fr> | 2014-09-17 20:51:40 +0200 |
---|---|---|
committer | Matthieu Sozeau <matthieu.sozeau@inria.fr> | 2014-09-17 20:51:40 +0200 |
commit | f96dc97f48df5d0fdf252be5f28478a58be77961 (patch) | |
tree | 5d741e02de71083b5e279121721dff7cb4b56516 /test-suite | |
parent | 17f68d403d248e899efbb76afeed169232946ecf (diff) |
Fix bug #3593, making constr_eq and progress work up to
equality of universes, along with a few other functions in evd.
Diffstat (limited to 'test-suite')
-rw-r--r-- | test-suite/bugs/closed/3593.v | 10 |
1 files changed, 10 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3593.v b/test-suite/bugs/closed/3593.v new file mode 100644 index 000000000..25f9db6b2 --- /dev/null +++ b/test-suite/bugs/closed/3593.v @@ -0,0 +1,10 @@ +Set Universe Polymorphism. +Set Printing All. +Set Implicit Arguments. +Record prod A B := pair { fst : A ; snd : B }. +Goal forall x : prod Set Set, let f := @fst _ in f _ x = @fst _ _ x. +simpl; intros. + constr_eq (@fst Set Set x) (fst (A := Set) (B := Set) x). + Fail progress change (@fst Set Set x) with (fst (A := Set) (B := Set) x). + reflexivity. +Qed. |