Trigonometric functions
Main definitions
This file contains the following definitions:
- π, arcsin, arccos, arctan
- argument of a complex number
- logarithm on complex numbers
Main statements
Many basic inequalities on trigonometric functions are established.
The continuity and differentiability of the usual trigonometric functions are proved, and their derivatives are computed.
Tags
log, sin, cos, tan, arcsin, arccos, arctan, angle, argument
The complex sine function is everywhere differentiable, with the derivative cos x
.
The complex cosine function is everywhere differentiable, with the derivative -sin x
.
The complex hyperbolic sine function is everywhere differentiable, with the derivative cosh x
.
The complex hyperbolic cosine function is everywhere differentiable, with the derivative sinh x
.
Register lemmas for the derivatives of the composition of complex.cos
, complex.sin
,
complex.cosh
and complex.sinh
with a differentiable function, for standalone use and use with
simp
.
Register lemmas for the derivatives of the composition of real.exp
, real.cos
, real.sin
,
real.cosh
and real.sinh
with a differentiable function, for standalone use and use with
simp
.
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
.
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
- x.sqrt_two_add_series (n + 1) = real.sqrt (2 + x.sqrt_two_add_series n)
- x.sqrt_two_add_series 0 = x
The type of angles
Equations
Equations
- real.angle.inhabited = {default := 0}
Equations
Inverse of the sin
function, returns values in the range -π / 2 ≤ arcsin x
and arcsin x ≤ π / 2
.
If the argument is not between -1
and 1
it defaults to 0
arg
returns values in the range (-π, π], such that for x ≠ 0
,
sin (arg x) = x.im / x.abs
and cos (arg x) = x.re / x.abs
,
arg 0
defaults to 0
Continuity and differentiability of arctan
The continuity of arctan
is difficult to prove due to arctan
being (indirectly) defined naively
via classical.some
. The proof therefore uses the general theorem that monotone functions are
homeomorphisms: homeomorph_of_strict_mono_continuous_Ioo
. We first prove that tan
(restricted)
is a homeomorphism whose inverse is definitionally equal to arctan
. The fact that arctan
is
continuous is then derived from the fact that it is equal to a homeomorphism, and its
differentiability is in turn derived from its continuity using has_deriv_at.of_local_left_inverse
.
The function tan
, restricted to the open interval (-π/2, π/2), is a homeomorphism. The inverse
function of that homeomorphism is definitionally equal to arctan
via homeomorph.change_inv
.
Equations
- real.tan_homeomorph = (homeomorph_of_strict_mono_continuous_Ioo real.tan real.tan_homeomorph._proof_1 real.tan_homeomorph._proof_2 real.continuous_on_tan_Ioo real.tendsto_tan_pi_div_two real.tendsto_tan_neg_pi_div_two).change_inv (λ (x : ℝ), ⟨x.arctan, _⟩) real.tan_arctan
Register lemmas for the derivatives of the composition of real.arctan
with a differentiable
function, for standalone use and use with simp
.