File tree Expand file tree Collapse file tree 1 file changed +6
-2
lines changed Expand file tree Collapse file tree 1 file changed +6
-2
lines changed Original file line number Diff line number Diff line change @@ -247,7 +247,9 @@ end FieldDivisionRing
247247
248248end algebraMap
249249
250- /-- Creating an algebra from a morphism to the center of a semiring. -/
250+ /-- Creating an algebra from a morphism to the center of a semiring.
251+ See note [reducible non-instances]. -/
252+ @[reducible]
251253def RingHom.toAlgebra' {R S} [CommSemiring R] [Semiring S] (i : R →+* S)
252254 (h : ∀ c x, i c * x = x * i c) : Algebra R S where
253255 smul c x := i c * x
@@ -256,7 +258,9 @@ def RingHom.toAlgebra' {R S} [CommSemiring R] [Semiring S] (i : R →+* S)
256258 toRingHom := i
257259#align ring_hom.to_algebra' RingHom.toAlgebra'
258260
259- /-- Creating an algebra from a morphism to a commutative semiring. -/
261+ /-- Creating an algebra from a morphism to a commutative semiring.
262+ See note [reducible non-instances]. -/
263+ @[reducible]
260264def RingHom.toAlgebra {R S} [CommSemiring R] [CommSemiring S] (i : R →+* S) : Algebra R S :=
261265 i.toAlgebra' fun _ => mul_comm _
262266#align ring_hom.to_algebra RingHom.toAlgebra
You can’t perform that action at this time.
0 commit comments