Skip to content

Commit

Permalink
Remove unnecessary assumptions
Browse files Browse the repository at this point in the history
  • Loading branch information
D-Thomine committed Oct 29, 2024
1 parent 00af82f commit 6a8142d
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Mathlib/Order/LiminfLimsup.lean
Original file line number Diff line number Diff line change
Expand Up @@ -345,12 +345,12 @@ lemma IsCoboundedUnder.frequently_le [LinearOrder α] {f : Filter ι} [NeBot f]
∃ a, ∃ᶠ x in f, u x ≤ a :=
IsCobounded.frequently_le h

lemma IsCoboundedUnder.of_frequently_ge [LinearOrder α] {f : Filter ι} [NeBot f] {u : ι → α}
lemma IsCoboundedUnder.of_frequently_ge [LinearOrder α] {f : Filter ι} {u : ι → α}
{a : α} (freq_ge : ∃ᶠ x in f, a ≤ u x) :
IsCoboundedUnder (· ≤ ·) f u :=
IsCobounded.of_frequently_ge freq_ge

lemma IsCoboundedUnder.of_frequently_le [LinearOrder α] {f : Filter ι} [NeBot f] {u : ι → α}
lemma IsCoboundedUnder.of_frequently_le [LinearOrder α] {f : Filter ι} {u : ι → α}
{a : α} (freq_le : ∃ᶠ x in f, u x ≤ a) :
IsCoboundedUnder (· ≥ ·) f u :=
IsCobounded.of_frequently_le freq_le
Expand Down

0 comments on commit 6a8142d

Please sign in to comment.