aboutsummaryrefslogtreecommitdiff
path: root/test-suite/micromega/zify.v
diff options
context:
space:
mode:
authorFrederic Besson2021-04-12 21:02:51 +0200
committerBESSON Frederic2021-04-16 23:53:38 +0200
commitd2c7022f0e16e6037c0d8c30c837abaad2c8194f (patch)
treea3df49a4565d69c2f288b479240878a741ce5ab2 /test-suite/micromega/zify.v
parentb78e6cfcb412d1c4e5902fb895c5ecaa0cb177ac (diff)
[zify] bugfix
- to zify the conclusion, we are using Tactics.apply (not rewrite) Closes #11089 - constrain the arguments of Add Zify X to be GlobRef.t Unset Primitive Projections so that projections are GlobRef.t. Closes #14043 Update doc/sphinx/addendum/micromega.rst Co-authored-by: Théo Zimmermann <theo.zimmi@gmail.com>
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) ->