src/HOL/Library/ListVector.thy
changeset 67399 eab6ce8368fa
parent 67006 b1278ed3cd46
child 69064 5840724b1d71
--- a/src/HOL/Library/ListVector.thy	Wed Jan 10 15:21:49 2018 +0100
+++ b/src/HOL/Library/ListVector.thy	Wed Jan 10 15:25:09 2018 +0100
@@ -13,7 +13,7 @@
 text\<open>Multiplication with a scalar:\<close>
 
 abbreviation scale :: "('a::times) \<Rightarrow> 'a list \<Rightarrow> 'a list" (infix "*\<^sub>s" 70)
-where "x *\<^sub>s xs \<equiv> map (op * x) xs"
+where "x *\<^sub>s xs \<equiv> map (( * ) x) xs"
 
 lemma scale1[simp]: "(1::'a::monoid_mult) *\<^sub>s xs = xs"
 by (induct xs) simp_all
@@ -31,7 +31,7 @@
 begin
 
 definition
-  list_add_def: "op + = zipwith0 (op +)"
+  list_add_def: "(+) = zipwith0 (+)"
 
 instance ..
 
@@ -51,7 +51,7 @@
 begin
 
 definition
-  list_diff_def: "op - = zipwith0 (op -)"
+  list_diff_def: "(-) = zipwith0 (-)"
 
 instance ..