src/Doc/Isar_Ref/HOL_Specific.thy
changeset 75878 fcd118d9242f
parent 75415 e0fa345f1aab
child 76063 24c9f56aa035
--- a/src/Doc/Isar_Ref/HOL_Specific.thy	Fri Aug 19 05:49:07 2022 +0000
+++ b/src/Doc/Isar_Ref/HOL_Specific.thy	Fri Aug 19 05:49:09 2022 +0000
@@ -2003,7 +2003,7 @@
   \begin{matharray}{rcl}
     @{method_def (HOL) arith} & : & \<open>method\<close> \\
     @{attribute_def (HOL) arith} & : & \<open>attribute\<close> \\
-    @{attribute_def (HOL) arith_split} & : & \<open>attribute\<close> \\
+    @{attribute_def (HOL) linarith_split} & : & \<open>attribute\<close> \\
   \end{matharray}
 
   \<^descr> @{method (HOL) arith} decides linear arithmetic problems (on types \<open>nat\<close>,
@@ -2013,7 +2013,7 @@
   \<^descr> @{attribute (HOL) arith} declares facts that are supplied to the
   arithmetic provers implicitly.
 
-  \<^descr> @{attribute (HOL) arith_split} attribute declares case split rules to be
+  \<^descr> @{attribute (HOL) linarith_split} attribute declares case split rules to be
   expanded before @{method (HOL) arith} is invoked.