src/HOL/Library/Code_Test.thy
changeset 61585 a9599d3d7610
parent 60500 903bb1495239
child 62597 b3f2b8c906a6
--- a/src/HOL/Library/Code_Test.thy	Thu Nov 05 10:35:37 2015 +0100
+++ b/src/HOL/Library/Code_Test.thy	Thu Nov 05 10:39:49 2015 +0100
@@ -131,7 +131,7 @@
   "xml_of_term (Code_Evaluation.Const x ty) = [xml.tagged (STR ''0'') (Some x) (xml_of_typ ty)]"
   "xml_of_term (Code_Evaluation.App t1 t2)  = [xml.tagged (STR ''5'') None [xml.node (xml_of_term t1), xml.node (xml_of_term t2)]]"
   "xml_of_term (Code_Evaluation.Abs x ty t) = [xml.tagged (STR ''4'') (Some x) [xml.node (xml_of_typ ty), xml.node (xml_of_term t)]]"
-  -- \<open>
+  \<comment> \<open>
     FIXME: @{const Code_Evaluation.Free} is used only in @{theory Quickcheck_Narrowing} to represent
     uninstantiated parameters in constructors. Here, we always translate them to @{ML Free} variables.
 \<close>