src/Doc/Functions/Functions.thy
changeset 70276 910dc065b869
parent 69597 ff784d5a5bfb
child 76649 9a6cb5ecc183
equal deleted inserted replaced
70275:91a2f79b546b 70276:910dc065b869
   343   occur in sequence).
   343   occur in sequence).
   344   \end{itemize}
   344   \end{itemize}
   345 
   345 
   346   Loading the theory \<open>Multiset\<close> makes the \<open>size_change\<close>
   346   Loading the theory \<open>Multiset\<close> makes the \<open>size_change\<close>
   347   method a bit stronger: it can then use multiset orders internally.
   347   method a bit stronger: it can then use multiset orders internally.
       
   348 \<close>
       
   349 
       
   350 subsection \<open>Configuring simplification rules for termination proofs\<close>
       
   351 
       
   352 text \<open>
       
   353   Since both \<open>lexicographic_order\<close> and \<open>size_change\<close> rely on the simplifier internally,
       
   354   there can sometimes be the need for adding additional simp rules to them.
       
   355   This can be done either as arguments to the methods themselves, or globally via the
       
   356   theorem attribute \<open>termination_simp\<close>, which is useful in rare cases.
   348 \<close>
   357 \<close>
   349 
   358 
   350 section \<open>Mutual Recursion\<close>
   359 section \<open>Mutual Recursion\<close>
   351 
   360 
   352 text \<open>
   361 text \<open>