Skip to content

Commit 894c511

Browse files
authored
chore: bump toolchain to v4.26.0-rc1 (#145)
1 parent 135329b commit 894c511

File tree

2 files changed

+2
-2
lines changed

2 files changed

+2
-2
lines changed

ProofWidgets/Component/MakeEditLink.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -7,7 +7,7 @@ public meta section
77

88
/-- Assuming that `s` is the content of a file starting at position `p`,
99
advance `p` to the end of `s`. -/
10-
def Lean.Lsp.Position.advance (p : Position) (s : Substring) : Position :=
10+
def Lean.Lsp.Position.advance (p : Position) (s : Substring.Raw) : Position :=
1111
let (nLinesAfter, lastLineUtf16Sz) := s.foldl
1212
(init := (0, 0))
1313
fun (n, l) c => if c == '\n' then (n + 1, 0) else (n, l + c.utf16Size.toNat)

lean-toolchain

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1 +1 @@
1-
leanprover/lean4:v4.25.1
1+
leanprover/lean4:v4.26.0-rc1

0 commit comments

Comments
 (0)