Documentation

SpherePacking.ModularForms.multipliable_lems

theorem Complex.summable_nat_multipliable_one_add (f : ) (hf : Summable f) :
Multipliable fun (n : ) => 1 + f n
theorem term_ne_zero (z : UpperHalfPlane) (n : ) :
1 - Complex.exp (2 * Real.pi * Complex.I * (n + 1) * z) 0
theorem ball_pow_ne_1 (x : ) (hx : x Metric.ball 0 1) (n : ) :
1 + (fun (n : ) => -x ^ (n + 1)) n 0
theorem multipliable_lt_one (x : ) (hx : x Metric.ball 0 1) :
Multipliable fun (i : ) => 1 - x ^ (i + 1)
theorem tprod_ne_zero (x : UpperHalfPlane) (f : UpperHalfPlane) (hf : ∀ (i : ) (x : UpperHalfPlane), 1 + f i x 0) (hu : ∀ (x : UpperHalfPlane), Summable fun (n : ) => f n x) :
∏' (i : ), (1 + f i) x 0
theorem Multipliable_pow {ι : Type u_1} (f : ι) (hf : Multipliable f) (n : ) :
Multipliable fun (i : ι) => f i ^ n
theorem tprod_pow (f : ) (hf : Multipliable f) (n : ) :
(∏' (i : ), f i) ^ n = ∏' (i : ), f i ^ n
theorem hasProd_le_nonneg {a₁ a₂ : } {ι : Type u_1} (f g : ι) (h : ∀ (i : ι), f i g i) (h0 : ∀ (i : ι), 0 f i) (hf : HasProd f a₁) (hg : HasProd g a₂) :
a₁ a₂
theorem hasSum_le_nonneg {a₁ a₂ : } {ι : Type u_1} (f g : ι) (h : ∀ (i : ι), f i g i) (h0 : ∀ (i : ι), 0 f i) (hf : HasProd f a₁) (hg : HasProd g a₂) :
a₁ a₂
theorem HasProd.le_one_nonneg {a : } (g : ) (h : ∀ (i : ), g i 1) (h0 : ∀ (i : ), 0 g i) (ha : HasProd g a) :
a 1
theorem HasSum.nonpos_nonneg {a : } (g : ) (h : ∀ (i : ), g i 1) (h0 : ∀ (i : ), 0 g i) (ha : HasProd g a) :
a 1
theorem one_le_tprod_nonneg (g : ) (h : ∀ (i : ), g i 1) (h0 : ∀ (i : ), 0 g i) :
∏' (i : ), g i 1
theorem nonneg_tsum_nonneg (g : ) (h : ∀ (i : ), g i 1) (h0 : ∀ (i : ), 0 g i) :
∏' (i : ), g i 1