src/Doc/JEdit/JEdit.thy
changeset 62154 b855771b3979
parent 62039 a77f4a9037d4
child 62183 7fdcc25c5c35
equal deleted inserted replaced
62153:df566b87e269 62154:b855771b3979
   946   \secref{sec:tooltips-hyperlinks}), or clicked directly to initiate certain
   946   \secref{sec:tooltips-hyperlinks}), or clicked directly to initiate certain
   947   actions (see \secref{sec:auto-tools} and \secref{sec:sledgehammer}).
   947   actions (see \secref{sec:auto-tools} and \secref{sec:sledgehammer}).
   948 \<close>
   948 \<close>
   949 
   949 
   950 
   950 
       
   951 section \<open>Proof state output \label{sec:state-output}\<close>
       
   952 
       
   953 text \<open>
       
   954   FIXME
       
   955   \figref{fig:output-and-state} versus \figref{fig:output-including-state}
       
   956 
       
   957   \begin{figure}[htb]
       
   958   \begin{center}
       
   959   \includegraphics[scale=0.333]{output-and-state}
       
   960   \end{center}
       
   961   \caption{Separate proof state display (right) and other output (bottom).}
       
   962   \label{fig:output-and-state}
       
   963   \end{figure}
       
   964 
       
   965   \begin{figure}[htb]
       
   966   \begin{center}
       
   967   \includegraphics[scale=0.333]{output-including-state}
       
   968   \end{center}
       
   969   \caption{Proof state display within the regular output panel}
       
   970   \label{fig:output-including-state}
       
   971   \end{figure}
       
   972 \<close>
       
   973 
   951 section \<open>Query \label{sec:query}\<close>
   974 section \<open>Query \label{sec:query}\<close>
   952 
   975 
   953 text \<open>
   976 text \<open>
   954   The \<^emph>\<open>Query\<close> panel provides various GUI forms to request extra information
   977   The \<^emph>\<open>Query\<close> panel provides various GUI forms to request extra information
   955   from the prover. In old times the user would have issued some diagnostic
   978   from the prover. In old times the user would have issued some diagnostic
   965 
   988 
   966   \begin{figure}[htb]
   989   \begin{figure}[htb]
   967   \begin{center}
   990   \begin{center}
   968   \includegraphics[scale=0.333]{query}
   991   \includegraphics[scale=0.333]{query}
   969   \end{center}
   992   \end{center}
   970   \caption{An instance of the Query panel}
   993   \caption{An instance of the Query panel: find theorems}
   971   \label{fig:query}
   994   \label{fig:query}
   972   \end{figure}
   995   \end{figure}
   973 
   996 
   974   \<^medskip>
   997   \<^medskip>
   975   The following GUI elements are common to all query modes:
   998   The following GUI elements are common to all query modes:
  1653   proofs. The alternative mode \<^verbatim>\<open>sidekick\<close> uses the document structure of the
  1676   proofs. The alternative mode \<^verbatim>\<open>sidekick\<close> uses the document structure of the
  1654   SideKick parser, as explained above.
  1677   SideKick parser, as explained above.
  1655 \<close>
  1678 \<close>
  1656 
  1679 
  1657 
  1680 
       
  1681 section \<open>Markdown structure\<close>
       
  1682 
       
  1683 text \<open>
       
  1684   FIXME
       
  1685   \figref{fig:markdown-document}
       
  1686 
       
  1687   \begin{figure}[htb]
       
  1688   \begin{center}
       
  1689   \includegraphics[scale=0.333]{markdown-document}
       
  1690   \end{center}
       
  1691   \caption{Markdown structure within document text}
       
  1692   \label{fig:markdown-document}
       
  1693   \end{figure}
       
  1694 \<close>
       
  1695 
       
  1696 
  1658 section \<open>Citations and Bib{\TeX} entries\<close>
  1697 section \<open>Citations and Bib{\TeX} entries\<close>
  1659 
  1698 
  1660 text \<open>
  1699 text \<open>
  1661   Citations are managed by {\LaTeX} and Bib{\TeX} in \<^verbatim>\<open>.bib\<close> files. The
  1700   Citations are managed by {\LaTeX} and Bib{\TeX} in \<^verbatim>\<open>.bib\<close> files. The
  1662   Isabelle session build process and the @{tool latex} tool @{cite
  1701   Isabelle session build process and the @{tool latex} tool @{cite
  1692   \label{fig:bibtex-mode}
  1731   \label{fig:bibtex-mode}
  1693   \end{figure}
  1732   \end{figure}
  1694 \<close>
  1733 \<close>
  1695 
  1734 
  1696 
  1735 
       
  1736 chapter \<open>ML debugger\<close>
       
  1737 
       
  1738 text \<open>
       
  1739   FIXME
       
  1740   \figref{fig:ml-debugger}
       
  1741 
       
  1742   \begin{figure}[htb]
       
  1743   \begin{center}
       
  1744   \includegraphics[scale=0.333]{ml-debugger}
       
  1745   \end{center}
       
  1746   \caption{ML debugger}
       
  1747   \label{fig:ml-debugger}
       
  1748   \end{figure}
       
  1749 \<close>
       
  1750 
       
  1751 
  1697 chapter \<open>Miscellaneous tools\<close>
  1752 chapter \<open>Miscellaneous tools\<close>
  1698 
  1753 
  1699 section \<open>Timing\<close>
  1754 section \<open>Timing\<close>
  1700 
  1755 
  1701 text \<open>
  1756 text \<open>