Skip to content

Commit ae4ed02

Browse files
committed
feat(Topology/Algebra/InfiniteSum/NatInt): Add pnat lems (#16544)
Add some basic results about tsums indexed by pnat. Co-authored-by: Chris Birkbeck <c.birkbeck@uea.ac.uk>
1 parent e58d5d7 commit ae4ed02

File tree

1 file changed

+13
-0
lines changed

1 file changed

+13
-0
lines changed

Mathlib/Topology/Algebra/InfiniteSum/NatInt.lean

Lines changed: 13 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -514,3 +514,16 @@ lemma multipliable_int_iff_multipliable_nat_and_neg {f : ℤ → G} :
514514
end UniformGroup
515515

516516
end Int
517+
518+
section pnat
519+
520+
@[to_additive]
521+
theorem pnat_multipliable_iff_multipliable_succ {α : Type*} [TopologicalSpace α] [CommMonoid α]
522+
{f : ℕ → α} : Multipliable (fun x : ℕ+ => f x) ↔ Multipliable fun x : ℕ => f (x + 1) :=
523+
Equiv.pnatEquivNat.symm.multipliable_iff.symm
524+
525+
@[to_additive]
526+
theorem tprod_pnat_eq_tprod_succ {α : Type*} [TopologicalSpace α] [CommMonoid α] (f : ℕ → α) :
527+
∏' n : ℕ+, f n = ∏' n, f (n + 1) := (Equiv.pnatEquivNat.symm.tprod_eq _).symm
528+
529+
end pnat

0 commit comments

Comments
 (0)