Additional lemmas about homomorphisms of semirings and rings #
These lemmas have been banished here to avoid unnecessary imports in
Mathlib.Algebra.Hom.Ring.Defs
.
They could be moved to more natural homes.
theorem
RingHom.codomain_trivial_iff_range_eq_singleton_zero
{α : Type u_1}
{β : Type u_2}
{x✝ : NonAssocSemiring α}
{x✝¹ : NonAssocSemiring β}
(f : α →+* β)
:
f : α →+* β
has a trivial codomain iff its range is {0}
.
theorem
Function.Injective.isDomain
{α : Type u_1}
{β : Type u_2}
[Semiring α]
[IsDomain α]
[Semiring β]
{F : Type u_3}
[FunLike F β α]
[MonoidWithZeroHomClass F β α]
(f : F)
(hf : Function.Injective ⇑f)
:
IsDomain β
Pullback IsDomain
instance along an injective function.