Skip to content

Commit

Permalink
chore(Normed.Group.BallSphere): address porting notes (#10510)
Browse files Browse the repository at this point in the history
There are no longer timeouts in typeclass synthesis.
  • Loading branch information
mattrobball committed Feb 14, 2024
1 parent 052755a commit 088de1d
Showing 1 changed file with 3 additions and 9 deletions.
12 changes: 3 additions & 9 deletions Mathlib/Analysis/Normed/Group/BallSphere.lean
Expand Up @@ -30,10 +30,8 @@ theorem coe_neg_sphere {r : ℝ} (v : sphere (0 : E) r) : ↑(-v) = (-v : E) :=
rfl
#align coe_neg_sphere coe_neg_sphere

-- porting note: todo: need to specify instance to avoid timeout
instance : ContinuousNeg (sphere (0 : E) r) :=
@Inducing.continuousNeg (sphere (0 : E) r) E _ _ _ _ TopologicalAddGroup.toContinuousNeg
Subtype.val inducing_subtype_val fun _ => rfl
Inducing.continuousNeg inducing_subtype_val fun _ => rfl

/-- We equip the ball, in a seminormed group, with a formal operation of negation, namely the
antipodal map. -/
Expand All @@ -44,10 +42,8 @@ instance {r : ℝ} : InvolutiveNeg (ball (0 : E) r) where
@[simp] theorem coe_neg_ball {r : ℝ} (v : ball (0 : E) r) : ↑(-v) = (-v : E) := rfl
#align coe_neg_ball coe_neg_ball

-- porting note: todo: need to specify instance to avoid timeout
instance : ContinuousNeg (ball (0 : E) r) :=
@Inducing.continuousNeg (ball (0 : E) r) E _ _ _ _ TopologicalAddGroup.toContinuousNeg
Subtype.val inducing_subtype_val fun _ => rfl
Inducing.continuousNeg inducing_subtype_val fun _ => rfl

/-- We equip the closed ball, in a seminormed group, with a formal operation of negation, namely the
antipodal map. -/
Expand All @@ -58,7 +54,5 @@ instance {r : ℝ} : InvolutiveNeg (closedBall (0 : E) r) where
@[simp] theorem coe_neg_closedBall {r : ℝ} (v : closedBall (0 : E) r) : ↑(-v) = (-v : E) := rfl
#align coe_neg_closed_ball coe_neg_closedBall

-- porting note: todo: need to specify instance to avoid timeout
instance : ContinuousNeg (closedBall (0 : E) r) :=
@Inducing.continuousNeg (closedBall (0 : E) r) E _ _ _ _ TopologicalAddGroup.toContinuousNeg
Subtype.val inducing_subtype_val fun _ => rfl
Inducing.continuousNeg inducing_subtype_val fun _ => rfl

0 comments on commit 088de1d

Please sign in to comment.