Skip to content

Commit

Permalink
isometry induced
Browse files Browse the repository at this point in the history
  • Loading branch information
winstonyin committed Jan 14, 2025
1 parent 9c0bf76 commit 503c53b
Showing 1 changed file with 12 additions and 0 deletions.
12 changes: 12 additions & 0 deletions Mathlib/Topology/MetricSpace/Isometry.lean
Original file line number Diff line number Diff line change
Expand Up @@ -258,6 +258,18 @@ theorem Topology.IsEmbedding.to_isometry {α β} [TopologicalSpace α] [MetricSp
@[deprecated (since := "2024-10-26")]
alias Embedding.to_isometry := IsEmbedding.to_isometry

theorem PseudoEMetricSpace.isometry_induced (f : α → β) [m : PseudoEMetricSpace β] :
letI := m.induced f; Isometry f := fun _ _ ↦ rfl

theorem PsuedoMetricSpace.isometry_induced (f : α → β) [m : PseudoMetricSpace β] :
letI := m.induced f; Isometry f := fun _ _ ↦ rfl

theorem EMetricSpace.isometry_induced (f : α → β) (hf : f.Injective) [m : EMetricSpace β] :
letI := m.induced f hf; Isometry f := fun _ _ ↦ rfl

theorem MetricSpace.isometry_induced (f : α → β) (hf : f.Injective) [m : MetricSpace β] :
letI := m.induced f hf; Isometry f := fun _ _ ↦ rfl

-- such a bijection need not exist
/-- `α` and `β` are isometric if there is an isometric bijection between them. -/
-- Porting note (https://github.com/leanprover-community/mathlib4/issues/5171): was @[nolint has_nonempty_instance]
Expand Down

0 comments on commit 503c53b

Please sign in to comment.