aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/5697.v
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-08-28 01:07:07 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-08-29 17:20:40 +0200
commit5fb53743cc14047b4be12c188c21c6f679bdbd8f (patch)
treef81997dfa6d64829e204335c1e63d8a47f29fecd /test-suite/bugs/closed/5697.v
parenta980d38681f7ab9bfd8a180f2252ce573e3ff211 (diff)
Fix BZ#5697: Congruence does not work with primitive projections.
The code generating the projection was unconditionally generating pattern-matchings, although this is incorrect for primitive records.
Diffstat (limited to 'test-suite/bugs/closed/5697.v')
-rw-r--r--test-suite/bugs/closed/5697.v10
1 files changed, 10 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/5697.v b/test-suite/bugs/closed/5697.v
new file mode 100644
index 000000000..a17229aaf
--- /dev/null
+++ b/test-suite/bugs/closed/5697.v
@@ -0,0 +1,10 @@
+Set Primitive Projections.
+
+Record foo : Type := Foo { foo_car: nat }.
+
+Goal forall x y : nat, x <> y -> Foo x <> Foo y.
+Proof.
+intros.
+intros H'.
+congruence.
+Qed.