We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 16c7442 commit 157486eCopy full SHA for 157486e
src/Init/Data/String/Basic.lean
@@ -94,7 +94,7 @@ where
94
(have := c.utf8Size_pos; have := le_size_of_utf8DecodeChar?_eq_some h; by omega)
95
termination_by structural fuel
96
97
-@[inline, expose]
+@[expose, extern "lean_string_validate_utf8"]
98
def ByteArray.validateUTF8 (b : ByteArray) : Bool :=
99
go (b.size + 1) 0 (by simp) (by simp)
100
where
0 commit comments