Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit c50a60d

Browse files
committed
feat(analysis/convex/specific_functions): sin is strictly concave (#11688)
1 parent 92c64c4 commit c50a60d

File tree

1 file changed

+18
-0
lines changed

1 file changed

+18
-0
lines changed

src/analysis/convex/specific_functions.lean

Lines changed: 18 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -214,3 +214,21 @@ begin
214214
rw [deriv_log', deriv_inv],
215215
exact neg_neg_of_pos (inv_pos.2 $ sq_pos_of_ne_zero _ hx.ne),
216216
end
217+
218+
open_locale real
219+
220+
lemma strict_concave_on_sin_Icc : strict_concave_on ℝ (Icc 0 π) sin :=
221+
begin
222+
apply strict_concave_on_of_deriv2_neg (convex_Icc _ _) continuous_on_sin
223+
differentiable_sin.differentiable_on (λ x hx, _),
224+
rw interior_Icc at hx,
225+
simp [sin_pos_of_mem_Ioo hx],
226+
end
227+
228+
lemma strict_concave_on_cos_Icc : strict_concave_on ℝ (Icc (-(π/2)) (π/2)) cos :=
229+
begin
230+
apply strict_concave_on_of_deriv2_neg (convex_Icc _ _) continuous_on_cos
231+
differentiable_cos.differentiable_on (λ x hx, _),
232+
rw interior_Icc at hx,
233+
simp [cos_pos_of_mem_Ioo hx],
234+
end

0 commit comments

Comments
 (0)