src/Doc/System/Basics.thy
changeset 52054 eaf17514aabd
parent 52052 892061142ba6
child 52056 fc458f304f93
--- a/src/Doc/System/Basics.thy	Fri May 17 18:23:39 2013 +0200
+++ b/src/Doc/System/Basics.thy	Fri May 17 18:39:49 2013 +0200
@@ -378,11 +378,9 @@
     -T ADDR      startup process wrapper, with socket address
     -W IN:OUT    startup process wrapper, with input/output fifos
     -e MLTEXT    pass MLTEXT to the ML session
-    -f           pass 'Session.finish();' to the ML session
     -m MODE      add print mode for output
     -q           non-interactive session
     -r           open heap file read-only
-    -u           pass 'use"ROOT.ML";' to the ML session
     -w           reset write permissions on OUTPUT
 
   INPUT (default "\$ISABELLE_LOGIC") and OUTPUT specify in/out heaps.
@@ -430,12 +428,6 @@
   may happen when errorneous ML code is provided. Also make sure that
   the ML commands are terminated properly by semicolon.
 
-  \medskip The @{verbatim "-u"} option is a shortcut for @{verbatim
-  "-e"} passing ``@{verbatim "use \"ROOT.ML\";"}'' to the ML session.
-  The @{verbatim "-f"} option passes ``@{verbatim
-  "Session.finish();"}'', which is intended mainly for administrative
-  purposes.
-
   \medskip The @{verbatim "-m"} option adds identifiers of print modes
   to be made active for this session. Typically, this is used by some
   user interface, e.g.\ to enable output of proper mathematical