--- a/src/HOL/Codegenerator_Test/Code_Test_GHC.thy Thu May 26 16:57:14 2016 +0200
+++ b/src/HOL/Codegenerator_Test/Code_Test_GHC.thy Thu May 26 17:51:22 2016 +0200
@@ -10,7 +10,7 @@
value [GHC] "14 + 7 * -12 :: integer"
-test_code -- \<open>Tests for the serialisation of @{const gcd} on @{typ integer}\<close>
+test_code \<comment> \<open>Tests for the serialisation of @{const gcd} on @{typ integer}\<close>
"gcd 15 10 = (5 :: integer)"
"gcd 15 (- 10) = (5 :: integer)"
"gcd (- 10) 15 = (5 :: integer)"