src/HOL/Library/Code_Real_Approx_By_Float.thy
changeset 69064 5840724b1d71
parent 67399 eab6ce8368fa
child 69906 55534affe445
--- a/src/HOL/Library/Code_Real_Approx_By_Float.thy	Sun Sep 23 21:49:31 2018 +0200
+++ b/src/HOL/Library/Code_Real_Approx_By_Float.thy	Mon Sep 24 14:30:09 2018 +0200
@@ -60,7 +60,7 @@
     and (OCaml) "Pervasives.( +. )"
 
 code_printing
-  constant "( * ) :: real \<Rightarrow> real \<Rightarrow> real" \<rightharpoonup>
+  constant "(*) :: real \<Rightarrow> real \<Rightarrow> real" \<rightharpoonup>
     (SML) "Real.* ((_), (_))"
     and (OCaml) "Pervasives.( *. )"