Skip to content

Commit

Permalink
fix: CompatibleSMul : Prop (#6065)
Browse files Browse the repository at this point in the history
Lean makes it `Type` otherwise. Why does this happen? Am I missing something?
  • Loading branch information
kbuzzard committed Jul 23, 2023
1 parent 560eeb2 commit 641f7a7
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Module/LinearMap.lean
Expand Up @@ -399,7 +399,7 @@ we can also add an instance for `AddCommGroup.intModule`, allowing `z •` to be
`R` does not support negation.
-/
class CompatibleSMul (R S : Type _) [Semiring S] [SMul R M] [Module S M] [SMul R M₂]
[Module S M₂] where
[Module S M₂] : Prop where
/-- Scalar multiplication by `R` of `M` can be moved through linear maps. -/
map_smul : ∀ (fₗ : M →ₗ[S] M₂) (c : R) (x : M), fₗ (c • x) = c • fₗ x
#align linear_map.compatible_smul LinearMap.CompatibleSMul
Expand Down

0 comments on commit 641f7a7

Please sign in to comment.