aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/cc.v
diff options
context:
space:
mode:
authorGravatar Pierre Corbineau <Pierre.Corbineau@NOSPAM@imag.fr>2014-12-16 15:59:35 +0100
committerGravatar Pierre Corbineau <Pierre.Corbineau@NOSPAM@imag.fr>2014-12-16 15:59:35 +0100
commitd4f5bdd6f7304fac541bb5f4555ecdd6aa42699a (patch)
treebef50df694a7188a35a298fe2a5b4633e83fc24b /test-suite/success/cc.v
parent8bda62e798c4e89c8c3f9406327899e394f7be0f (diff)
fix bug #2447 in congruence
Diffstat (limited to 'test-suite/success/cc.v')
-rw-r--r--test-suite/success/cc.v27
1 files changed, 27 insertions, 0 deletions
diff --git a/test-suite/success/cc.v b/test-suite/success/cc.v
index b565183b9..a70d91963 100644
--- a/test-suite/success/cc.v
+++ b/test-suite/success/cc.v
@@ -102,5 +102,32 @@ Proof.
auto.
Qed.
+(* bug 2447 is now closed (PC, 2014) *)
+
+Section bug_2447.
+
+Variable T:Type.
+
+Record R := mkR {x:T;y:T;z:T}.
+
+Variables a a' b b' c c':T.
+
+
+
+Lemma bug_2447: mkR a b c = mkR a' b c -> a = a'.
+congruence.
+Qed.
+
+Lemma bug_2447_variant1: mkR a b c = mkR a b' c -> b = b'.
+congruence.
+Qed.
+
+Lemma bug_2447_variant2: mkR a b c = mkR a b c' -> c = c'.
+congruence.
+Qed.
+
+
+End bug_2447.
+