aboutsummaryrefslogtreecommitdiff
path: root/test-suite/micromega/bug_11089.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/bug_11089.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/bug_11089.v')
-rw-r--r--test-suite/micromega/bug_11089.v13
1 files changed, 13 insertions, 0 deletions
diff --git a/test-suite/micromega/bug_11089.v b/test-suite/micromega/bug_11089.v
new file mode 100644
index 0000000000..e62b5b8d9e
--- /dev/null
+++ b/test-suite/micromega/bug_11089.v
@@ -0,0 +1,13 @@
+Require Import Lia.
+Unset Lia Cache.
+Definition t := nat.
+Goal forall (n : t), n = n.
+Proof.
+ intros.
+ lia.
+Qed.
+Goal let t' := nat in forall (n : t'), n = n.
+Proof.
+ intros.
+ lia.
+Qed.