src/HOL/Quotient_Examples/Quotient_Rat.thy
changeset 69064 5840724b1d71
parent 67399 eab6ce8368fa
--- a/src/HOL/Quotient_Examples/Quotient_Rat.thy	Sun Sep 23 21:49:31 2018 +0200
+++ b/src/HOL/Quotient_Examples/Quotient_Rat.thy	Mon Sep 24 14:30:09 2018 +0200
@@ -41,7 +41,7 @@
   "times_rat_raw (a :: int, b :: int) (c, d) = (a * c, b * d)"
 
 quotient_definition
-  "(( * )) :: (rat \<Rightarrow> rat \<Rightarrow> rat)" is times_rat_raw by (auto simp add: mult.assoc mult.left_commute)
+  "((*)) :: (rat \<Rightarrow> rat \<Rightarrow> rat)" is times_rat_raw by (auto simp add: mult.assoc mult.left_commute)
 
 fun plus_rat_raw where
   "plus_rat_raw (a :: int, b :: int) (c, d) = (a * d + c * b, b * d)"