src/Doc/System/Server.thy
changeset 69464 2323dce4a0db
parent 68957 eef4e983fd9d
child 69593 3dda49e08b9d
--- a/src/Doc/System/Server.thy	Thu Dec 13 17:37:14 2018 +0100
+++ b/src/Doc/System/Server.thy	Thu Dec 13 20:33:18 2018 +0100
@@ -183,7 +183,7 @@
 \<close>
 
 
-subsection \<open>Byte messages\<close>
+subsection \<open>Byte messages \label{sec:byte-messages}\<close>
 
 text \<open>
   The client-server connection is a raw byte-channel for bidirectional
@@ -281,10 +281,13 @@
 
 text \<open>
   Whenever a new client opens the server socket, the initial message needs to
-  be its unique password. The server replies either with \<^verbatim>\<open>OK\<close> (and some
-  information about the Isabelle version) or by silent disconnection of what
-  is considered an illegal connection attempt. Note that @{tool client}
-  already presents the correct password internally.
+  be its unique password as a single line, without length indication (i.e.\ a
+  ``short message'' in the sense of \secref{sec:byte-messages}).
+
+  The server replies either with \<^verbatim>\<open>OK\<close> (and some information about the
+  Isabelle version) or by silent disconnection of what is considered an
+  illegal connection attempt. Note that @{tool client} already presents the
+  correct password internally.
 
   Server passwords are created as Universally Unique Identifier (UUID) in
   Isabelle/Scala and stored in a per-user database, with restricted