Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit b430316

Browse files
committed
chore(topology/algebra/module/basic): add continuous_linear_map.is_central_scalar (#11291)
1 parent 3b7a783 commit b430316

File tree

1 file changed

+3
-0
lines changed

1 file changed

+3
-0
lines changed

src/topology/algebra/module/basic.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1103,6 +1103,9 @@ variables [has_continuous_add M₂] [has_continuous_add M₃] [has_continuous_ad
11031103
instance : module S₃ (M →SL[σ₁₃] M₃) :=
11041104
{ zero_smul := λ _, ext $ λ _, zero_smul _ _,
11051105
add_smul := λ _ _ _, ext $ λ _, add_smul _ _ _ }
1106+
1107+
instance [module S₃ᵐᵒᵖ M₃] [is_central_scalar S₃ M₃] : is_central_scalar S₃ (M →SL[σ₁₃] M₃) :=
1108+
{ op_smul_eq_smul := λ _ _, ext $ λ _, op_smul_eq_smul _ _ }
11061109

11071110
variables (S) [has_continuous_add N₃]
11081111

0 commit comments

Comments
 (0)