Skip to content

Commit

Permalink
doc(order/filter/small_sets): fix in doc (#13648)
Browse files Browse the repository at this point in the history
  • Loading branch information
fpvandoorn committed Apr 28, 2022
1 parent c096a33 commit 220d4b8
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions src/order/filter/small_sets.lean
Expand Up @@ -13,9 +13,9 @@ containing all powersets of members of `f`.
`g` converges to `f.small_sets` if for all `s ∈ f`, eventually we have `g x ⊆ s`.
An example usage is that if `f : ι → ℝ` is a family of nonnegative functions with integral 1, then
saying that `f` tendsto `(𝓝 0).small_sets` is a way of saying that `f` tends to the Dirac delta
distribution.
An example usage is that if `f : ι → E → ℝ` is a family of nonnegative functions with integral 1,
then saying that `λ i, support (f i)` tendsto `(𝓝 0).small_sets` is a way of saying that
`f` tends to the Dirac delta distribution.
-/

open_locale filter
Expand Down

0 comments on commit 220d4b8

Please sign in to comment.