diff -r 73487ebd7332 -r 12c984b7d391 src/Tools/Haskell/Haskell.thy --- a/src/Tools/Haskell/Haskell.thy Fri Jul 30 22:39:08 2021 +0200 +++ b/src/Tools/Haskell/Haskell.thy Fri Jul 30 22:54:50 2021 +0200 @@ -200,7 +200,7 @@ the, the_default, - fold, fold_rev, single, map_index, get_index, + fold, fold_rev, single, map_index, get_index, separate, proper_string, quote, space_implode, commas, commas_quote, cat_lines, space_explode, split_lines, trim_line, clean_name) @@ -1483,7 +1483,7 @@ commas, enclose, enum, list, str_list, big_list) where -import Isabelle.Library hiding (quote, commas) +import Isabelle.Library hiding (quote, separate, commas) import qualified Data.List as List import qualified Isabelle.Buffer as Buffer import qualified Isabelle.Markup as Markup