aboutsummaryrefslogtreecommitdiff
path: root/test-suite
diff options
context:
space:
mode:
authorVincent Laporte2021-01-07 09:58:51 +0100
committerVincent Laporte2021-01-07 09:58:51 +0100
commitad9fdf76897ada659dc1ca6d2d931452f6361f93 (patch)
tree2fa1044833d278136f6c706b9453ef7be41bc3a6 /test-suite
parent30f497eaf34f2cf641c3fe854fc9066ae19eea67 (diff)
parentac64cad9e6c0496afc600380d5c21fd1129db400 (diff)
Merge PR #13715: [micromega] Add missing support for `implb`
Reviewed-by: vbgl
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/micromega/reify_bool.v18
1 files changed, 18 insertions, 0 deletions
diff --git a/test-suite/micromega/reify_bool.v b/test-suite/micromega/reify_bool.v
new file mode 100644
index 0000000000..501fafc0b3
--- /dev/null
+++ b/test-suite/micromega/reify_bool.v
@@ -0,0 +1,18 @@
+Require Import ZArith.
+Require Import Lia.
+Import Z.
+Unset Lia Cache.
+
+Goal forall (x y : Z),
+ implb (Z.eqb x y) (Z.eqb y x) = true.
+Proof.
+ intros.
+ lia.
+Qed.
+
+Goal forall (x y :Z), implb (Z.eqb x 0) (Z.eqb y 0) = true <->
+ orb (negb (Z.eqb x 0))(Z.eqb y 0) = true.
+Proof.
+ intro.
+ lia.
+Qed.