src/HOL/Bali/Term.thy
changeset 74887 56247fdb8bbb
parent 69597 ff784d5a5bfb
--- a/src/HOL/Bali/Term.thy	Mon Dec 06 15:10:15 2021 +0100
+++ b/src/HOL/Bali/Term.thy	Mon Dec 06 15:34:54 2021 +0100
@@ -110,7 +110,7 @@
                | UNot     \<comment> \<open>{\tt !} logical complement\<close>
 
 \<comment> \<open>function codes for binary operations\<close>
-datatype binop = Mul     \<comment> \<open>{\tt * }   multiplication\<close>
+datatype binop = Mul     \<comment> \<open>{\tt *}   multiplication\<close>
                | Div     \<comment> \<open>{\tt /}   division\<close>
                | Mod     \<comment> \<open>{\tt \%}   remainder\<close>
                | Plus    \<comment> \<open>{\tt +}   addition\<close>