aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2017-05-03 19:44:56 +0200
committerGravatar Maxime Dénès <mail@maximedenes.fr>2017-05-03 19:44:56 +0200
commit773d95f915996b581b7ea82d9193197649c951a0 (patch)
tree63b1e5f68e830a538871b2edf0257303707b4671 /test-suite
parent14a50277b58eae50f14f7dea965dec7f8bc416a3 (diff)
parentedb21eab674b170d125a5b6fbc8213066b356d17 (diff)
Merge PR#541: Fixing "decide equality" bug #5449
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/bugs/closed/5449.v6
1 files changed, 6 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/5449.v b/test-suite/bugs/closed/5449.v
new file mode 100644
index 000000000..d7fc2aaa0
--- /dev/null
+++ b/test-suite/bugs/closed/5449.v
@@ -0,0 +1,6 @@
+(* An example of decide equality which was failing due to a lhs dep into the rhs *)
+
+Require Import Coq.PArith.BinPos.
+Goal forall x y, {Pos.compare_cont Gt x y = Gt} + {Pos.compare_cont Gt x y <> Gt}.
+intros.
+decide equality.