src/Doc/Isar_Ref/Inner_Syntax.thy
changeset 81274 5e4a3237fc86
parent 81178 8e7bd0566759
child 81276 59b5696b00a3
--- a/src/Doc/Isar_Ref/Inner_Syntax.thy	Sun Oct 27 12:13:34 2024 +0100
+++ b/src/Doc/Isar_Ref/Inner_Syntax.thy	Sun Oct 27 12:23:48 2024 +0100
@@ -94,16 +94,12 @@
     \<^descr> @{command "print_state"} prints the current proof state (if present),
     including current facts and goals.
 
-  All of the diagnostic commands above admit a list of \<open>modes\<close> to be
-  specified, which is appended to the current print mode; see also
-  \secref{sec:print-modes}. Thus the output behavior may be modified according
-  particular print mode features. For example, @{command
-  "print_state"}~\<open>(latex)\<close> prints the current proof state with mathematical
-  symbols and special characters represented in {\LaTeX} source, according to
-  the Isabelle style \<^cite>\<open>"isabelle-system"\<close>.
-
-  Note that antiquotations (cf.\ \secref{sec:antiq}) provide a more systematic
-  way to include formal items into the printed text document.
+  The diagnostic commands above accept an optional list of \<open>modes\<close>, which is
+  appended to the current print mode; see also \secref{sec:print-modes}. Thus
+  the output behavior may be modified according particular print mode
+  features. For example, @{command "thm"}~\<^verbatim>\<open>("") symmetric\<close> prints a theorem
+  without any special markup, bypassing the print mode setup of the Prover
+  IDE.
 \<close>