aboutsummaryrefslogtreecommitdiff
path: root/test-suite
diff options
context:
space:
mode:
authorKazuhiko Sakaguchi2019-09-20 18:58:51 +0200
committerKazuhiko Sakaguchi2019-09-24 00:25:15 +0200
commite7b83e2a07fffaba0b19c62ef1a02c40d6ef603a (patch)
tree64daeb1e336ff86934cc5b529d9d6926ed8bfad8 /test-suite
parentdc690e7067aa91a05472b5d573cb463223ef4dec (diff)
Make `zify` does work for `Z.to_N`
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/micromega/bug_9162.v8
1 files changed, 8 insertions, 0 deletions
diff --git a/test-suite/micromega/bug_9162.v b/test-suite/micromega/bug_9162.v
new file mode 100644
index 0000000000..4aedf57faf
--- /dev/null
+++ b/test-suite/micromega/bug_9162.v
@@ -0,0 +1,8 @@
+Require Import ZArith Lia.
+Local Open Scope Z_scope.
+
+Goal Z.of_N (Z.to_N 0) = 0.
+Proof. lia. Qed.
+
+Goal forall q, (Z.of_N (Z.to_N 0) = 0 -> q = 0) -> Z.of_N (Z.to_N 0) = q.
+Proof. lia. Qed.