aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Ratan.v
diff options
context:
space:
mode:
authorGravatar Guillaume Melquiond <guillaume.melquiond@inria.fr>2017-03-05 21:50:19 +0100
committerGravatar Maxime Dénès <mail@maximedenes.fr>2017-03-22 17:56:02 +0100
commit4e6fa17a3ef0b8d12cb8d55305f302338589ad1c (patch)
treeb6ed89f849f9423c9a2b3bee42bd8b9f5b176305 /theories/Reals/Ratan.v
parentd6ced637d9b7acabef2ccc9e761ec149bc7c93da (diff)
Make IZR a morphism for field.
There are now two field structures for R: one in RealField and one in RIneq. The first one is used to prove that IZR is a morphism which is needed to define the second one.
Diffstat (limited to 'theories/Reals/Ratan.v')
-rw-r--r--theories/Reals/Ratan.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/theories/Reals/Ratan.v b/theories/Reals/Ratan.v
index 3e5362efe..e438750df 100644
--- a/theories/Reals/Ratan.v
+++ b/theories/Reals/Ratan.v
@@ -319,10 +319,10 @@ apply PI2_lower_bound;[split; fourier | ].
destruct (pre_cos_bound (3/2) 1) as [t _]; [fourier | fourier | ].
apply Rlt_le_trans with (2 := t); clear t.
unfold cos_approx; simpl; unfold cos_term.
-unfold INR.
+rewrite !INR_IZR_INZ.
simpl.
field_simplify.
-change (0 */ 1 < 9925632 / 141557760).
+unfold Rdiv.
rewrite Rmult_0_l.
apply Rdiv_lt_0_compat ; now apply IZR_lt.
Qed.