src/Doc/IsarImplementation/Logic.thy
changeset 56243 2e10a36b8d46
parent 55837 154855d9a564
equal deleted inserted replaced
56242:d0a9100a5a38 56243:2e10a36b8d46
   848   @{text "\<turnstile> A &&& B \<equiv> (\<And>C. (A \<Longrightarrow> B \<Longrightarrow> C) \<Longrightarrow> C)"} \\[1ex]
   848   @{text "\<turnstile> A &&& B \<equiv> (\<And>C. (A \<Longrightarrow> B \<Longrightarrow> C) \<Longrightarrow> C)"} \\[1ex]
   849   @{text "prop :: prop \<Rightarrow> prop"} & (prefix @{text "#"}, suppressed) \\
   849   @{text "prop :: prop \<Rightarrow> prop"} & (prefix @{text "#"}, suppressed) \\
   850   @{text "#A \<equiv> A"} \\[1ex]
   850   @{text "#A \<equiv> A"} \\[1ex]
   851   @{text "term :: \<alpha> \<Rightarrow> prop"} & (prefix @{text "TERM"}) \\
   851   @{text "term :: \<alpha> \<Rightarrow> prop"} & (prefix @{text "TERM"}) \\
   852   @{text "term x \<equiv> (\<And>A. A \<Longrightarrow> A)"} \\[1ex]
   852   @{text "term x \<equiv> (\<And>A. A \<Longrightarrow> A)"} \\[1ex]
   853   @{text "TYPE :: \<alpha> itself"} & (prefix @{text "TYPE"}) \\
   853   @{text "type :: \<alpha> itself"} & (prefix @{text "TYPE"}) \\
   854   @{text "(unspecified)"} \\
   854   @{text "(unspecified)"} \\
   855   \end{tabular}
   855   \end{tabular}
   856   \caption{Definitions of auxiliary connectives}\label{fig:pure-aux}
   856   \caption{Definitions of auxiliary connectives}\label{fig:pure-aux}
   857   \end{center}
   857   \end{center}
   858   \end{figure}
   858   \end{figure}