Trigonometric functions #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Main definitions #
This file contains the definition of π
.
See also analysis.special_functions.trigonometric.inverse
and
analysis.special_functions.trigonometric.arctan
for the inverse trigonometric functions.
See also analysis.special_functions.complex.arg
and
analysis.special_functions.complex.log
for the complex argument function
and the complex logarithm.
Main statements #
Many basic inequalities on the real trigonometric functions are established.
The continuity of the usual trigonometric functions is proved.
Several facts about the real trigonometric functions have the proofs deferred to
analysis.special_functions.trigonometric.complex
,
as they are most easily proved by appealing to the corresponding fact for
complex trigonometric functions.
See also analysis.special_functions.trigonometric.chebyshev
for the multiple angle formulas
in terms of Chebyshev polynomials.
Tags #
sin, cos, tan, angle
The number π = 3.14159265... Defined here using choice as twice a zero of cos in [1,2], from
which one can derive all its properties. For explicit bounds on π, see data.real.pi.bounds
.
Equations
the series sqrt_two_add_series x n
is sqrt(2 + sqrt(2 + ... ))
with n
square roots,
starting with x
. We define it here because cos (pi / 2 ^ (n+1)) = sqrt_two_add_series 0 n / 2
Equations
- real.sqrt_two_add_series x (n + 1) = √ (2 + real.sqrt_two_add_series x n)
- real.sqrt_two_add_series x 0 = x
real.sin
as an order_iso
between [-(π / 2), π / 2]
and [-1, 1]
.
A supporting lemma for the Phragmen-Lindelöf principle in a horizontal strip. If z : ℂ
belongs to a horizontal strip |complex.im z| ≤ b
, b ≤ π / 2
, and a ≤ 0
, then
$$\left|exp^{a\left(e^{z}+e^{-z}\right)}\right| \le e^{a\cos b \exp^{|re z|}}.$$