src/Tools/Haskell/Haskell.thy
changeset 69968 1a400b14fd3a
parent 69794 a19fdf64726c
child 70047 96fe857a7a6f
--- a/src/Tools/Haskell/Haskell.thy	Sun Mar 24 17:45:00 2019 +0100
+++ b/src/Tools/Haskell/Haskell.thy	Sun Mar 24 17:53:46 2019 +0100
@@ -327,7 +327,7 @@
   markupN, consistentN, unbreakableN, indentN, widthN,
   blockN, block, breakN, break, fbreakN, fbreak, itemN, item,
 
-  wordsN, words, no_wordsN, no_words,
+  wordsN, words,
 
   tfreeN, tfree, tvarN, tvar, freeN, free, skolemN, skolem, boundN, bound, varN, var,
   numeralN, numeral, literalN, literal, delimiterN, delimiter, inner_stringN, inner_string,
@@ -510,9 +510,6 @@
 wordsN :: String; words :: T
 (wordsN, words) = markup_elem \<open>Markup.wordsN\<close>
 
-no_wordsN :: String; no_words :: T
-(no_wordsN, no_words) = markup_elem \<open>Markup.no_wordsN\<close>
-
 
 {- inner syntax -}