aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/fourier/Fourier_util.v
diff options
context:
space:
mode:
authorGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2013-12-03 16:43:14 +0100
committerGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2013-12-03 16:43:14 +0100
commit943133d5a47ce4663a9b77a03b36c7c87c78d886 (patch)
tree6321ab6fab78b5fb723310096be3eaba9ce753a1 /plugins/fourier/Fourier_util.v
parentaca9c227772e3765833605866ac413e61a98d04a (diff)
Fix statement of Rplus_lt_reg_r and add Rplus_lt_reg_l.
Diffstat (limited to 'plugins/fourier/Fourier_util.v')
-rw-r--r--plugins/fourier/Fourier_util.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/plugins/fourier/Fourier_util.v b/plugins/fourier/Fourier_util.v
index b10c304c8..3ab7ad84a 100644
--- a/plugins/fourier/Fourier_util.v
+++ b/plugins/fourier/Fourier_util.v
@@ -164,7 +164,7 @@ Qed.
Lemma Rnot_lt_lt : forall x y:R, ~ 0 < y - x -> ~ x < y.
unfold not; intros.
apply H.
-apply Rplus_lt_reg_r with x.
+apply Rplus_lt_reg_l with x.
replace (x + 0) with x.
replace (x + (y - x)) with y.
try exact H0.
@@ -177,7 +177,7 @@ unfold not; intros.
apply H.
case H0; intros.
left.
-apply Rplus_lt_reg_r with x.
+apply Rplus_lt_reg_l with x.
replace (x + 0) with x.
replace (x + (y - x)) with y.
try exact H1.