Skip to content

Commit 8ae29d1

Browse files
alokclaude
andcommitted
style: fix spelling errors in Lean/ docstrings
This PR fixes spelling errors in Lean compiler documentation: - "occuring" → "occurring" in LibrarySuggestions/Basic.lean (2 occurrences) - "the the" → "the" in Meta/Match/Match.lean - "interatively" → "iteratively" in Meta/Match/Match.lean 🤖 Generated with [Claude Code](https://claude.com/claude-code) Co-Authored-By: Claude Opus 4.5 <noreply@anthropic.com>
1 parent ef9777e commit 8ae29d1

File tree

2 files changed

+4
-4
lines changed

2 files changed

+4
-4
lines changed

src/Lean/LibrarySuggestions/Basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -92,10 +92,10 @@ end FoldRelevantConstantsImpl
9292
@[implemented_by FoldRelevantConstantsImpl.foldUnsafe]
9393
public opaque foldRelevantConstants {α : Type} (e : Expr) (init : α) (f : Name → α → MetaM α) : MetaM α := pure init
9494

95-
/-- Collect the constants occuring in `e` (once each), skipping instance arguments and proofs. -/
95+
/-- Collect the constants occurring in `e` (once each), skipping instance arguments and proofs. -/
9696
public def relevantConstants (e : Expr) : MetaM (Array Name) := foldRelevantConstants e #[] (fun n ns => return ns.push n)
9797

98-
/-- Collect the constants occuring in `e` (once each), skipping instance arguments and proofs. -/
98+
/-- Collect the constants occurring in `e` (once each), skipping instance arguments and proofs. -/
9999
public def relevantConstantsAsSet (e : Expr) : MetaM NameSet := foldRelevantConstants e ∅ (fun n ns => return ns.insert n)
100100

101101
end Lean.Expr

src/Lean/Meta/Match/Match.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -22,9 +22,9 @@ import Lean.Meta.Match.NamedPatterns
2222

2323
/-!
2424
This module implements the backend of match compilation. The elaborator has already elaborated
25-
the patterns and the the expected type of the matcher is known.
25+
the patterns and the expected type of the matcher is known.
2626
27-
The match compilation task is represented as a `Problem`, which is then processed interatively by
27+
The match compilation task is represented as a `Problem`, which is then processed iteratively by
2828
the `process` function. It has various “moves” which it tries in a particular order, to make progress
2929
on the problem, possibly splitting it.
3030

0 commit comments

Comments
 (0)