src/Tools/Haskell/Haskell.thy
changeset 69482 186b03abb764
parent 69480 2cc9212342a7
child 69486 59ada9f63cc5
--- a/src/Tools/Haskell/Haskell.thy	Wed Dec 19 13:07:02 2018 +0100
+++ b/src/Tools/Haskell/Haskell.thy	Wed Dec 19 21:37:48 2018 +0100
@@ -751,9 +751,11 @@
 
 {- wrapped elements -}
 
+wrap_elem :: ((Markup.T, Body), [Tree]) -> Tree
 wrap_elem (((a, atts), body1), body2) =
   Elem ((\<open>XML.xml_elemN\<close>, (\<open>XML.xml_nameN\<close>, a) : atts), Elem ((\<open>XML.xml_bodyN\<close>, []), body1) : body2)
 
+unwrap_elem :: Tree -> Maybe ((Markup.T, Body), [Tree])
 unwrap_elem
   (Elem ((\<open>XML.xml_elemN\<close>, (\<open>XML.xml_nameN\<close>, a) : atts), Elem ((\<open>XML.xml_bodyN\<close>, []), body1) : body2)) =
   Just (((a, atts), body1), body2)
@@ -762,6 +764,7 @@
 
 {- text content -}
 
+add_content :: Tree -> Buffer.T -> Buffer.T
 add_content tree =
   case unwrap_elem tree of
     Just (_, ts) -> fold add_content ts
@@ -770,6 +773,7 @@
         Elem (_, ts) -> fold add_content ts
         Text s -> Buffer.add s
 
+content_of :: Body -> String
 content_of body = Buffer.empty |> fold add_content body |> Buffer.content