diff -r cdfa8f027bb9 -r e2ad50885887 src/Doc/System/Sessions.thy --- a/src/Doc/System/Sessions.thy Tue Apr 28 19:50:36 2020 +0200 +++ b/src/Doc/System/Sessions.thy Tue Apr 28 21:47:22 2020 +0200 @@ -709,4 +709,50 @@ sessions, notably from the Archive of Formal Proofs. \ + +section \Explore sessions structure\ + +text \ + The @{tool_def "sessions"} tool explores the sessions structure. Its + command-line usage is: + @{verbatim [display] +\Usage: isabelle sessions [OPTIONS] [SESSIONS ...] + + Options are: + -B NAME include session NAME and all descendants + -D DIR include session directory and select its sessions + -R refer to requirements of selected sessions + -X NAME exclude sessions from group NAME and all descendants + -a select all sessions + -d DIR include session directory + -g NAME select session group NAME + -x NAME exclude session NAME and all descendants + + Explore the structure of Isabelle sessions and print result names in + topological order (on stdout).\} + + Arguments and options for session selection resemble @{tool build} + (\secref{sec:tool-build}). +\ + + +subsubsection \Examples\ + +text \ + All sessions of the Isabelle distribution: + @{verbatim [display] \isabelle sessions -a\} + + \<^medskip> + Sessions that are based on \<^verbatim>\ZF\ (and required by it): + @{verbatim [display] \isabelle sessions -B ZF\} + + \<^medskip> + All sessions of Isabelle/AFP (based in directory \<^path>\AFP\): + @{verbatim [display] \isabelle sessions -D AFP/thys\} + + \<^medskip> + Sessions required by Isabelle/AFP (based in directory \<^path>\AFP\): + @{verbatim [display] \isabelle sessions -R -D AFP/thys\} +\ + end