src/Doc/System/Sessions.thy
changeset 70796 2739631ac368
parent 70771 2071dbe5547d
child 70858 f76126e6a1ab
equal deleted inserted replaced
70795:a90e40118874 70796:2739631ac368
   544 \<open>Usage: isabelle dump [OPTIONS] [SESSIONS ...]
   544 \<open>Usage: isabelle dump [OPTIONS] [SESSIONS ...]
   545 
   545 
   546   Options are:
   546   Options are:
   547     -A NAMES     dump named aspects (default: ...)
   547     -A NAMES     dump named aspects (default: ...)
   548     -B NAME      include session NAME and all descendants
   548     -B NAME      include session NAME and all descendants
   549     -C           observe option dump_checkpoint for theories
       
   550     -D DIR       include session directory and select its sessions
   549     -D DIR       include session directory and select its sessions
   551     -O DIR       output directory for dumped files (default: "dump")
   550     -O DIR       output directory for dumped files (default: "dump")
   552     -R           operate on requirements of selected sessions
   551     -R           operate on requirements of selected sessions
   553     -X NAME      exclude sessions from group NAME and all descendants
   552     -X NAME      exclude sessions from group NAME and all descendants
   554     -a           select all sessions
   553     -a           select all sessions
   581   list. The default is to dump all known aspects, as given in the command-line
   580   list. The default is to dump all known aspects, as given in the command-line
   582   usage of the tool. The underlying Isabelle/Scala function
   581   usage of the tool. The underlying Isabelle/Scala function
   583   \<^verbatim>\<open>isabelle.Dump.dump()\<close> takes aspects as user-defined operations on the
   582   \<^verbatim>\<open>isabelle.Dump.dump()\<close> takes aspects as user-defined operations on the
   584   final PIDE state and document version. This allows to imitate Prover IDE
   583   final PIDE state and document version. This allows to imitate Prover IDE
   585   rendering under program control.
   584   rendering under program control.
   586 
       
   587   \<^medskip> Option \<^verbatim>\<open>-C\<close> observes option \<^verbatim>\<open>dump_checkpoint\<close> within the
       
   588   \isakeyword{theories} specification of session ROOT definitions. This helps
       
   589   to structure the load process of large collections of theories, and thus
       
   590   reduce overall resource requirements.
       
   591 \<close>
   585 \<close>
   592 
   586 
   593 
   587 
   594 subsubsection \<open>Examples\<close>
   588 subsubsection \<open>Examples\<close>
   595 
   589