Skip to content

Commit

Permalink
chore: WithLp inherits decidable equality (#22250)
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed Feb 24, 2025
1 parent 69f2481 commit 4ea41dd
Showing 1 changed file with 1 addition and 0 deletions.
1 change: 1 addition & 0 deletions Mathlib/Analysis/Normed/Lp/WithLp.lean
Original file line number Diff line number Diff line change
Expand Up @@ -56,6 +56,7 @@ protected def equiv : WithLp p V ≃ V := Equiv.refl _

instance instNontrivial [Nontrivial V] : Nontrivial (WithLp p V) := ‹Nontrivial V›
instance instUnique [Unique V] : Unique (WithLp p V) := ‹Unique V›
instance instDecidableEq [DecidableEq V] : DecidableEq (WithLp p V) := ‹DecidableEq V›

variable [Semiring K] [Semiring K'] [AddCommGroup V]

Expand Down

0 comments on commit 4ea41dd

Please sign in to comment.