doc-src/IsarImplementation/Thy/Logic.thy
changeset 46254 e18ccb00fb8f
parent 46253 3e427a12f0f3
child 46256 bc874d2ee55a
equal deleted inserted replaced
46253:3e427a12f0f3 46254:e18ccb00fb8f
   828   \end{description}
   828   \end{description}
   829 
   829 
   830 *}
   830 *}
   831 
   831 
   832 
   832 
   833 subsection {* Auxiliary definitions \label{sec:logic-aux} *}
   833 subsection {* Auxiliary connectives \label{sec:logic-aux} *}
   834 
   834 
   835 text {*
   835 text {* Theory @{text "Pure"} provides a few auxiliary connectives
   836   Theory @{text "Pure"} provides a few auxiliary definitions, see
   836   that are defined on top of the primitive ones, see
   837   \figref{fig:pure-aux}.  These special constants are normally not
   837   \figref{fig:pure-aux}.  These special constants are useful in
   838   exposed to the user, but appear in internal encodings.
   838   certain internal encodings, and are normally not directly exposed to
       
   839   the user.
   839 
   840 
   840   \begin{figure}[htb]
   841   \begin{figure}[htb]
   841   \begin{center}
   842   \begin{center}
   842   \begin{tabular}{ll}
   843   \begin{tabular}{ll}
   843   @{text "conjunction :: prop \<Rightarrow> prop \<Rightarrow> prop"} & (infix @{text "&&&"}) \\
   844   @{text "conjunction :: prop \<Rightarrow> prop \<Rightarrow> prop"} & (infix @{text "&&&"}) \\