Metric on the upper half-plane #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define a metric_space
structure on the upper_half_plane
. We use hyperbolic
(Poincaré) distance given by
dist z w = 2 * arsinh (dist (z : ℂ) w / (2 * real.sqrt (z.im * w.im)))
instead of the induced
Euclidean distance because the hyperbolic distance is invariant under holomorphic automorphisms of
the upper half-plane. However, we ensure that the projection to topological_space
is
definitionally equal to the induced topological space structure.
We also prove that a metric ball/closed ball/sphere in Poincaré metric is a Euclidean ball/closed ball/sphere with another center and radius.
Equations
- upper_half_plane.has_dist = {dist := λ (z w : upper_half_plane), 2 * real.arsinh (has_dist.dist ↑z ↑w / (2 * √ (z.im * w.im)))}
An auxiliary metric_space
instance on the upper half-plane. This instance has bad projection
to topological_space
. We replace it later.
Equations
- upper_half_plane.metric_space_aux = {to_pseudo_metric_space := {to_has_dist := {dist := has_dist.dist upper_half_plane.has_dist}, dist_self := upper_half_plane.metric_space_aux._proof_1, dist_comm := upper_half_plane.dist_comm, dist_triangle := upper_half_plane.dist_triangle, edist := λ (x y : upper_half_plane), ↑⟨has_dist.dist x y, _⟩, edist_dist := upper_half_plane.metric_space_aux._proof_3, to_uniform_space := uniform_space_of_dist has_dist.dist upper_half_plane.metric_space_aux._proof_4 upper_half_plane.dist_comm upper_half_plane.dist_triangle, uniformity_dist := upper_half_plane.metric_space_aux._proof_5, to_bornology := bornology.of_dist has_dist.dist upper_half_plane.metric_space_aux._proof_6 upper_half_plane.dist_comm upper_half_plane.dist_triangle, cobounded_sets := upper_half_plane.metric_space_aux._proof_7}, eq_of_dist_eq_zero := upper_half_plane.metric_space_aux._proof_8}
Euclidean center of the circle with center z
and radius r
in the hyperbolic metric.
For two points on the same vertical line, the distance is equal to the distance between the logarithms of their imaginary parts.
Hyperbolic distance between two points is greater than or equal to the distance between the logarithms of their imaginary parts.
An upper estimate on the complex distance between two points in terms of the hyperbolic distance and the imaginary part of one of the points.
An upper estimate on the complex distance between two points in terms of the hyperbolic distance and the imaginary part of one of the points.
The hyperbolic metric on the upper half plane. We ensure that the projection to
topological_space
is definitionally equal to the subtype topology.
Equations
- upper_half_plane.metric_space = upper_half_plane.metric_space_aux.replace_topology upper_half_plane.metric_space._proof_1
SL(2, ℝ)
acts on the upper half plane as an isometry.