Skip to content

Commit

Permalink
fix: Mathlib/Control/ULiftable doc typos (#6349)
Browse files Browse the repository at this point in the history
small typos in docstrings
  • Loading branch information
JamesGallicchio committed Aug 3, 2023
1 parent 32fa6fe commit 74ee5fb
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Mathlib/Control/ULiftable.lean
Expand Up @@ -48,7 +48,7 @@ class ULiftable (f : Type u₀ → Type u₁) (g : Type v₀ → Type v₁) wher

namespace ULiftable

/-- The most common practical use `ULiftable` (together with `up`), this function takes
/-- The most common practical use `ULiftable` (together with `down`), this function takes
`x : M.{u} α` and lifts it to `M.{max u v} (ULift.{v} α)` -/
@[reducible]
def up {f : Type u₀ → Type u₁} {g : Type max u₀ v₀ → Type v₁} [ULiftable f g] {α} :
Expand All @@ -57,7 +57,7 @@ def up {f : Type u₀ → Type u₁} {g : Type max u₀ v₀ → Type v₁} [ULi
#align uliftable.up ULiftable.up

/-- The most common practical use of `ULiftable` (together with `up`), this function takes
`x : M.{max u v} (ulift.{v} α)` and lowers it to `M.{u} α` -/
`x : M.{max u v} (ULift.{v} α)` and lowers it to `M.{u} α` -/
@[reducible]
def down {f : Type u₀ → Type u₁} {g : Type max u₀ v₀ → Type v₁} [ULiftable f g] {α} :
g (ULift.{v₀} α) → f α :=
Expand Down

0 comments on commit 74ee5fb

Please sign in to comment.