src/Doc/Isar_Ref/HOL_Specific.thy
changeset 70276 910dc065b869
parent 70261 efbdfcaa6258
child 71567 9a29e883a934
--- a/src/Doc/Isar_Ref/HOL_Specific.thy	Tue May 21 11:47:11 2019 +0200
+++ b/src/Doc/Isar_Ref/HOL_Specific.thy	Tue May 21 11:30:30 2019 +0200
@@ -489,6 +489,7 @@
     @{method_def (HOL) relation} & : & \<open>method\<close> \\
     @{method_def (HOL) lexicographic_order} & : & \<open>method\<close> \\
     @{method_def (HOL) size_change} & : & \<open>method\<close> \\
+    @{attribute_def (HOL) termination_simp} & : & \<open>attribute\<close> \\
     @{method_def (HOL) induction_schema} & : & \<open>method\<close> \\
   \end{matharray}
 
@@ -535,6 +536,10 @@
   For local descent proofs, the @{syntax clasimpmod} modifiers are accepted
   (as for @{method auto}).
 
+  \<^descr> @{attribute (HOL) termination_simp} declares extra rules for the
+  simplifier, when invoked in termination proofs. This can be useful, e.g.,
+  for special rules involving size estimations.
+
   \<^descr> @{method (HOL) induction_schema} derives user-specified induction rules
   from well-founded induction and completeness of patterns. This factors out
   some operations that are done internally by the function package and makes