Skip to content

Commit

Permalink
Update Mathlib/Topology/Algebra/Module/Basic.lean
Browse files Browse the repository at this point in the history
Co-authored-by: Eric Wieser <[email protected]>
  • Loading branch information
kbuzzard and eric-wieser authored Oct 15, 2024
1 parent 88d1ec6 commit 533b2be
Showing 1 changed file with 1 addition and 0 deletions.
1 change: 1 addition & 0 deletions Mathlib/Topology/Algebra/Module/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2407,6 +2407,7 @@ variable (R : Type*) [Semiring R] [τR : TopologicalSpace R] [TopologicalSemirin
{M : Type*} [AddCommMonoid M] [Module R M] [TopologicalSpace M] [ContinuousSMul R M]

/-- The function `op` is a continuous linear equivalence. -/
@[simps!]
def opContinuousLinearEquiv : M ≃L[R] Mᵐᵒᵖ where
__ := MulOpposite.opLinearEquiv R

Expand Down

0 comments on commit 533b2be

Please sign in to comment.