Documentation

Mathlib.Algebra.Regular.Pow

Product of regular elements #

TODO #

Move to Mathlib.Algebra.BigOperators.Group.Finset.Basic?

theorem IsLeftRegular.prod {ι : Type u_2} {R : Type u_3} [CommMonoid R] {s : Finset ι} {f : ιR} (h : is, IsLeftRegular (f i)) :
IsLeftRegular (∏ is, f i)
theorem IsRightRegular.prod {ι : Type u_2} {R : Type u_3} [CommMonoid R] {s : Finset ι} {f : ιR} (h : is, IsRightRegular (f i)) :
IsRightRegular (∏ is, f i)
theorem IsRegular.prod {ι : Type u_2} {R : Type u_3} [CommMonoid R] {s : Finset ι} {f : ιR} (h : is, IsRegular (f i)) :
IsRegular (∏ is, f i)