src/HOL/Computational_Algebra/Formal_Laurent_Series.thy
changeset 81132 dff7dfd8dce3
parent 81107 ad5fc948e053
equal deleted inserted replaced
81131:bad7156a7814 81132:dff7dfd8dce3
  4599   unfolding open_dist subset_eq by simp
  4599   unfolding open_dist subset_eq by simp
  4600 
  4600 
  4601 
  4601 
  4602 subsection \<open>Notation\<close>
  4602 subsection \<open>Notation\<close>
  4603 
  4603 
  4604 no_notation fls_nth (infixl \<open>$$\<close> 75)
       
  4605 
       
  4606 bundle fps_syntax
  4604 bundle fps_syntax
  4607 begin
  4605 begin
  4608 notation fls_nth (infixl \<open>$$\<close> 75)
  4606 notation fls_nth (infixl \<open>$$\<close> 75)
  4609 end
  4607 end
  4610 
  4608 
       
  4609 unbundle no fps_syntax
       
  4610 
  4611 end
  4611 end