Skip to content

Commit fe6b078

Browse files
committed
[Cos_rel] drop dependency on Lra
lra, nra -> field,ring
1 parent 79e9edc commit fe6b078

File tree

1 file changed

+4
-4
lines changed

1 file changed

+4
-4
lines changed

theories/Reals/Cos_rel.v

+4-4
Original file line numberDiff line numberDiff line change
@@ -12,7 +12,7 @@ From Stdlib Require Import Rbase.
1212
From Stdlib Require Import Rfunctions.
1313
From Stdlib Require Import SeqSeries.
1414
From Stdlib Require Import Rtrigo_def.
15-
From Stdlib Require Import Lia Lra.
15+
From Stdlib Require Import Lia.
1616
From Stdlib Require Import Arith.Factorial.
1717
Local Open Scope R_scope.
1818

@@ -77,7 +77,7 @@ replace
7777
y ^ (2 * (S n - l)))) (pred (S n - k))) (
7878
pred (S n))) with (Reste1 x y (S n)).
7979
2:{ unfold Reste1; apply sum_eq; intros.
80-
apply sum_eq; intros. nra. }
80+
apply sum_eq; intros. ring. }
8181
replace
8282
(sum_f_R0
8383
(fun k:nat =>
@@ -89,7 +89,7 @@ replace
8989
y ^ (2 * (n - l) + 1))) (pred (n - k))) (
9090
pred n)) with (Reste2 x y n).
9191
2:{ unfold Reste2; apply sum_eq; intros.
92-
apply sum_eq; intros. nra. }
92+
apply sum_eq; intros. ring. }
9393
replace
9494
(sum_f_R0
9595
(fun k:nat =>
@@ -153,7 +153,7 @@ replace
153153
unfold C1.
154154
apply sum_eq; intros.
155155
induction i as [| i Hreci].
156-
{ unfold C; simpl. nra. }
156+
{ unfold C; simpl. field. }
157157
unfold sin_nnn.
158158
rewrite <- Rmult_plus_distr_l.
159159
apply Rmult_eq_compat_l.

0 commit comments

Comments
 (0)