diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Algebra/Indexed_Polynomials.thy --- a/src/HOL/Algebra/Indexed_Polynomials.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Algebra/Indexed_Polynomials.thy Fri Sep 20 19:51:08 2024 +0200 @@ -23,13 +23,13 @@ definition (in ring) indexed_const :: "'a \ ('c multiset \ 'a)" where "indexed_const k = (\m. if m = {#} then k else \)" -definition (in ring) indexed_pmult :: "('c multiset \ 'a) \ 'c \ ('c multiset \ 'a)" (infixl "\" 65) +definition (in ring) indexed_pmult :: "('c multiset \ 'a) \ 'c \ ('c multiset \ 'a)" (infixl \\\ 65) where "indexed_pmult P i = (\m. if i \# m then P (m - {# i #}) else \)" -definition (in ring) indexed_padd :: "_ \ _ \ ('c multiset \ 'a)" (infixl "\" 65) +definition (in ring) indexed_padd :: "_ \ _ \ ('c multiset \ 'a)" (infixl \\\ 65) where "indexed_padd P Q = (\m. (P m) \ (Q m))" -definition (in ring) indexed_var :: "'c \ ('c multiset \ 'a)" ("\\") +definition (in ring) indexed_var :: "'c \ ('c multiset \ 'a)" (\\\\) where "indexed_var i = (indexed_const \) \ i" definition (in ring) index_free :: "('c multiset \ 'a) \ 'c \ bool" @@ -38,7 +38,7 @@ definition (in ring) carrier_coeff :: "('c multiset \ 'a) \ bool" where "carrier_coeff P \ (\m. P m \ carrier R)" -inductive_set (in ring) indexed_pset :: "'c set \ 'a set \ ('c multiset \ 'a) set" ("_ [\\]" 80) +inductive_set (in ring) indexed_pset :: "'c set \ 'a set \ ('c multiset \ 'a) set" (\_ [\\]\ 80) for I and K where indexed_const: "k \ K \ indexed_const k \ (K[\\<^bsub>I\<^esub>])" | indexed_padd: "\ P \ (K[\\<^bsub>I\<^esub>]); Q \ (K[\\<^bsub>I\<^esub>]) \ \ P \ Q \ (K[\\<^bsub>I\<^esub>])"