File tree Expand file tree Collapse file tree 1 file changed +0
-2
lines changed Expand file tree Collapse file tree 1 file changed +0
-2
lines changed Original file line number Diff line number Diff line change @@ -248,7 +248,6 @@ end FieldDivisionRing
248248end algebraMap
249249
250250/-- Creating an algebra from a morphism to the center of a semiring. -/
251- @[reducible]
252251def RingHom.toAlgebra' {R S} [CommSemiring R] [Semiring S] (i : R →+* S)
253252 (h : ∀ c x, i c * x = x * i c) : Algebra R S where
254253 smul c x := i c * x
@@ -258,7 +257,6 @@ def RingHom.toAlgebra' {R S} [CommSemiring R] [Semiring S] (i : R →+* S)
258257#align ring_hom.to_algebra' RingHom.toAlgebra'
259258
260259/-- Creating an algebra from a morphism to a commutative semiring. -/
261- @[reducible]
262260def RingHom.toAlgebra {R S} [CommSemiring R] [CommSemiring S] (i : R →+* S) : Algebra R S :=
263261 i.toAlgebra' fun _ => mul_comm _
264262#align ring_hom.to_algebra RingHom.toAlgebra
You can’t perform that action at this time.
0 commit comments