Skip to content

Commit

Permalink
chore: another non-class instance (#7250)
Browse files Browse the repository at this point in the history
Following #7245, https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/isClass.3F.20panic!/near/391779504.

There is one exception that it is unclear how to fix, it seems lean makes the internal declarations in a block of mutual instances also instances perhaps? Seeing as it is internal I hope it won't cause too much trouble
  • Loading branch information
alexjbest committed Sep 20, 2023
1 parent 14b1439 commit a2b2bcf
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean
Expand Up @@ -120,7 +120,7 @@ theorem restrictScalars.smul_def' {R : Type u₁} {S : Type u₂} [Ring R] [Ring

instance (priority := 100) sMulCommClass_mk {R : Type u₁} {S : Type u₂} [Ring R] [CommRing S]
(f : R →+* S) (M : Type v) [I : AddCommGroup M] [Module S M] :
have : SMul R M := (RestrictScalars.obj' f (ModuleCat.mk M)).isModule.toSMul
haveI : SMul R M := (RestrictScalars.obj' f (ModuleCat.mk M)).isModule.toSMul
SMulCommClass R S M :=
-- Porting note: cannot synth SMul R M
have : SMul R M := (RestrictScalars.obj' f (ModuleCat.mk M)).isModule.toSMul
Expand Down

0 comments on commit a2b2bcf

Please sign in to comment.