Skip to content

Commit

Permalink
feat(analysis/asymptotics/asymptotics): add is_O.exists_mem_basis (#…
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed May 6, 2022
1 parent d989305 commit 97c4d4e
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions src/analysis/asymptotics/asymptotics.lean
Expand Up @@ -177,6 +177,12 @@ is_O_iff_is_O_with.trans
lemma is_O_iff_eventually : is_O f g' l ↔ ∀ᶠ c in at_top, ∀ᶠ x in l, ∥f x∥ ≤ c * ∥g' x∥ :=
is_O_iff_eventually_is_O_with.trans $ by simp only [is_O_with]

lemma is_O.exists_mem_basis {ι} {p : ι → Prop} {s : ι → set α} (h : is_O f g' l)
(hb : l.has_basis p s) :
∃ (c : ℝ) (hc : 0 < c) (i : ι) (hi : p i), ∀ x ∈ s i, ∥f x∥ ≤ c * ∥g' x∥ :=
flip Exists₂.imp h.exists_pos $ λ c hc h,
by simpa only [is_O_with_iff, hb.eventually_iff, exists_prop] using h

/-! ### Subsingleton -/

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

0 comments on commit 97c4d4e

Please sign in to comment.