src/Doc/System/Sessions.thy
changeset 68314 2acbf8129d8b
parent 68292 7ca0c23179e6
child 68348 2ac3a5c07dfa
equal deleted inserted replaced
68311:c551d8acaa42 68314:2acbf8129d8b
   555   The @{tool_def "export"} tool retrieves theory exports from the session
   555   The @{tool_def "export"} tool retrieves theory exports from the session
   556   database. Its command-line usage is: @{verbatim [display]
   556   database. Its command-line usage is: @{verbatim [display]
   557 \<open>Usage: isabelle export [OPTIONS] SESSION
   557 \<open>Usage: isabelle export [OPTIONS] SESSION
   558 
   558 
   559   Options are:
   559   Options are:
   560     -D DIR       target directory for exported files (default: "export")
   560     -O DIR       output directory for exported files (default: "export")
   561     -d DIR       include session directory
   561     -d DIR       include session directory
   562     -l           list exports
   562     -l           list exports
   563     -n           no build of session
   563     -n           no build of session
   564     -o OPTION    override Isabelle system OPTION (via NAME=VAL or NAME)
   564     -o OPTION    override Isabelle system OPTION (via NAME=VAL or NAME)
   565     -s           system build mode for session image
   565     -s           system build mode for session image
   588   separators ``\<^verbatim>\<open>:\<close>'' and ``\<^verbatim>\<open>/\<close>''; the wild card \<^verbatim>\<open>**\<close> matches over directory
   588   separators ``\<^verbatim>\<open>:\<close>'' and ``\<^verbatim>\<open>/\<close>''; the wild card \<^verbatim>\<open>**\<close> matches over directory
   589   name hierarchies separated by ``\<^verbatim>\<open>/\<close>''. Thus the pattern ``\<^verbatim>\<open>*:**\<close>'' matches
   589   name hierarchies separated by ``\<^verbatim>\<open>/\<close>''. Thus the pattern ``\<^verbatim>\<open>*:**\<close>'' matches
   590   \<^emph>\<open>all\<close> theory exports. Multiple options \<^verbatim>\<open>-x\<close> refer to the union of all
   590   \<^emph>\<open>all\<close> theory exports. Multiple options \<^verbatim>\<open>-x\<close> refer to the union of all
   591   specified patterns.
   591   specified patterns.
   592 
   592 
   593   Option \<^verbatim>\<open>-D\<close> specifies an alternative base directory for option \<^verbatim>\<open>-x\<close>: the
   593   Option \<^verbatim>\<open>-O\<close> specifies an alternative output directory for option \<^verbatim>\<open>-x\<close>: the
   594   default is \<^verbatim>\<open>export\<close> within the current directory. Each theory creates its
   594   default is \<^verbatim>\<open>export\<close> within the current directory. Each theory creates its
   595   own sub-directory hierarchy, using the session-qualified theory name.
   595   own sub-directory hierarchy, using the session-qualified theory name.
   596 \<close>
   596 \<close>
   597 
   597 
   598 end
   598 end