src/HOL/Codegenerator_Test/Code_Test_OCaml.thy
changeset 69597 ff784d5a5bfb
parent 68155 8b50f29a1992
--- a/src/HOL/Codegenerator_Test/Code_Test_OCaml.thy	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/HOL/Codegenerator_Test/Code_Test_OCaml.thy	Sat Jan 05 17:24:33 2019 +0100
@@ -10,7 +10,7 @@
 
 value [OCaml] "14 + 7 * -12 :: integer"
 
-test_code \<comment> \<open>Tests for the serialisation of @{const gcd} on @{typ integer}\<close>
+test_code \<comment> \<open>Tests for the serialisation of \<^const>\<open>gcd\<close> on \<^typ>\<open>integer\<close>\<close>
   "gcd 15 10 = (5 :: integer)"
   "gcd 15 (- 10) = (5 :: integer)"
   "gcd (- 10) 15 = (5 :: integer)"