aboutsummaryrefslogtreecommitdiff
path: root/test-suite/micromega/bug_12184.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/micromega/bug_12184.v')
-rw-r--r--test-suite/micromega/bug_12184.v8
1 files changed, 8 insertions, 0 deletions
diff --git a/test-suite/micromega/bug_12184.v b/test-suite/micromega/bug_12184.v
new file mode 100644
index 0000000000..d329a3fa7f
--- /dev/null
+++ b/test-suite/micromega/bug_12184.v
@@ -0,0 +1,8 @@
+Require Import Lia.
+Require Import ZArith.
+
+Goal forall p : positive, (0 < Z.pos (2^p)%positive)%Z.
+Proof.
+ intros p.
+ lia.
+Qed.