aboutsummaryrefslogtreecommitdiff
path: root/test-suite
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
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')
-rw-r--r--test-suite/micromega/bug_11270.v6
-rw-r--r--test-suite/output/MExtraction.v5
2 files changed, 9 insertions, 2 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.
diff --git a/test-suite/output/MExtraction.v b/test-suite/output/MExtraction.v
index 668be1fdbc..357afb51eb 100644
--- a/test-suite/output/MExtraction.v
+++ b/test-suite/output/MExtraction.v
@@ -1,6 +1,6 @@
(************************************************************************)
(* * The Coq Proof Assistant / The Coq Development Team *)
-(* v * INRIA, CNRS and contributors - Copyright 1999-2018 *)
+(* v * INRIA, CNRS and contributors - Copyright 1999-2019 *)
(* <O___,, * (see CREDITS file for the list of authors) *)
(* \VV/ **************************************************************)
(* // * This file is distributed under the terms of the *)
@@ -56,10 +56,11 @@ Extract Constant Rinv => "fun x -> 1 / x".
Recursive Extraction
Tauto.mapX Tauto.foldA Tauto.collect_annot Tauto.ids_of_formula Tauto.map_bformula
Tauto.abst_form
- ZMicromega.cnfZ ZMicromega.bound_problem_fr ZMicromega.Zeval_const QMicromega.cnfQ
+ ZMicromega.cnfZ ZMicromega.Zeval_const QMicromega.cnfQ
List.map simpl_cone (*map_cone indexes*)
denorm Qpower vm_add
normZ normQ normQ n_of_Z N.of_nat ZTautoChecker ZWeakChecker QTautoChecker RTautoChecker find.
+
(* Local Variables: *)
(* coding: utf-8 *)
(* End: *)