aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/opened/4717.v
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2016-11-17 10:27:36 +0100
committerGravatar Maxime Dénès <mail@maximedenes.fr>2016-11-17 10:27:36 +0100
commitca9e00ff9b2a8ee17430398a5e0bef2345c39341 (patch)
tree1f35be33dcc6ca7117bb85db4415d6f728b80641 /test-suite/bugs/opened/4717.v
parent63bb79ab8b488db728e46e5ada38d86d384acff1 (diff)
parent633ed9c528c64dc2daa0b3e83749bc392aab7fd2 (diff)
Merge commit '633ed9c' into v8.6
Was PR#192: Add test suite files for 4700-4785
Diffstat (limited to 'test-suite/bugs/opened/4717.v')
-rw-r--r--test-suite/bugs/opened/4717.v19
1 files changed, 19 insertions, 0 deletions
diff --git a/test-suite/bugs/opened/4717.v b/test-suite/bugs/opened/4717.v
new file mode 100644
index 000000000..9ad474672
--- /dev/null
+++ b/test-suite/bugs/opened/4717.v
@@ -0,0 +1,19 @@
+(*See below. They sometimes work, and sometimes do not. Is this a bug?*)
+
+Require Import Omega Psatz.
+
+Definition foo := nat.
+
+Goal forall (n : foo), 0 = n - n.
+Proof. intros. omega. (* works *) Qed.
+
+Goal forall (x n : foo), x = x + n - n.
+Proof.
+ intros.
+ Fail omega. (* Omega can't solve this system *)
+ Fail lia. (* Cannot find witness. *)
+ unfold foo in *.
+ omega. (* works *)
+Qed.
+
+(* Guillaume Melquiond: What matters is the equality. In the first case, it is @eq nat. In the second case, it is @eq foo. The same issue exists for ring and field. So it is not a bug, but it is worth fixing.*)