--- a/src/Tools/Haskell/Buffer.hs Sat Nov 10 17:07:17 2018 +0100
+++ b/src/Tools/Haskell/Buffer.hs Sat Nov 10 17:12:09 2018 +0100
@@ -5,6 +5,8 @@
LICENSE: BSD 3-clause (Isabelle)
Efficient text buffers.
+
+See also "$ISABELLE_HOME/src/Pure/General/buffer.ML".
-}
module Isabelle.Buffer (T, empty, add, content)
--- a/src/Tools/Haskell/File.hs Sat Nov 10 17:07:17 2018 +0100
+++ b/src/Tools/Haskell/File.hs Sat Nov 10 17:12:09 2018 +0100
@@ -4,7 +4,9 @@
Author: Makarius
LICENSE: BSD 3-clause (Isabelle)
-File-system operations
+File-system operations.
+
+See also "$ISABELLE_HOME/src/Pure/General/file.ML".
-}
module Isabelle.File (setup, read, write, append) where
--- a/src/Tools/Haskell/Haskell.thy Sat Nov 10 17:07:17 2018 +0100
+++ b/src/Tools/Haskell/Haskell.thy Sat Nov 10 17:12:09 2018 +0100
@@ -33,6 +33,8 @@
LICENSE: BSD 3-clause (Isabelle)
Basic library of Isabelle idioms.
+
+See also \<^file>\<open>$ISABELLE_HOME/src/Pure/General/basics.ML\<close>, \<^file>\<open>$ISABELLE_HOME/src/Pure/library.ML\<close>.
-}
module Isabelle.Library (
@@ -122,6 +124,8 @@
LICENSE: BSD 3-clause (Isabelle)
Plain values, represented as string.
+
+See also \<^file>\<open>$ISABELLE_HOME/src/Pure/General/value.ML\<close>.
-}
module Isabelle.Value
@@ -173,6 +177,8 @@
LICENSE: BSD 3-clause (Isabelle)
Efficient text buffers.
+
+See also \<^file>\<open>$ISABELLE_HOME/src/Pure/General/buffer.ML\<close>.
-}
module Isabelle.Buffer (T, empty, add, content)
@@ -197,6 +203,8 @@
LICENSE: BSD 3-clause (Isabelle)
Property lists.
+
+See also \<^file>\<open>$ISABELLE_HOME/src/Pure/General/properties.ML\<close>.
-}
module Isabelle.Properties (Entry, T, defined, get, put, remove)
@@ -229,6 +237,8 @@
LICENSE: BSD 3-clause (Isabelle)
Quasi-abstract markup elements.
+
+See also \<^file>\<open>$ISABELLE_HOME/src/Pure/PIDE/markup.ML\<close>.
-}
module Isabelle.Markup (
@@ -521,7 +531,9 @@
Author: Makarius
LICENSE: BSD 3-clause (Isabelle)
-File-system operations
+File-system operations.
+
+See also \<^file>\<open>$ISABELLE_HOME/src/Pure/General/file.ML\<close>.
-}
module Isabelle.File (setup, read, write, append) where
@@ -555,6 +567,8 @@
LICENSE: BSD 3-clause (Isabelle)
Untyped XML trees and representation of ML values.
+
+See also \<^file>\<open>$ISABELLE_HOME/src/Pure/PIDE/xml.ML\<close>.
-}
module Isabelle.XML (Attributes, Body, Tree(..), wrap_elem, unwrap_elem, content_of)
@@ -632,6 +646,8 @@
LICENSE: BSD 3-clause (Isabelle)
XML as data representation language.
+
+See also \<^file>\<open>$ISABELLE_HOME/src/Pure/PIDE/xml.ML\<close>.
-}
module Isabelle.XML.Encode (
@@ -716,6 +732,8 @@
LICENSE: BSD 3-clause (Isabelle)
XML as data representation language.
+
+See also \<^file>\<open>$ISABELLE_HOME/src/Pure/PIDE/xml.ML\<close>.
-}
module Isabelle.XML.Decode (
@@ -825,6 +843,8 @@
LICENSE: BSD 3-clause (Isabelle)
Generic pretty printing module.
+
+See also \<^file>\<open>$ISABELLE_HOME/src/Pure/General/pretty.ML\<close>.
-}
module Isabelle.Pretty (
@@ -978,6 +998,8 @@
Efficient text representation of XML trees. Suitable for direct
inlining into plain text.
+
+See also \<^file>\<open>$ISABELLE_HOME/src/Pure/PIDE/yxml.ML\<close>.
-}
module Isabelle.YXML (charX, charY, strX, strY, detect, output_markup,
@@ -1103,6 +1125,8 @@
LICENSE: BSD 3-clause (Isabelle)
Lambda terms, types, sorts.
+
+See also \<^file>\<open>$ISABELLE_HOME/src/Pure/term.scala\<close>.
-}
module Isabelle.Term (
@@ -1148,6 +1172,8 @@
LICENSE: BSD 3-clause (Isabelle)
XML data representation of lambda terms.
+
+See also \<^file>\<open>$ISABELLE_HOME/src/Pure/term_xml.ML\<close>.
-}
{-# LANGUAGE LambdaCase #-}
@@ -1188,6 +1214,8 @@
LICENSE: BSD 3-clause (Isabelle)
XML data representation of lambda terms.
+
+See also \<^file>\<open>$ISABELLE_HOME/src/Pure/term_xml.ML\<close>.
-}
module Isabelle.Term_XML.Decode (sort, typ, term)
--- a/src/Tools/Haskell/Library.hs Sat Nov 10 17:07:17 2018 +0100
+++ b/src/Tools/Haskell/Library.hs Sat Nov 10 17:12:09 2018 +0100
@@ -5,6 +5,8 @@
LICENSE: BSD 3-clause (Isabelle)
Basic library of Isabelle idioms.
+
+See also "$ISABELLE_HOME/src/Pure/General/basics.ML", "$ISABELLE_HOME/src/Pure/library.ML".
-}
module Isabelle.Library (
--- a/src/Tools/Haskell/Markup.hs Sat Nov 10 17:07:17 2018 +0100
+++ b/src/Tools/Haskell/Markup.hs Sat Nov 10 17:12:09 2018 +0100
@@ -5,6 +5,8 @@
LICENSE: BSD 3-clause (Isabelle)
Quasi-abstract markup elements.
+
+See also "$ISABELLE_HOME/src/Pure/PIDE/markup.ML".
-}
module Isabelle.Markup (
--- a/src/Tools/Haskell/Pretty.hs Sat Nov 10 17:07:17 2018 +0100
+++ b/src/Tools/Haskell/Pretty.hs Sat Nov 10 17:12:09 2018 +0100
@@ -5,6 +5,8 @@
LICENSE: BSD 3-clause (Isabelle)
Generic pretty printing module.
+
+See also "$ISABELLE_HOME/src/Pure/General/pretty.ML".
-}
module Isabelle.Pretty (
--- a/src/Tools/Haskell/Properties.hs Sat Nov 10 17:07:17 2018 +0100
+++ b/src/Tools/Haskell/Properties.hs Sat Nov 10 17:12:09 2018 +0100
@@ -5,6 +5,8 @@
LICENSE: BSD 3-clause (Isabelle)
Property lists.
+
+See also "$ISABELLE_HOME/src/Pure/General/properties.ML".
-}
module Isabelle.Properties (Entry, T, defined, get, put, remove)
--- a/src/Tools/Haskell/Term.hs Sat Nov 10 17:07:17 2018 +0100
+++ b/src/Tools/Haskell/Term.hs Sat Nov 10 17:12:09 2018 +0100
@@ -5,6 +5,8 @@
LICENSE: BSD 3-clause (Isabelle)
Lambda terms, types, sorts.
+
+See also "$ISABELLE_HOME/src/Pure/term.scala".
-}
module Isabelle.Term (
--- a/src/Tools/Haskell/Term_XML/Decode.hs Sat Nov 10 17:07:17 2018 +0100
+++ b/src/Tools/Haskell/Term_XML/Decode.hs Sat Nov 10 17:12:09 2018 +0100
@@ -5,6 +5,8 @@
LICENSE: BSD 3-clause (Isabelle)
XML data representation of lambda terms.
+
+See also "$ISABELLE_HOME/src/Pure/term_xml.ML".
-}
module Isabelle.Term_XML.Decode (sort, typ, term)
--- a/src/Tools/Haskell/Term_XML/Encode.hs Sat Nov 10 17:07:17 2018 +0100
+++ b/src/Tools/Haskell/Term_XML/Encode.hs Sat Nov 10 17:12:09 2018 +0100
@@ -5,6 +5,8 @@
LICENSE: BSD 3-clause (Isabelle)
XML data representation of lambda terms.
+
+See also "$ISABELLE_HOME/src/Pure/term_xml.ML".
-}
{-# LANGUAGE LambdaCase #-}
--- a/src/Tools/Haskell/Value.hs Sat Nov 10 17:07:17 2018 +0100
+++ b/src/Tools/Haskell/Value.hs Sat Nov 10 17:12:09 2018 +0100
@@ -5,6 +5,8 @@
LICENSE: BSD 3-clause (Isabelle)
Plain values, represented as string.
+
+See also "$ISABELLE_HOME/src/Pure/General/value.ML".
-}
module Isabelle.Value
--- a/src/Tools/Haskell/XML.hs Sat Nov 10 17:07:17 2018 +0100
+++ b/src/Tools/Haskell/XML.hs Sat Nov 10 17:12:09 2018 +0100
@@ -5,6 +5,8 @@
LICENSE: BSD 3-clause (Isabelle)
Untyped XML trees and representation of ML values.
+
+See also "$ISABELLE_HOME/src/Pure/PIDE/xml.ML".
-}
module Isabelle.XML (Attributes, Body, Tree(..), wrap_elem, unwrap_elem, content_of)
--- a/src/Tools/Haskell/XML/Decode.hs Sat Nov 10 17:07:17 2018 +0100
+++ b/src/Tools/Haskell/XML/Decode.hs Sat Nov 10 17:12:09 2018 +0100
@@ -5,6 +5,8 @@
LICENSE: BSD 3-clause (Isabelle)
XML as data representation language.
+
+See also "$ISABELLE_HOME/src/Pure/PIDE/xml.ML".
-}
module Isabelle.XML.Decode (
--- a/src/Tools/Haskell/XML/Encode.hs Sat Nov 10 17:07:17 2018 +0100
+++ b/src/Tools/Haskell/XML/Encode.hs Sat Nov 10 17:12:09 2018 +0100
@@ -5,6 +5,8 @@
LICENSE: BSD 3-clause (Isabelle)
XML as data representation language.
+
+See also "$ISABELLE_HOME/src/Pure/PIDE/xml.ML".
-}
module Isabelle.XML.Encode (
--- a/src/Tools/Haskell/YXML.hs Sat Nov 10 17:07:17 2018 +0100
+++ b/src/Tools/Haskell/YXML.hs Sat Nov 10 17:12:09 2018 +0100
@@ -6,6 +6,8 @@
Efficient text representation of XML trees. Suitable for direct
inlining into plain text.
+
+See also "$ISABELLE_HOME/src/Pure/PIDE/yxml.ML".
-}
module Isabelle.YXML (charX, charY, strX, strY, detect, output_markup,