Products of lists of prime elements. #
This file contains some theorems relating prime
and products of list
s.
theorem
prime.dvd_prod_iff
{M : Type u_1}
[comm_monoid_with_zero M]
{p : M}
{L : list M}
(pp : prime p) :
Prime p
divides the product of a list L
iff it divides some a ∈ L
theorem
prime_dvd_prime_iff_eq
{M : Type u_1}
[cancel_comm_monoid_with_zero M]
[unique Mˣ]
{p q : M}
(pp : prime p)
(qp : prime q) :