@@ -1818,7 +1818,7 @@ theorem Nat.succ_pos (n : Nat) : LT.lt 0 (succ n) :=
18181818
18191819set_option bootstrap.genMatcherCode false in
18201820/--
1821- The predecessor of a natural number is one less than it. The precedessor of `0` is defined to be
1821+ The predecessor of a natural number is one less than it. The predecessor of `0` is defined to be
18221822`0`.
18231823
18241824This definition is overridden in the compiler with an efficient implementation. This definition is
@@ -1958,7 +1958,7 @@ instance instSubNat : Sub Nat where
19581958 sub := Nat.sub
19591959
19601960/--
1961- Gets the word size of the curent platform. The word size may be 64 or 32 bits.
1961+ Gets the word size of the current platform. The word size may be 64 or 32 bits.
19621962
19631963This function is opaque because there is no guarantee at compile time that the target will have the
19641964same word size as the host. It also helps avoid having type checking be architecture-dependent.
@@ -3409,7 +3409,7 @@ instance {ε : Type u} {α : Type v} [Inhabited ε] : Inhabited (Except ε α) w
34093409Exception monads provide the ability to throw errors and handle errors.
34103410
34113411In this class, `ε` is a `semiOutParam`, which means that it can influence the choice of instance.
3412- `MonadExcept ε` provides the same operations, but requires that `ε` be inferrable from `m`.
3412+ `MonadExcept ε` provides the same operations, but requires that `ε` be inferable from `m`.
34133413
34143414`tryCatchThe`, which takes an explicit exception type, is used to desugar `try ... catch ...` steps
34153415inside `do`-blocks when the handlers have type annotations.
@@ -3589,7 +3589,7 @@ be read, but not written. A `MonadWithReader ρ` instance additionally allows th
35893589overridden for a sub-computation.
35903590
35913591In this class, `ρ` is a `semiOutParam`, which means that it can influence the choice of instance.
3592- `MonadReader ρ` provides the same operations, but requires that `ρ` be inferrable from `m`.
3592+ `MonadReader ρ` provides the same operations, but requires that `ρ` be inferable from `m`.
35933593-/
35943594-- Note: This class can be seen as a simplification of the more "principled" definition
35953595-- ```
@@ -3641,7 +3641,7 @@ instance {ρ : Type u} {m : Type u → Type v} [Monad m] : MonadReaderOf ρ (Rea
36413641A reader monad that additionally allows the value to be locally overridden.
36423642
36433643In this class, `ρ` is a `semiOutParam`, which means that it can influence the choice of instance.
3644- `MonadWithReader ρ` provides the same operations, but requires that `ρ` be inferrable from `m`.
3644+ `MonadWithReader ρ` provides the same operations, but requires that `ρ` be inferable from `m`.
36453645-/
36463646class MonadWithReaderOf (ρ : semiOutParam (Type u)) (m : Type u → Type v) where
36473647 /--
@@ -3698,7 +3698,7 @@ Instances may implement these operations by passing state values around, by usin
36983698reference cell (e.g. `ST.Ref σ`), or in other ways.
36993699
37003700In this class, `σ` is a `semiOutParam`, which means that it can influence the choice of instance.
3701- `MonadState σ` provides the same operations, but requires that `σ` be inferrable from `m`.
3701+ `MonadState σ` provides the same operations, but requires that `σ` be inferable from `m`.
37023702
37033703The mutable state of a state monad is visible between multiple `do`-blocks or functions, unlike
37043704[ local mutable state ] (lean-manual://section/do-notation-let-mut) in `do`-notation.
0 commit comments