You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
refactor: use String.ofList and String.toList for String <-> List Char conversion (#11017)
This PR establishes `String.ofList` and `String.toList` as the preferred
method for converting between strings and lists of characters and
deprecates the alternatives `String.mk`, `List.asString` and
`String.data`.
protectedtheoremle_trans {a b c : String} : a ≤ b → b ≤ c → a ≤ c := List.le_trans
35
37
protectedtheoremlt_trans {a b c : String} : a < b → b < c → a < c := List.lt_trans
36
38
protectedtheoremle_total (a b : String) : a ≤ b ∨ b ≤ a := List.le_total _ _
37
-
protectedtheoremle_antisymm {a b : String} : a ≤ b → b ≤ a → a = b := fun h₁ h₂ => String.ext (List.le_antisymm (as := a.data) (bs := b.data) h₁ h₂)
39
+
protectedtheoremle_antisymm {a b : String} : a ≤ b → b ≤ a → a = b := fun h₁ h₂ => String.ext (List.le_antisymm (as := a.toList) (bs := b.toList) h₁ h₂)
38
40
protectedtheoremlt_asymm {a b : String} (h : a < b) : ¬ b < a := List.lt_asymm h
39
41
protectedtheoremne_of_lt {a b : String} (h : a < b) : a ≠ b := by
if (c.fileMap.toPosition info.getPos?.get!).column != col then
1084
-
s.mkErrorAt s!"closing '{String.mk <| List.replicate fenceWidth ':'}' from directive on line {l} at column {col}, but it's at column {(c.fileMap.toPosition info.getPos?.get!).column}" info.getPos?.get!
1084
+
s.mkErrorAt s!"closing '{String.ofList <| List.replicate fenceWidth ':'}' from directive on line {l} at column {col}, but it's at column {(c.fileMap.toPosition info.getPos?.get!).column}" info.getPos?.get!
1085
1085
else
1086
1086
s))
1087
1087
@@ -1114,7 +1114,7 @@ mutual
1114
1114
else skipFn
1115
1115
1116
1116
closeFence (line width : Nat) :=
1117
-
let str := String.mk (.replicate width ':')
1117
+
let str := String.ofList (.replicate width ':')
1118
1118
bolThen (description := s!"closing '{str}' for directive from line {line}")
0 commit comments