Skip to content

Commit

Permalink
refining type classes constraints
Browse files Browse the repository at this point in the history
  • Loading branch information
jtristan committed Jun 4, 2024
1 parent 66e51de commit c6d5c46
Showing 1 changed file with 13 additions and 1 deletion.
14 changes: 13 additions & 1 deletion SampCert/Util/Shift.lean
Original file line number Diff line number Diff line change
Expand Up @@ -13,10 +13,14 @@ import Mathlib.Topology.Algebra.InfiniteSum.NatInt
This file contains lemmas about invariance of sums under integer shifts.
-/

variable {M : Type*} [AddCommGroup M] [UniformSpace M] [T2Space M] [UniformAddGroup M] [CompleteSpace M] {m m' : M}
variable {M : Type*} {m m' : M}

open Summable

section A

variable [AddCommGroup M] [UniformSpace M] [T2Space M] [UniformAddGroup M]

/--
A series is right-ℕ-shift-invariant provided its shifted positive and negative parts are summable.
-/
Expand Down Expand Up @@ -116,6 +120,12 @@ theorem tsum_shift₂ (f : ℤ → M) (μ : ℕ)
. exact (h2 μ)
. exact (h3 μ)

end A

section B

variable [AddCommGroup M] [UniformSpace M] [T2Space M] [UniformAddGroup M] [CompleteSpace M]

/--
A series is invariant under integer shifts provided its shifted positive and negative parts are summable.
-/
Expand Down Expand Up @@ -157,3 +167,5 @@ theorem tsum_shift (f : ℤ → M) (μ : ℤ)
apply tsum_congr
intro b
congr

end B

0 comments on commit c6d5c46

Please sign in to comment.