Skip to content

Commit 31686f3

Browse files
committed
chore: fix spelling ("the the")
1 parent 03a6e58 commit 31686f3

File tree

12 files changed

+14
-14
lines changed

12 files changed

+14
-14
lines changed

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/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/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.

src/Init/Tactics.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1004,7 +1004,7 @@ You can use `with` to provide the variables names for each constructor.
10041004
syntax (name := cases) "cases " elimTarget,+ (" using " term)? (inductionAlts)? : tactic
10051005

10061006
/--
1007-
The `fun_induction` tactic is a convenience wrapper around the `induction` tactic to use the the
1007+
The `fun_induction` tactic is a convenience wrapper around the `induction` tactic to use the
10081008
functional induction principle.
10091009
10101010
The tactic invocation

src/Lean/Elab/PreDefinition/FixedParams.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -307,7 +307,7 @@ def FixedParamPerm.isFixed (perm : FixedParamPerm) (i : Nat) : Bool :=
307307
perm[i]?.join.isSome
308308

309309
/--
310-
Brings the fixed parameters from `type`, which should the the type of the `funIdx`'s function, into
310+
Brings the fixed parameters from `type`, which should be the type of the `funIdx`'s function, into
311311
scope.
312312
-/
313313
private partial def FixedParamPerm.forallTelescopeImpl (perm : FixedParamPerm)

src/Lean/Elab/StructInst.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -804,7 +804,7 @@ private def synthOptParamFields : StructInstM Unit := do
804804
/-
805805
We must use `checkedAssign` here to ensure we do not create a cyclic
806806
assignment. See #3150.
807-
This can happen when there are holes in the the fields the default value
807+
This can happen when there are holes in the fields the default value
808808
depends on.
809809
Possible improvement: create a new `_` instead of returning `false` when
810810
`checkedAssign` fails. Reason: the field will not be needed after the

src/Lean/Elab/Tactic/Induction.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -49,7 +49,7 @@ def getAltName? (alt : Syntax) : Option Name :=
4949
else
5050
let ident := head[1]
5151
if ident.isOfKind identKind then some ident.getId.eraseMacroScopes else none
52-
/-- Returns true if the the alternative is for a wildcard, and that the wildcard is not due to a syntax error. -/
52+
/-- Returns true if the alternative is for a wildcard, and that the wildcard is not due to a syntax error. -/
5353
def isAltWildcard (altStx : Syntax) : Bool :=
5454
getAltName? altStx == some `_
5555
/-- Returns the `inductionAlt` `ident <|> hole` -/
@@ -233,7 +233,7 @@ public partial def mkElimApp (elimInfo : ElimInfo) (targets : Array Expr) (tag :
233233

234234
/--
235235
Given a goal `... targets ... |- C[targets, complexArgs]` associated with `mvarId`,
236-
where `complexArgs` are the the complex (i.e. non-target) arguments to the motive in the conclusion
236+
where `complexArgs` are the complex (i.e. non-target) arguments to the motive in the conclusion
237237
of the eliminator, construct `motiveArg := fun targets rs => C[targets, rs]`
238238
239239
This checks if the type of the complex arguments match what's expected by the motive, and

src/Lean/Meta/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1867,7 +1867,7 @@ def withLetDecl (name : Name) (type : Expr) (val : Expr) (k : Expr → n α) (no
18671867
/--
18681868
Runs `k x` with the local declaration `<name> : <type> := <val>` added to the local context, where `x` is the new free variable.
18691869
Afterwards, the result is wrapped in the given `let`/`have` expression (according to the value of `nondep`).
1870-
- If `usedLetOnly := true` (the default) then the the `let`/`have` is not created if the variable is unused.
1870+
- If `usedLetOnly := true` (the default) then the `let`/`have` is not created if the variable is unused.
18711871
-/
18721872
def mapLetDecl [MonadLiftT MetaM n] (name : Name) (type : Expr) (val : Expr) (k : Expr → n Expr) (nondep : Bool := false) (kind : LocalDeclKind := .default) (usedLetOnly : Bool := true) : n Expr :=
18731873
withLetDecl name type val (nondep := nondep) (kind := kind) fun x => do

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

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -61,7 +61,7 @@ def addCongrTable (e : Expr) : GoalM Unit := do
6161
pushEqHEq e e' congrPlaceholderProof
6262
if (← swapCgrRepr e e') then
6363
/-
64-
Recall that `isDiseq` and `mkDiseqProof?` are implemented using the the congruence table.
64+
Recall that `isDiseq` and `mkDiseqProof?` are implemented using the congruence table.
6565
So, if `e` is an equality `a = b`, and is the equivalence class of `False`, but `e'` is not,
6666
we **must** make `e` the representative of the congruence class.
6767
The equivalence classes of `e` and `e'` will be merged eventually since we used `pushEqHEq` above,

tests/lean/grind/experiments/bitvec.lean

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

51925192
/-- Negating a bitvector created from a natural number equals
5193-
creating a bitvector from the the negative of that number.
5193+
creating a bitvector from the negative of that number.
51945194
-/
51955195
theorem neg_ofNat_eq_ofInt_neg {w : Nat} {x : Nat} :
51965196
- BitVec.ofNat w x = BitVec.ofInt w (- x) := by

0 commit comments

Comments
 (0)