src/Tools/Haskell/Haskell.thy
changeset 77029 1046a69fabaa
parent 75073 f8008b40b8a0
child 78021 ce6e3bc34343
--- a/src/Tools/Haskell/Haskell.thy	Fri Jan 20 19:52:52 2023 +0100
+++ b/src/Tools/Haskell/Haskell.thy	Fri Jan 20 20:26:42 2023 +0100
@@ -737,8 +737,6 @@
 
   expressionN, expression,
 
-  citationN, citation,
-
   pathN, path, urlN, url, docN, doc,
 
   markupN, consistentN, unbreakableN, indentN, widthN,
@@ -905,14 +903,6 @@
 expression kind = (expressionN, if kind == "" then [] else [(kindN, kind)])
 
 
-{- citation -}
-
-citationN :: Bytes
-citationN = \<open>Markup.citationN\<close>
-citation :: Bytes -> T
-citation = markup_string nameN citationN
-
-
 {- external resources -}
 
 pathN :: Bytes