The circle #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines circle to be the metric sphere (metric.sphere) in ℂ centred at 0 of
radius 1.  We equip it with the following structure:
- a submonoid of ℂ
- a group
- a topological group
We furthermore define exp_map_circle to be the natural map λ t, exp (t * I) from ℝ to
circle, and show that this map is a group homomorphism.
Implementation notes #
Because later (in geometry.manifold.instances.sphere) one wants to equip the circle with a smooth
manifold structure borrowed from metric.sphere, the underlying set is
{z : ℂ | abs (z - 0) = 1}.  This prevents certain algebraic facts from working definitionally --
for example, the circle is not defeq to {z : ℂ | abs z = 1}, which is the kernel of complex.abs
considered as a homomorphism from ℂ to ℝ, nor is it defeq to {z : ℂ | norm_sq z = 1}, which
is the kernel of the homomorphism complex.norm_sq from ℂ to ℝ.
The unit circle in ℂ, here given the structure of a submonoid of ℂ.
Equations
Instances for ↥circle
        - circle.comm_group
- circle.compact_space
- circle.topological_group
- pontryagin_dual.circle.continuous_monoid_hom_class
- complex.unit_disc.circle_action
- complex.unit_disc.is_scalar_tower_circle_circle
- complex.unit_disc.is_scalar_tower_circle
- complex.unit_disc.smul_comm_class_circle
- complex.unit_disc.smul_comm_class_circle'
- complex.unit_disc.smul_comm_class_circle_closed_ball
- complex.unit_disc.smul_comm_class_closed_ball_circle
- circle.charted_space
- circle.smooth_manifold_with_corners
- circle.lie_group
Equations
The elements of the circle embed into the units.
Equations
If z is a nonzero complex number, then conj z / z belongs to the unit circle.
Equations
- circle.of_conj_div_self z hz = ⟨⇑(star_ring_end ℂ) z / z, _⟩
The map λ t, exp (t * I) from ℝ to the unit circle in ℂ, considered as a homomorphism of
groups.