--- a/src/HOL/Decision_Procs/Approximation.thy Wed Oct 02 11:17:47 2024 +0200
+++ b/src/HOL/Decision_Procs/Approximation.thy Wed Oct 02 11:27:19 2024 +0200
@@ -1143,7 +1143,8 @@
section "Avoid pollution of name space"
-bundle floatarith_notation begin
+bundle floatarith_notation
+begin
notation Add (\<open>Add\<close>)
notation Minus (\<open>Minus\<close>)
@@ -1166,7 +1167,8 @@
end
-bundle no_floatarith_notation begin
+bundle no_floatarith_notation
+begin
no_notation Add (\<open>Add\<close>)
no_notation Minus (\<open>Minus\<close>)