File tree Expand file tree Collapse file tree 1 file changed +3
-3
lines changed Expand file tree Collapse file tree 1 file changed +3
-3
lines changed Original file line number Diff line number Diff line change @@ -885,19 +885,19 @@ theorem sin_pos_of_pos_of_le_two {x : ℝ} (hx0 : 0 < x) (hx : x ≤ 2) : 0 < si
885
885
(cos_pos_of_le_one (by rwa [abs_of_nonneg (le_of_lt (half_pos hx0))]))
886
886
_ = sin x := by rw [← sin_two_mul, two_mul, add_halves]
887
887
888
- theorem cos_one_le : cos 1 ≤ 2 / 3 :=
888
+ theorem cos_one_le : cos 1 ≤ 5 / 9 :=
889
889
calc
890
890
cos 1 ≤ |(1 : ℝ)| ^ 4 * (5 / 96 ) + (1 - 1 ^ 2 / 2 ) :=
891
891
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
893
893
894
894
theorem cos_one_pos : 0 < cos 1 :=
895
895
cos_pos_of_le_one (le_of_eq abs_one)
896
896
897
897
theorem cos_two_neg : cos 2 < 0 :=
898
898
calc cos 2 = cos (2 * 1 ) := congr_arg cos (mul_one _).symm
899
899
_ = _ := Real.cos_two_mul 1
900
- _ ≤ 2 * (2 / 3 ) ^ 2 - 1 := by
900
+ _ ≤ 2 * (5 / 9 ) ^ 2 - 1 := by
901
901
gcongr
902
902
· exact cos_one_pos.le
903
903
· apply cos_one_le
You can’t perform that action at this time.
0 commit comments