diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Library/ListVector.thy --- a/src/HOL/Library/ListVector.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Library/ListVector.thy Fri Sep 20 19:51:08 2024 +0200 @@ -12,7 +12,7 @@ text\Multiplication with a scalar:\ -abbreviation scale :: "('a::times) \ 'a list \ 'a list" (infix "*\<^sub>s" 70) +abbreviation scale :: "('a::times) \ 'a list \ 'a list" (infix \*\<^sub>s\ 70) where "x *\<^sub>s xs \ map ((*) x) xs" lemma scale1[simp]: "(1::'a::monoid_mult) *\<^sub>s xs = xs" @@ -99,7 +99,7 @@ subsection "Inner product" -definition iprod :: "'a::ring list \ 'a list \ 'a" ("\_,_\") where +definition iprod :: "'a::ring list \ 'a list \ 'a" (\\_,_\\) where "\xs,ys\ = (\(x,y) \ zip xs ys. x*y)" lemma iprod_Nil[simp]: "\[],ys\ = 0"