aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/cc.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-03-05 18:23:05 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-03-05 20:50:24 +0100
commiteb0feed6d22c11c44e7091c64ce5b1c9d5af987a (patch)
tree317c806bf3f55ff2ab0673cb9ce85f8fc40a7482 /test-suite/success/cc.v
parentc6d6e27330f0a1c9e89b6b60953d4df757edfdb8 (diff)
Using build_selector from Equality as a replacement of the selector
in cctac which does not support indices properly. Incidentally, this should fix a failure in RelationAlgebra, where making prod_applist more robust (e8c47b652) revealed the discriminate bug in congruence.
Diffstat (limited to 'test-suite/success/cc.v')
-rw-r--r--test-suite/success/cc.v7
1 files changed, 6 insertions, 1 deletions
diff --git a/test-suite/success/cc.v b/test-suite/success/cc.v
index a70d91963..dc0527d82 100644
--- a/test-suite/success/cc.v
+++ b/test-suite/success/cc.v
@@ -129,5 +129,10 @@ Qed.
End bug_2447.
+(* congruence was supposed to do discriminate but it was bugged for
+ types with indices *)
-
+Inductive I : nat -> Type := C : I 0 | D : I 0.
+Goal ~C=D.
+congruence.
+Qed.