diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Analysis/Finite_Cartesian_Product.thy --- a/src/HOL/Analysis/Finite_Cartesian_Product.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Analysis/Finite_Cartesian_Product.thy Fri Sep 20 19:51:08 2024 +0200 @@ -22,14 +22,14 @@ bundle vec_syntax begin notation - vec_nth (infixl "$" 90) and - vec_lambda (binder "\" 10) + vec_nth (infixl \$\ 90) and + vec_lambda (binder \\\ 10) end bundle no_vec_syntax begin no_notation - vec_nth (infixl "$" 90) and - vec_lambda (binder "\" 10) + vec_nth (infixl \$\ 90) and + vec_lambda (binder \\\ 10) end unbundle vec_syntax @@ -39,7 +39,7 @@ \<^item> \'a^'b\ becomes \('a, 'b::finite) vec\ \<^item> \'a^'b::_\ becomes \('a, 'b) vec\ without extra sort-constraint \ -syntax "_vec_type" :: "type \ type \ type" (infixl "^" 15) +syntax "_vec_type" :: "type \ type \ type" (infixl \^\ 15) syntax_types "_vec_type" \ vec parse_translation \ let @@ -283,7 +283,7 @@ text\Also the scalar-vector multiplication.\ -definition vector_scalar_mult:: "'a::times \ 'a ^ 'n \ 'a ^ 'n" (infixl "*s" 70) +definition vector_scalar_mult:: "'a::times \ 'a ^ 'n \ 'a ^ 'n" (infixl \*s\ 70) where "c *s x = (\ i. c * (x$i))" text \scalar product\ @@ -986,15 +986,15 @@ by (simp add: map_matrix_def) definition\<^marker>\tag important\ matrix_matrix_mult :: "('a::semiring_1) ^'n^'m \ 'a ^'p^'n \ 'a ^ 'p ^'m" - (infixl "**" 70) + (infixl \**\ 70) where "m ** m' == (\ i j. sum (\k. ((m$i)$k) * ((m'$k)$j)) (UNIV :: 'n set)) ::'a ^ 'p ^'m" definition\<^marker>\tag important\ matrix_vector_mult :: "('a::semiring_1) ^'n^'m \ 'a ^'n \ 'a ^ 'm" - (infixl "*v" 70) + (infixl \*v\ 70) where "m *v x \ (\ i. sum (\j. ((m$i)$j) * (x$j)) (UNIV ::'n set)) :: 'a^'m" definition\<^marker>\tag important\ vector_matrix_mult :: "'a ^ 'm \ ('a::semiring_1) ^'n^'m \ 'a ^'n " - (infixl "v*" 70) + (infixl \v*\ 70) where "v v* m == (\ j. sum (\i. ((m$i)$j) * (v$i)) (UNIV :: 'm set)) :: 'a^'n" definition\<^marker>\tag unimportant\ "(mat::'a::zero => 'a ^'n^'n) k = (\ i j. if i = j then k else 0)"