src/HOL/Analysis/ex/Approximations.thy
changeset 82967 73af47bc277c
parent 72222 01397b6e5eb0
--- a/src/HOL/Analysis/ex/Approximations.thy	Thu Aug 07 20:33:28 2025 +0200
+++ b/src/HOL/Analysis/ex/Approximations.thy	Thu Aug 07 21:40:03 2025 +0200
@@ -472,7 +472,7 @@
 ML \<open>
   fun machin_term_conv ctxt ct =
     let
-      val ctxt' = ctxt addsimps @{thms arctan_double' arctan_add_small}
+      val ctxt' = ctxt |> Simplifier.add_simps @{thms arctan_double' arctan_add_small}
     in
       case Thm.term_of ct of
         Const (\<^const_name>\<open>MACHIN_TAG\<close>, _) $ _ $
@@ -494,7 +494,7 @@
         Local_Defs.unfold_tac ctxt
           @{thms tag_machin[THEN eq_reflection] numeral_horner_MACHIN_TAG[THEN eq_reflection]}
         THEN REPEAT (CHANGED (HEADGOAL (CONVERSION conv))))
-      THEN' Simplifier.simp_tac (ctxt addsimps @{thms arctan_add_small arctan_diff_small})
+      THEN' Simplifier.simp_tac (ctxt |> Simplifier.add_simps @{thms arctan_add_small arctan_diff_small})
     end
 \<close>