aboutsummaryrefslogtreecommitdiff
path: root/test-suite/micromega
diff options
context:
space:
mode:
authorFrédéric Besson2019-12-09 15:28:14 +0100
committerMaxime Dénès2019-12-17 11:14:21 +0100
commit7d961a914a8eaa889a982a4f84b3ba368d9e8ebc (patch)
treeff057865c1656b2c2db45f25f4f3fb08b15103c0 /test-suite/micromega
parent82918ec41ccab3b1623e41139b448938f4760a80 (diff)
[micromega] fix efficiency regression
PR #9725 fixes completness bugs introduces some inefficiency. The current PR intends to fix the inefficiency while retaining completness. The fix removes a pre-processing step and instead relies on a more elaborate proof format introducing positivity constraints on the fly. Solve bootstrapping issues: RMicromega <-> Rbase <-> lia. Fixes #11063 and fixes #11242 and fixes #11270
Diffstat (limited to 'test-suite/micromega')
-rw-r--r--test-suite/micromega/bug_11270.v6
1 files changed, 6 insertions, 0 deletions
diff --git a/test-suite/micromega/bug_11270.v b/test-suite/micromega/bug_11270.v
new file mode 100644
index 0000000000..80abc6d0e9
--- /dev/null
+++ b/test-suite/micromega/bug_11270.v
@@ -0,0 +1,6 @@
+Require Import Psatz.
+Theorem foo : forall a b, 1 <= S (a + a * S b).
+Proof.
+intros.
+lia.
+Qed.