Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 97c4d4e

Browse files
committed
feat(analysis/asymptotics/asymptotics): add is_O.exists_mem_basis (#13973)
1 parent d989305 commit 97c4d4e

File tree

1 file changed

+6
-0
lines changed

1 file changed

+6
-0
lines changed

src/analysis/asymptotics/asymptotics.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -177,6 +177,12 @@ is_O_iff_is_O_with.trans
177177
lemma is_O_iff_eventually : is_O f g' l ↔ ∀ᶠ c in at_top, ∀ᶠ x in l, ∥f x∥ ≤ c * ∥g' x∥ :=
178178
is_O_iff_eventually_is_O_with.trans $ by simp only [is_O_with]
179179

180+
lemma is_O.exists_mem_basis {ι} {p : ι → Prop} {s : ι → set α} (h : is_O f g' l)
181+
(hb : l.has_basis p s) :
182+
∃ (c : ℝ) (hc : 0 < c) (i : ι) (hi : p i), ∀ x ∈ s i, ∥f x∥ ≤ c * ∥g' x∥ :=
183+
flip Exists₂.imp h.exists_pos $ λ c hc h,
184+
by simpa only [is_O_with_iff, hb.eventually_iff, exists_prop] using h
185+
180186
/-! ### Subsingleton -/
181187

182188
@[nontriviality] lemma is_o_of_subsingleton [subsingleton E'] : is_o f' g' l :=

0 commit comments

Comments
 (0)