src/Tools/Haskell/Haskell.thy
changeset 74087 12c984b7d391
parent 74086 73487ebd7332
child 74088 6d8674ffb962
equal deleted inserted replaced
74086:73487ebd7332 74087:12c984b7d391
   198 module Isabelle.Library (
   198 module Isabelle.Library (
   199   (|>), (|->), (#>), (#->),
   199   (|>), (|->), (#>), (#->),
   200 
   200 
   201   the, the_default,
   201   the, the_default,
   202 
   202 
   203   fold, fold_rev, single, map_index, get_index,
   203   fold, fold_rev, single, map_index, get_index, separate,
   204 
   204 
   205   proper_string, quote, space_implode, commas, commas_quote, cat_lines,
   205   proper_string, quote, space_implode, commas, commas_quote, cat_lines,
   206   space_explode, split_lines, trim_line, clean_name)
   206   space_explode, split_lines, trim_line, clean_name)
   207 where
   207 where
   208 
   208 
  1481   str, brk_indent, brk, fbrk, breaks, fbreaks, blk, block, strs, markup, mark, mark_str, marks_str,
  1481   str, brk_indent, brk, fbrk, breaks, fbreaks, blk, block, strs, markup, mark, mark_str, marks_str,
  1482   item, text_fold, keyword1, keyword2, text, paragraph, para, quote, cartouche, separate,
  1482   item, text_fold, keyword1, keyword2, text, paragraph, para, quote, cartouche, separate,
  1483   commas, enclose, enum, list, str_list, big_list)
  1483   commas, enclose, enum, list, str_list, big_list)
  1484 where
  1484 where
  1485 
  1485 
  1486 import Isabelle.Library hiding (quote, commas)
  1486 import Isabelle.Library hiding (quote, separate, commas)
  1487 import qualified Data.List as List
  1487 import qualified Data.List as List
  1488 import qualified Isabelle.Buffer as Buffer
  1488 import qualified Isabelle.Buffer as Buffer
  1489 import qualified Isabelle.Markup as Markup
  1489 import qualified Isabelle.Markup as Markup
  1490 import qualified Isabelle.XML as XML
  1490 import qualified Isabelle.XML as XML
  1491 import qualified Isabelle.YXML as YXML
  1491 import qualified Isabelle.YXML as YXML