Documentation

Mathlib.Algebra.Divisibility.Hom

Mapping divisibility across multiplication-preserving homomorphisms #

Main definitions #

Tags #

divisibility, divides

theorem map_dvd {M : Type u_1} {N : Type u_2} [Semigroup M] [Semigroup N] {F : Type u_3} [FunLike F M N] [MulHomClass F M N] (f : F) {a b : M} :
a bf a f b
theorem MulHom.map_dvd {M : Type u_1} {N : Type u_2} [Semigroup M] [Semigroup N] (f : M →ₙ* N) {a b : M} :
a bf a f b
theorem MonoidHom.map_dvd {M : Type u_1} {N : Type u_2} [Monoid M] [Monoid N] (f : M →* N) {a b : M} :
a bf a f b