Skip to content

Commit

Permalink
doc(tactic/core,uniform_space/basic): minor doc fixes (#3115)
Browse files Browse the repository at this point in the history
Co-authored-by: Rob Lewis <rob.y.lewis@gmail.com>
  • Loading branch information
robertylewis and robertylewis committed Jun 19, 2020
1 parent 8e44b9f commit 103743e
Show file tree
Hide file tree
Showing 2 changed files with 5 additions and 3 deletions.
2 changes: 1 addition & 1 deletion src/tactic/core.lean
Expand Up @@ -1915,7 +1915,7 @@ do e ← pformat_macro () s,

reserve prefix `trace! `:100
/--
The combination of `pformat` and `fail`.
The combination of `pformat` and `trace`.
-/
@[user_notation]
meta def trace_macro (_ : parse $ tk "trace!") (s : string) : parser pexpr :=
Expand Down
6 changes: 4 additions & 2 deletions src/topology/uniform_space/basic.lean
Expand Up @@ -29,8 +29,10 @@ Those examples are generalizations in two different directions of the elementary
`X = ℝ` and `V ∈ 𝓤 ℝ ↔ ∃ ε > 0, { p | |p.2 - p.1| < ε } ⊆ V` which features both the topological
group structure on `ℝ` and its metric space structure.
Each uniform structure on `X` induces a topology on `X` characterized by:
Each uniform structure on `X` induces a topology on `X` characterized by
> `nhds_eq_comap_uniformity : ∀ {x : X}, 𝓝 x = comap (prod.mk x) (𝓤 X)`
where `prod.mk x : X → X × X := (λ y, (x, y))` is the partial evaluation of the product
constructor.
Expand Down Expand Up @@ -206,7 +208,7 @@ lemma uniform_space.core_eq : ∀{u₁ u₂ : uniform_space.core α}, u₁.unifo

section prio

/-- Suppose that one can put two mathematical structures on a type, a rich one `R` and a poor one
/-- Suppose that one can put two mathematical structures on a type, a rich one `R` and a poor one
`P`, and that one can deduce the poor structure from the rich structure through a map `F` (called a
forgetful functor) (think `R = metric_space` and `P = topological_space`). A possible
implementation would be to have a type class `rich` containing a field `R`, a type class `poor`
Expand Down

0 comments on commit 103743e

Please sign in to comment.