We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 082b030 commit d5addf3Copy full SHA for d5addf3
Mathlib/Dynamics/BirkhoffSum/Maximal.lean
@@ -190,6 +190,8 @@ lemma birkhoffSupSet_eq_iSup_birkhoffMax_support {f : α → α} {g : α → ℝ
190
rcases exists_partialSups_eq (birkhoffSum f g · x) n with ⟨m, _, hm₂⟩
191
exact ⟨m, hm₂ ▸ h⟩
192
193
+/-- The set of `x` for which `birkhoffAverage ℝ f g n x` greater than some `a`
194
+for at least one value of `n`. -/
195
public def birkhoffAverageSupSet (f : α → α) (g : α → ℝ) (a : ℝ) : Set α :=
196
{x | ∃ n : ℕ, a < birkhoffAverage ℝ f g n x}
197
0 commit comments