Skip to content

Commit

Permalink
feat: patch for std4#219
Browse files Browse the repository at this point in the history
  • Loading branch information
fgdorais committed Aug 17, 2023
1 parent d72f88a commit e22dff1
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
2 changes: 1 addition & 1 deletion Mathlib/Tactic/ToAdditive.lean
Original file line number Diff line number Diff line change
Expand Up @@ -96,7 +96,7 @@ Id.run do
if (s.get i₁).isUpper then
if let some strs := endCapitalNames.find? (s.extract 0 i₁) then
if let some (pref, newS) := strs.findSome?
fun x ↦ (s.extract i₁ s.endPos).dropPrefix? x |>.map (x, ·.toString) then
fun x : String ↦ (s.extract i₁ s.endPos).dropPrefix? x |>.map (x, ·.toString) then
return splitCase newS 0 <| (s.extract 0 i₁ ++ pref)::r
if !(s.get i₀).isUpper then
return splitCase (s.extract i₁ s.endPos) 0 <| (s.extract 0 i₁)::r
Expand Down
2 changes: 1 addition & 1 deletion lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -28,6 +28,6 @@
{"git":
{"url": "https://github.com/leanprover/std4",
"subDir?": null,
"rev": "dbffa8cb31b0c51b151453c4ff8f00ede2a84ed8",
"rev": "7d287609cc2e574326f642bd0c52567c01d2dcba",
"name": "std",
"inputRev?": "main"}}]}

0 comments on commit e22dff1

Please sign in to comment.