src/Tools/Haskell/Haskell.thy
changeset 69463 6439c9024dcc
parent 69462 fe125722f7a9
child 69465 16fa609a62b1
--- a/src/Tools/Haskell/Haskell.thy	Thu Dec 13 17:03:59 2018 +0100
+++ b/src/Tools/Haskell/Haskell.thy	Thu Dec 13 17:37:14 2018 +0100
@@ -1589,7 +1589,7 @@
 TCP server on localhost.
 -}
 
-module Isabelle.Server (publish_text, publish_stdout, server) where
+module Isabelle.Server (localhost_name, localhost, publish_text, publish_stdout, server) where
 
 import Control.Monad (forever)
 import qualified Control.Exception as Exception
@@ -1603,12 +1603,12 @@
 
 {- server address -}
 
+localhost_name :: String
+localhost_name = "127.0.0.1"
+
 localhost :: Socket.HostAddress
 localhost = Socket.tupleToHostAddress (127, 0, 0, 1)
 
-localhost_name :: String
-localhost_name = "127.0.0.1"
-
 publish_text :: String -> String -> UUID.T -> String
 publish_text name address password =
   "server " ++ quote name ++ " = " ++ address ++ " (password " ++ quote (show password) ++ ")"