src/HOL/Library/ListVector.thy
changeset 81142 6ad2c917dd2e
parent 80914 d97fdabd9e2b
child 81804 5a2e05eb7001
--- a/src/HOL/Library/ListVector.thy	Wed Oct 09 22:01:33 2024 +0200
+++ b/src/HOL/Library/ListVector.thy	Wed Oct 09 23:38:29 2024 +0200
@@ -99,8 +99,8 @@
 
 subsection "Inner product"
 
-definition iprod :: "'a::ring list \<Rightarrow> 'a list \<Rightarrow> 'a" (\<open>\<langle>_,_\<rangle>\<close>) where
-"\<langle>xs,ys\<rangle> = (\<Sum>(x,y) \<leftarrow> zip xs ys. x*y)"
+definition iprod :: "'a::ring list \<Rightarrow> 'a list \<Rightarrow> 'a" (\<open>(\<open>open_block notation=\<open>mixfix iprod\<close>\<close>\<langle>_,_\<rangle>)\<close>)
+  where "\<langle>xs,ys\<rangle> = (\<Sum>(x,y) \<leftarrow> zip xs ys. x*y)"
 
 lemma iprod_Nil[simp]: "\<langle>[],ys\<rangle> = 0"
 by(simp add: iprod_def)