# HG changeset patch # User wenzelm # Date 1403120850 -7200 # Node ID 3bb94256e0ed46c23bbf362b39a276aaecc72e36 # Parent 06d533a24713ea24e05e05d749e270a80b25fb2b added screenshot; diff -r 06d533a24713 -r 3bb94256e0ed src/Doc/JEdit/JEdit.thy --- a/src/Doc/JEdit/JEdit.thy Wed Jun 18 21:23:10 2014 +0200 +++ b/src/Doc/JEdit/JEdit.thy Wed Jun 18 21:47:30 2014 +0200 @@ -690,13 +690,22 @@ subsection {* Theories \label{sec:theories} *} text {* - The \emph{Theories} panel (see also \figref{fig:output}) provides an + The \emph{Theories} panel (see also \figref{fig:theories}) provides an overview of the status of continuous checking of theory nodes within the document model. Unlike batch sessions of @{tool build} \cite{isabelle-sys}, theory nodes are identified by full path names; this allows to work with multiple (disjoint) Isabelle sessions simultaneously within the same editor session. + \begin{figure}[htb] + \begin{center} + \includegraphics[scale=0.333]{theories} + \end{center} + \caption{Theories panel with an overview of the document-model, and some + jEdit text areas as editable view on some of the document nodes} + \label{fig:theories} + \end{figure} + Certain events to open or update editor buffers cause Isabelle/jEdit to resolve dependencies of theory imports. The system requests to load additional files into editor buffers, in order to be included in the diff -r 06d533a24713 -r 3bb94256e0ed src/Doc/JEdit/document/theories.png Binary file src/Doc/JEdit/document/theories.png has changed diff -r 06d533a24713 -r 3bb94256e0ed src/Doc/ROOT --- a/src/Doc/ROOT Wed Jun 18 21:23:10 2014 +0200 +++ b/src/Doc/ROOT Wed Jun 18 21:47:30 2014 +0200 @@ -188,6 +188,7 @@ "root.tex" "sidekick.png" "sledgehammer.png" + "theories.png" session Sugar (doc) in "Sugar" = HOL + options [document_variants = "sugar"]