Skip to content

Commit 36a0240

Browse files
committed
feat(Data/Complex/Trigonometric): closer upper bound for cos 1 (#22945)
cos 1 is approximately 0.5403..., so this bound is fairly tight. Co-authored-by: Vlad Tsyrklevich <vlad@tsyrklevich.net>
1 parent 3a94488 commit 36a0240

File tree

1 file changed

+3
-3
lines changed

1 file changed

+3
-3
lines changed

Mathlib/Data/Complex/Trigonometric.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -885,19 +885,19 @@ theorem sin_pos_of_pos_of_le_two {x : ℝ} (hx0 : 0 < x) (hx : x ≤ 2) : 0 < si
885885
(cos_pos_of_le_one (by rwa [abs_of_nonneg (le_of_lt (half_pos hx0))]))
886886
_ = sin x := by rw [← sin_two_mul, two_mul, add_halves]
887887

888-
theorem cos_one_le : cos 12 / 3 :=
888+
theorem cos_one_le : cos 15 / 9 :=
889889
calc
890890
cos 1 ≤ |(1 : ℝ)| ^ 4 * (5 / 96) + (1 - 1 ^ 2 / 2) :=
891891
sub_le_iff_le_add.1 (abs_sub_le_iff.1 (cos_bound (by simp))).1
892-
_ ≤ 2 / 3 := by norm_num
892+
_ ≤ 5 / 9 := by norm_num
893893

894894
theorem cos_one_pos : 0 < cos 1 :=
895895
cos_pos_of_le_one (le_of_eq abs_one)
896896

897897
theorem cos_two_neg : cos 2 < 0 :=
898898
calc cos 2 = cos (2 * 1) := congr_arg cos (mul_one _).symm
899899
_ = _ := Real.cos_two_mul 1
900-
_ ≤ 2 * (2 / 3) ^ 2 - 1 := by
900+
_ ≤ 2 * (5 / 9) ^ 2 - 1 := by
901901
gcongr
902902
· exact cos_one_pos.le
903903
· apply cos_one_le

0 commit comments

Comments
 (0)