Skip to content

Commit 52e0742

Browse files
authored
chore: fix spelling mistakes (#8711)
Co-authored-by: euprunin <[email protected]>
1 parent 614e612 commit 52e0742

File tree

19 files changed

+28
-28
lines changed

19 files changed

+28
-28
lines changed

src/Init/Grind/Tactics.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -55,7 +55,7 @@ and stores `c` in `x`, `b` in `a`, and the proof that `c = some b` in `h`.
5555
-/
5656
def genPattern {α : Sort u} (_h : Prop) (x : α) (_val : α) : α := x
5757

58-
/-- Similar to `genPattern` but for the heterogenous case -/
58+
/-- Similar to `genPattern` but for the heterogeneous case -/
5959
def genHEqPattern {α β : Sort u} (_h : Prop) (x : α) (_val : β) : α := x
6060
end Lean.Grind
6161

src/Lean/Elab/Tactic/Induction.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -243,10 +243,10 @@ def setMotiveArg (mvarId : MVarId) (motiveArg : MVarId) (targets : Array FVarId)
243243
if (← isTypeCorrect absType') then
244244
absType := absType'
245245
else
246-
trace[Elab.induction] "Not abstracing goal over {complexArg}, resulting term is not type correct:{indentExpr absType'} }"
246+
trace[Elab.induction] "Not abstracting goal over {complexArg}, resulting term is not type correct:{indentExpr absType'} }"
247247
absType := .lam (← mkFreshUserName `x) complexArgType absType .default
248248
else
249-
trace[Elab.induction] "Not abstracing goal over {complexArg}, its type {complexArgType} does not match the expected {exptComplexArgType}"
249+
trace[Elab.induction] "Not abstracting goal over {complexArg}, its type {complexArgType} does not match the expected {exptComplexArgType}"
250250
absType := .lam (← mkFreshUserName `x) exptComplexArgType absType .default
251251

252252
let motive ← mkLambdaFVars (targets.map mkFVar) absType

src/Lean/EnvExtension.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -151,7 +151,7 @@ def insert (ext : MapDeclarationExtension α) (env : Environment) (declName : Na
151151
have : Inhabited Environment := ⟨env⟩
152152
assert! env.getModuleIdxFor? declName |>.isNone -- See comment at `MapDeclarationExtension`
153153
if !env.asyncMayContain declName then
154-
panic! s!"MapDeclarationExtension.insert: cannot insert {declName} into {ext.name}, it is not contined in {env.asyncPrefix?}"
154+
panic! s!"MapDeclarationExtension.insert: cannot insert {declName} into {ext.name}, it is not contained in {env.asyncPrefix?}"
155155
else
156156
ext.addEntry env (declName, val)
157157

src/Lean/Environment.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1859,7 +1859,7 @@ partial def importModulesCore
18591859
ImportStateM Unit := go imports (importAll := true) (isExported := isModule)
18601860
/-
18611861
When the module system is disabled for the root, we import all transitively referenced modules and
1862-
ignore any module sytem annotations on the way.
1862+
ignore any module system annotations on the way.
18631863
18641864
When the module system is enabled for the root, each module may need to be imported at one of the
18651865
following levels:

src/Lean/Linter/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -37,7 +37,7 @@ This structure contains all the data required to do so, the `Options` set on the
3737
or by the `set_option` command, and the `LinterSets` that have been declared.
3838
3939
A single structure holding this data is useful since we want `getLinterValue` to be a pure
40-
function: determinining the `LinterSets` would otherwise require a `MonadEnv` instance.
40+
function: determining the `LinterSets` would otherwise require a `MonadEnv` instance.
4141
-/
4242
structure LinterOptions where
4343
toOptions : Options

src/Lean/Meta/Constructions/NoConfusionLinear.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -10,7 +10,7 @@ import Lean.Meta.CompletionName
1010

1111
/-!
1212
This module produces a construction for the `noConfusionType` that is linear in size in the number of
13-
constructors of the inductive type. This is in contrast to the previous construction (definde in
13+
constructors of the inductive type. This is in contrast to the previous construction (defined in
1414
`no_confusion.cpp`), that is quadratic in size due to nested `.brecOn` applications.
1515
1616
We still use the old construction when processing the prelude, for the few inductives that we need

src/Lean/Meta/Tactic/FunInd.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1506,7 +1506,7 @@ where doRealize inductName := do
15061506

15071507
/--
15081508
Given an expression `fun x y z => body`, returns a bit mask of the functinon's arity length
1509-
that has `true` whenver that parameter of the function appears as a scrutinee of a `match` in
1509+
that has `true` whenever that parameter of the function appears as a scrutinee of a `match` in
15101510
tail position. These are the parameters that are likely useful as targets of the motive
15111511
of the functional cases theorem. All others become parameters or may be dropped.
15121512

src/Lean/Meta/Tactic/Grind/EMatch.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -407,7 +407,7 @@ private def applyAssignment (mvars : Array Expr) : OptionT (StateT Choice M) Uni
407407
theorem getElem_reverse {xs : Array α} {i : Nat} (hi : i < xs.reverse.size) :
408408
(xs.reverse)[i] = xs[xs.size - 1 - i]'(by simp at hi; omega)
409409
```
410-
The pattern for this theorem is `xs.reverese[i]`. Note that `hi` occurs there as an implicit argument.
410+
The pattern for this theorem is `xs.reverse[i]`. Note that `hi` occurs there as an implicit argument.
411411
The term `xs[j]` in our goal e-matches the pattern because we have the equality `xs.reverse = xs`.
412412
However, the implicit proof at `xs[j]` has type `j < xs.size` instead of `j < xs.reverse.size`.
413413
-/

src/Lean/Setup.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -15,7 +15,7 @@ Data types used by Lean module headers and the `--setup` CLI.
1515

1616
namespace Lean
1717

18-
/- Abstract sturcture of an `import` statement. -/
18+
/- Abstract structure of an `import` statement. -/
1919
structure Import where
2020
module : Name
2121
/-- `import all`; whether to import and expose all data saved by the module. -/

src/Std/Data/Iterators.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -67,7 +67,7 @@ steps are called productive. This behavior is encoded in the `Std.Iterators.Prod
6767
## Stability
6868
6969
The API for the usage of iterators provided in this module can be considered stable, as well as
70-
the API for the verification of programms using iterators, unless explicitly stated otherwise.
70+
the API for the verification of programs using iterators, unless explicitly stated otherwise.
7171
7272
Contrarily, the API for implementation of new iterators, including the design of the `Iterator`
7373
typeclass, is still experimental and will change in the future. It is already planned that there

0 commit comments

Comments
 (0)