aboutsummaryrefslogtreecommitdiff
path: root/test-suite/micromega/zify.v
diff options
context:
space:
mode:
authorVincent Laporte2021-04-19 13:22:05 +0200
committerVincent Laporte2021-04-19 13:22:05 +0200
commitb53642ec813178fedd3e646832e7c033b8163f52 (patch)
treee93f364cec8238a4f95ebbe48e84dda5606eea07 /test-suite/micromega/zify.v
parentf82dd4e968d1b948f4288687cb9458ec90b66270 (diff)
parentd2c7022f0e16e6037c0d8c30c837abaad2c8194f (diff)
Merge PR #14108: [zify] bugfix
Reviewed-by: Zimmi48 Reviewed-by: vbgl
Diffstat (limited to 'test-suite/micromega/zify.v')
-rw-r--r--test-suite/micromega/zify.v7
1 files changed, 7 insertions, 0 deletions
diff --git a/test-suite/micromega/zify.v b/test-suite/micromega/zify.v
index a12623c3c0..2ea320047d 100644
--- a/test-suite/micromega/zify.v
+++ b/test-suite/micromega/zify.v
@@ -167,6 +167,12 @@ Goal @zero znat = 0%nat.
reflexivity.
Qed.
+Require Import ZifyBool.
+Instance Op_bool_inj : UnOp (inj : bool -> bool) :=
+ { TUOp := id; TUOpInj := fun _ => eq_refl }.
+Add Zify UnOp Op_bool_inj.
+
+
Goal forall (x y : positive) (F : forall (P: Pos.le x y) , positive) (P : Pos.le x y),
(F P + 1 = 1 + F P)%positive.
Proof.
@@ -228,6 +234,7 @@ Proof.
intros. lia.
Qed.
+
Ltac Zify.zify_pre_hook ::= unfold is_true in *.
Goal forall x y : nat, is_true (Nat.eqb x 1) ->