Skip to content

Commit d5addf3

Browse files
committed
add missing docstring
1 parent 082b030 commit d5addf3

File tree

1 file changed

+2
-0
lines changed

1 file changed

+2
-0
lines changed

Mathlib/Dynamics/BirkhoffSum/Maximal.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -190,6 +190,8 @@ lemma birkhoffSupSet_eq_iSup_birkhoffMax_support {f : α → α} {g : α → ℝ
190190
rcases exists_partialSups_eq (birkhoffSum f g · x) n with ⟨m, _, hm₂⟩
191191
exact ⟨m, hm₂ ▸ h⟩
192192

193+
/-- The set of `x` for which `birkhoffAverage ℝ f g n x` greater than some `a`
194+
for at least one value of `n`. -/
193195
public def birkhoffAverageSupSet (f : α → α) (g : α → ℝ) (a : ℝ) : Set α :=
194196
{x | ∃ n : ℕ, a < birkhoffAverage ℝ f g n x}
195197

0 commit comments

Comments
 (0)