--- a/src/Tools/Haskell/Haskell.thy Fri Sep 20 13:30:55 2024 +0200
+++ b/src/Tools/Haskell/Haskell.thy Fri Sep 20 14:28:13 2024 +0200
@@ -1564,7 +1564,7 @@
show_tree (Text s) = Buffer.add (encode_text s)
show_elem name atts =
- space_implode " " (name : map (\(a, x) -> a <> "=\"" <> encode_text x <> "\"") atts)
+ implode_space (name : map (\(a, x) -> a <> "=\"" <> encode_text x <> "\"") atts)
\<close>
generate_file "Isabelle/XML/Encode.hs" = \<open>
@@ -3473,7 +3473,7 @@
else "\\" <> Bytes.singleton b
strings :: [Bytes] -> Bytes
-strings = space_implode " " . map string
+strings = implode_space . map string
{- server parameters -}