Skip to content

Commit e53b625

Browse files
committed
merge bump/nightly-2025-11-17
2 parents 344b192 + 8db306d commit e53b625

File tree

2 files changed

+4
-2
lines changed

2 files changed

+4
-2
lines changed

Batteries/Data/String/Lemmas.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -956,7 +956,8 @@ theorem get : ∀ {s}, ValidFor l (m₁ ++ c :: m₂) r s → s.get ⟨utf8Len m
956956
theorem next : ∀ {s}, ValidFor l (m₁ ++ c :: m₂) r s →
957957
s.next ⟨utf8Len m₁⟩ = ⟨utf8Len m₁ + c.utf8Size⟩
958958
| _, ⟨⟩ => by
959-
simp only [Substring.Raw.next, utf8Len_append, utf8Len_cons, List.append_assoc, List.cons_append]
959+
simp only [Substring.Raw.next, utf8Len_append, utf8Len_cons, List.append_assoc,
960+
List.cons_append]
960961
rw [if_neg (mt Pos.Raw.ext_iff.1 ?a)]
961962
case a =>
962963
simpa [Nat.add_assoc, Nat.add_comm, Nat.add_left_comm] using

Batteries/Data/String/Matcher.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -52,7 +52,8 @@ partial def Matcher.findAll (m : Matcher) (s : Substring.Raw) : Array Substring.
5252
loop s m.toMatcher #[]
5353
where
5454
/-- Accumulator loop for `String.Matcher.findAll` -/
55-
loop (s : Substring.Raw) (am : Array.Matcher Char) (occs : Array Substring.Raw) : Array Substring.Raw :=
55+
loop (s : Substring.Raw) (am : Array.Matcher Char) (occs : Array Substring.Raw) :
56+
Array Substring.Raw :=
5657
match am.next? s with
5758
| none => occs
5859
| some (s, am) =>

0 commit comments

Comments
 (0)