aboutsummaryrefslogtreecommitdiff
path: root/test-suite
diff options
context:
space:
mode:
authorFrédéric Besson2020-04-30 10:03:46 +0200
committerFrédéric Besson2020-04-30 14:46:57 +0200
commit5d514890669296e5d25a342c15aa930595f3af10 (patch)
treeb4eb670f22ec51187f2243ce3ffed1f59d1fe24f /test-suite
parentd436c45a19de2f91aad94f492b547225f8c5b305 (diff)
[zify] add support for Nat.le, Nat.lt and Nat.eq
Nat.le, Nat.lt and Nat.eq are aliased to le, lt and @eq nat. The required declarations are now added in ZifyInst.
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/micromega/bug_12210.v19
1 files changed, 19 insertions, 0 deletions
diff --git a/test-suite/micromega/bug_12210.v b/test-suite/micromega/bug_12210.v
new file mode 100644
index 0000000000..ca011def09
--- /dev/null
+++ b/test-suite/micromega/bug_12210.v
@@ -0,0 +1,19 @@
+Require Import PeanoNat Lia.
+
+Goal forall x, Nat.le x x.
+Proof.
+intros.
+lia.
+Qed.
+
+Goal forall x, Nat.lt x x -> False.
+Proof.
+intros.
+lia.
+Qed.
+
+Goal forall x, Nat.eq x x.
+Proof.
+intros.
+lia.
+Qed.