Skip to content

Commit 26afb8a

Browse files
committed
chore: fix spelling
1 parent 31686f3 commit 26afb8a

Some content is hidden

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

45 files changed

+56
-56
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/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/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/Lean/Attributes.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -250,7 +250,7 @@ structure ParametricAttributeImpl (α : Type) extends AttributeImplCore where
250250
afterSet : Name → α → AttrM Unit := fun _ _ _ => pure ()
251251
/--
252252
If set, entries are not resorted on export and `getParam?` will fall back to a linear instead of
253-
binary search insde an imported module's entries.
253+
binary search inside an imported module's entries.
254254
-/
255255
preserveOrder : Bool := false
256256
/--

src/Lean/Compiler/IR/LiveVars.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -68,7 +68,7 @@ partial def visitFnBody (w : Index) : FnBody → M Bool
6868
-- Instead of marking the join points that we have already been visited, we permanently remove `j` from the context.
6969
set (ctx.eraseJoinPointDecl j) *> visitFnBody w b
7070
| none =>
71-
-- `j` must be a local join point. So do nothing since we have already visite its body.
71+
-- `j` must be a local join point. So do nothing since we have already visited its body.
7272
pure false
7373
| .ret x =>
7474
visitArg w x

src/Lean/Elab/Coinductive.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -72,7 +72,7 @@ builtin_initialize
7272
Note that at this point `PartialFixpoint` machinery applies the attributes and modifiers. We
7373
use the syntax references from the original `InductiveView`s and set them to those declarations.
7474
75-
Moreover, we have following theorem (generated by `generateEqLemmas`) that connets the coinductive
75+
Moreover, we have following theorem (generated by `generateEqLemmas`) that connects the coinductive
7676
predicate to its flat inductive:
7777
```
7878
info: infSeq.functor_unfold (α : Type) (r : α → α → Prop) (a✝ : α) : infSeq α r a✝ = infSeq._functor α r (infSeq α r) a✝
@@ -250,7 +250,7 @@ private def generateCoinductiveConstructor (infos : Array InductiveVal) (ctorSyn
250250
let newHole ← hole.replaceTargetEq rewriteResult.eNew rewriteResult.eqProof
251251

252252
/-
253-
Now, all it suffices is to call an approprate constructor of the flat inductive.
253+
Now, all it suffices is to call an appropriate constructor of the flat inductive.
254254
-/
255255
let constructor := mkConst ctor.name levelParams
256256
let constructor := mkAppN constructor params
@@ -365,7 +365,7 @@ private def mkCasesOnCoinductive (infos : Array InductiveVal) : MetaM Unit := do
365365
-- Then we apply the metavariable to the `casesOn` of the flat inductive
366366
let originalCasesOn := mkApp originalCasesOn motiveMVar
367367

368-
-- The next arguemnts of the `casesOn` are type indices
368+
-- The next arguments of the `casesOn` are type indices
369369
forallBoundedTelescope goalType info.numIndices fun indices goalType => do
370370
/-
371371
The types do not change, so we just make free variables for them

0 commit comments

Comments
 (0)