src/HOL/Computational_Algebra/Formal_Power_Series.thy
changeset 81132 dff7dfd8dce3
parent 81107 ad5fc948e053
child 82338 1eb12389c499
--- a/src/HOL/Computational_Algebra/Formal_Power_Series.thy	Tue Oct 08 16:14:36 2024 +0200
+++ b/src/HOL/Computational_Algebra/Formal_Power_Series.thy	Tue Oct 08 16:15:31 2024 +0200
@@ -6191,11 +6191,11 @@
 qed
 
 (* TODO: Figure out better notation for this thing *)
-no_notation fps_nth (infixl \<open>$\<close> 75)
-
 bundle fps_syntax
 begin
 notation fps_nth (infixl \<open>$\<close> 75)
 end
 
+unbundle no fps_syntax
+
 end