Skip to content

Commit

Permalink
chore: fix typos, remove extra spaces (#121)
Browse files Browse the repository at this point in the history
Co-authored-by: euprunin <[email protected]>
  • Loading branch information
euprunin and euprunin authored Nov 1, 2024
1 parent b6b502e commit 2c73f5c
Show file tree
Hide file tree
Showing 5 changed files with 7 additions and 7 deletions.
2 changes: 1 addition & 1 deletion Manual/BasicTypes/String/Logical.lean
Original file line number Diff line number Diff line change
Expand Up @@ -19,4 +19,4 @@ set_option pp.rawOnError true
{docstring String}

The logical model of strings in Lean is a structure that contains a single field, which is a list of characters.
This is convenient when specifying and proving properties of string-processing fuctions at a low level.
This is convenient when specifying and proving properties of string-processing functions at a low level.
4 changes: 2 additions & 2 deletions Manual/Meta/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -39,7 +39,7 @@ def runParserCategory (env : Environment) (opts : Lean.Options) (catName : Name)
let p := andthenFn whitespace (categoryParserFnImpl catName)
let ictx := mkInputContext input fileName
let s := p.run ictx { env, options := opts } (getTokenTable env) (mkParserState input)
if !s.allErrors.isEmpty then
if !s.allErrors.isEmpty then
Except.error (toErrorMsg ictx s)
else if ictx.input.atEnd s.pos then
Except.ok s.stxStack.back
Expand All @@ -58,7 +58,7 @@ def runParser (env : Environment) (opts : Lean.Options) (p : Parser) (input : St
let ictx := mkInputContext input fileName
let p' := adaptCacheableContext ({· with prec}) p
let s := p'.fn.run ictx { env, options := opts } (getTokenTable env) (mkParserState input)
if !s.allErrors.isEmpty then
if !s.allErrors.isEmpty then
Except.error (toErrorMsg ictx s)
else if ictx.input.atEnd s.pos then
Except.ok s.stxStack.back
Expand Down
2 changes: 1 addition & 1 deletion Manual/Meta/Lean.lean
Original file line number Diff line number Diff line change
Expand Up @@ -541,7 +541,7 @@ defmethod Lean.NameMap.getOrSuggest [Monad m] [MonadInfoTree m] [MonadError m]
| none =>
for (n, _) in map do
-- TODO once Levenshtein is merged upstream, use it here
if FuzzyMatching.fuzzyMatch key.getId.toString n.toString || FuzzyMatching.fuzzyMatch n.toString key.getId.toString then
if FuzzyMatching.fuzzyMatch key.getId.toString n.toString || FuzzyMatching.fuzzyMatch n.toString key.getId.toString then
Suggestion.saveSuggestion key n.toString n.toString
throwErrorAt key "'{key}' not found - options are {map.toList.map (·.fst)}"

Expand Down
4 changes: 2 additions & 2 deletions Manual/Tactics.lean
Original file line number Diff line number Diff line change
Expand Up @@ -111,7 +111,7 @@ intro n k
```
::::

The {tactic}`case` and {tactic}`case'` tactics can be used to select a new main goal using the desired goal's name.
The {tactic}`case` and {tactic}`case'` tactics can be used to select a new main goal using the desired goal's name.
When names are assigned in the context of a goal which itself has a name, the new goals's names are appended to the main goal's name with a dot (`'.', Unicode FULL STOP (0x2e)`) between them.

::::example "Hierarchical Goal Names"
Expand Down Expand Up @@ -789,7 +789,7 @@ When proving that {goal}`∀ (n : Nat), 0 + n = n`, the initial proof state is:
⊢ ∀ (n : Nat), 0 + n = n
```

The tactic {tacticStep}`intro` results in a proof state with an inaccessible assumption:
The tactic {tacticStep}`intro` results in a proof state with an inaccessible assumption:

```post
n✝ : Nat
Expand Down
2 changes: 1 addition & 1 deletion Manual/Tactics/Conv.lean
Original file line number Diff line number Diff line change
Expand Up @@ -53,7 +53,7 @@ example (x y z : Nat) : x + (y + z) = (x + z) + y := by

In this example, addition occurs under binders, so {tactic}`rw` can't be used.
However, after using {tactic}`conv` to navigate to the function body, it succeeds.
The nested use of {tactic}`conv` causes control to return to the current position in the term after performing further coversions on one of its subterms.
The nested use of {tactic}`conv` causes control to return to the current position in the term after performing further conversions on one of its subterms.
Because the goal is a reflexive equation after rewriting, {tactic}`conv` automatically closes it.

```lean
Expand Down

0 comments on commit 2c73f5c

Please sign in to comment.