Skip to content

Commit

Permalink
chore(MetricSpace.PseudoMetric): make `PseudoEMetricSpace.toPseudoMet…
Browse files Browse the repository at this point in the history
…ricSpaceOfDist` reducible (#10012)

`PseudoEMetricSpace.toPseudoMetricSpaceOfDist` is used in instances so needs to be reducible for unification.
  • Loading branch information
mattrobball committed Jan 26, 2024
1 parent f2b0b27 commit 4529fc1
Showing 1 changed file with 2 additions and 1 deletion.
3 changes: 2 additions & 1 deletion Mathlib/Topology/MetricSpace/PseudoMetric.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1274,7 +1274,8 @@ theorem PseudoMetricSpace.replaceTopology_eq {γ} [U : TopologicalSpace γ] (m :
is everywhere finite, by pushing the edistance to reals. We set it up so that the edist and the
uniformity are defeq in the pseudometric space and the pseudoemetric space. In this definition, the
distance is given separately, to be able to prescribe some expression which is not defeq to the
push-forward of the edistance to reals. -/
push-forward of the edistance to reals. See note [reducible non-instances]. -/
@[reducible]
def PseudoEMetricSpace.toPseudoMetricSpaceOfDist {α : Type u} [e : PseudoEMetricSpace α]
(dist : α → α → ℝ) (edist_ne_top : ∀ x y : α, edist x y ≠ ⊤)
(h : ∀ x y, dist x y = ENNReal.toReal (edist x y)) : PseudoMetricSpace α where
Expand Down

0 comments on commit 4529fc1

Please sign in to comment.