Skip to content

Commit 2ca3bc2

Browse files
authored
chore: fix spelling (#11531)
Hi, these are just some spelling corrections. There is one I wasn't completely sure about in src/Init/Data/List/Lemmas.lean: > See also > ... > Also > \* \`Init.Data.List.Monadic\` for **addiation** _(additional?)_ lemmas about \`List.mapM\` and \`List.forM\`
1 parent 03a6e58 commit 2ca3bc2

Some content is hidden

Large Commits have some content hidden by default. Use the searchbox below for content that may be hidden.

57 files changed

+70
-70
lines changed

src/Init/Data/BitVec/Bitblast.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -835,7 +835,7 @@ execution. -/
835835
structure DivModArgs (w : Nat) where
836836
/-- the numerator (aka, dividend) -/
837837
n : BitVec w
838-
/-- the denumerator (aka, divisor)-/
838+
/-- the denominator (aka, divisor)-/
839839
d : BitVec w
840840

841841
/-- A `DivModState` is lawful if the remainder width `wr` plus the numerator width `wn` equals `w`,

src/Init/Data/BitVec/Lemmas.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5601,7 +5601,7 @@ theorem msb_eq_toNat {x : BitVec w}:
56015601
simp only [msb_eq_decide, ge_iff_le]
56025602

56035603
/-- Negating a bitvector created from a natural number equals
5604-
creating a bitvector from the the negative of that number.
5604+
creating a bitvector from the negative of that number.
56055605
-/
56065606
theorem neg_ofNat_eq_ofInt_neg {w : Nat} {x : Nat} :
56075607
- BitVec.ofNat w x = BitVec.ofInt w (- x) := by

src/Init/Data/Bool.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -260,7 +260,7 @@ instance : Std.Associative (· != ·) := ⟨bne_assoc⟩
260260

261261
theorem eq_not_of_ne : ∀ {x y : Bool}, x ≠ y → x = !y := by decide
262262

263-
/-! ### coercision related normal forms -/
263+
/-! ### coercion related normal forms -/
264264

265265
theorem beq_eq_decide_eq [BEq α] [LawfulBEq α] [DecidableEq α] (a b : α) :
266266
(a == b) = decide (a = b) := by

src/Init/Data/List/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -2252,7 +2252,7 @@ def eraseReps {α} [BEq α] (as : List α) : List α := eraseRepsBy (· == ·) a
22522252
/-! ### span -/
22532253

22542254
/--
2255-
Splits a list into the the longest initial segment for which `p` returns `true`, paired with the
2255+
Splits a list into the longest initial segment for which `p` returns `true`, paired with the
22562256
remainder of the list.
22572257
22582258
`O(|l|)`.

src/Init/Data/List/Lemmas.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -77,7 +77,7 @@ Further results, which first require developing further automation around `Nat`,
7777
* `Init.Data.List.Nat.TakeDrop`: `List.take` and `List.drop`
7878
7979
Also
80-
* `Init.Data.List.Monadic` for addiation lemmas about `List.mapM` and `List.forM`.
80+
* `Init.Data.List.Monadic` for additional lemmas about `List.mapM` and `List.forM`.
8181
8282
-/
8383

src/Init/Data/List/Sublist.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -249,7 +249,7 @@ theorem Sublist.eq_of_length : l₁ <+ l₂ → length l₁ = length l₂ → l
249249
| .cons a s, h => nomatch Nat.not_lt.2 s.length_le (h ▸ lt_succ_self _)
250250
| .cons₂ a s, h => by rw [s.eq_of_length (succ.inj h)]
251251

252-
-- Only activative `eq_of_length` if we're already thinking about lengths.
252+
-- Only activate `eq_of_length` if we're already thinking about lengths.
253253
grind_pattern Sublist.eq_of_length => l₁ <+ l₂, length l₁, length l₂
254254

255255
theorem Sublist.eq_of_length_le (s : l₁ <+ l₂) (h : length l₂ ≤ length l₁) : l₁ = l₂ :=

src/Init/Data/String/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1177,7 +1177,7 @@ position. -/
11771177
def Slice.Pos.get? {s : Slice} (pos : s.Pos) : Option Char :=
11781178
if h : pos = s.endPos then none else some (pos.get h)
11791179

1180-
/-- Returns the byte at the given position in the string, or panicks if the position is the end
1180+
/-- Returns the byte at the given position in the string, or panics if the position is the end
11811181
position. -/
11821182
@[expose]
11831183
def Slice.Pos.get! {s : Slice} (pos : s.Pos) : Char :=

src/Init/Data/String/Decode.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -529,7 +529,7 @@ public def assemble₂ (w x : UInt8) : Option Char :=
529529
else
530530
let r := assemble₂Unchecked w x
531531
if r < 0x80 then
532-
none -- overlong encodinlg
532+
none -- overlong encoding
533533
else
534534
some ⟨r, ?onemore⟩
535535
where finally

src/Init/Data/UInt/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -517,7 +517,7 @@ protected def UInt32.shiftRight (a b : UInt32) : UInt32 := ⟨a.toBitVec >>> (UI
517517
Strict inequality of 32-bit unsigned integers, defined as inequality of the corresponding
518518
natural numbers. Usually accessed via the `<` operator.
519519
-/
520-
-- These need to be exposed as `Init.Prelude` already has an instance for bootstrapping puproses and
520+
-- These need to be exposed as `Init.Prelude` already has an instance for bootstrapping purposes and
521521
-- they should be defeq
522522
@[expose] protected def UInt32.lt (a b : UInt32) : Prop := a.toBitVec < b.toBitVec
523523
/--

src/Init/System/IO.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -837,7 +837,7 @@ Encountering an EOF does not close a handle. Subsequent reads may block and retu
837837
-/
838838
@[extern "lean_io_prim_handle_read"] opaque read (h : @& Handle) (bytes : USize) : IO ByteArray
839839
/--
840-
Writes the provided bytes to the the handle.
840+
Writes the provided bytes to the handle.
841841
842842
Writing to a handle is typically buffered, and may not immediately modify the file on disk. Use
843843
`IO.FS.Handle.flush` to write changes to buffers to the associated device.

0 commit comments

Comments
 (0)