aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2018-06-22 13:45:03 +0200
committerGravatar Maxime Dénès <mail@maximedenes.fr>2018-07-17 14:15:59 +0200
commit8c43e795c772090b336c0f170a6e5dcab196125d (patch)
tree98508f7e342142dd017da56872f74df73e6fce58 /test-suite/success
parentb799252775563b4f46f5ea39cbfc469759e7a296 (diff)
Remove fourier plugin
As stated in the manual, the fourier tactic is subsumed by lra.
Diffstat (limited to 'test-suite/success')
-rw-r--r--test-suite/success/LraTest.v (renamed from test-suite/success/Fourier.v)10
1 files changed, 6 insertions, 4 deletions
diff --git a/test-suite/success/Fourier.v b/test-suite/success/LraTest.v
index b63bead47..bf3a87da2 100644
--- a/test-suite/success/Fourier.v
+++ b/test-suite/success/LraTest.v
@@ -1,12 +1,14 @@
-Require Import Rfunctions.
-Require Import Fourier.
+Require Import Reals.
+Require Import Lra.
+
+Open Scope R_scope.
Lemma l1 : forall x y z : R, Rabs (x - z) <= Rabs (x - y) + Rabs (y - z).
-intros; split_Rabs; fourier.
+intros; split_Rabs; lra.
Qed.
Lemma l2 :
forall x y : R, x < Rabs y -> y < 1 -> x >= 0 -> - y <= 1 -> Rabs x <= 1.
intros.
-split_Rabs; fourier.
+split_Rabs; lra.
Qed.