back to formal comment (see 23a380cc45f4, 3094b0edd6b5);
authorwenzelm
Mon, 20 Oct 2014 17:02:46 +0200
changeset 58719 ac4f764c5be1
parent 58718 48395c763059
child 58720 e4f4925d4a9d
back to formal comment (see 23a380cc45f4, 3094b0edd6b5);
src/HOL/Library/Code_Test.thy
--- a/src/HOL/Library/Code_Test.thy	Mon Oct 20 17:00:13 2014 +0200
+++ b/src/HOL/Library/Code_Test.thy	Mon Oct 20 17:02:46 2014 +0200
@@ -131,10 +131,10 @@
   "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)]]"
-  (*
+  -- {*
     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.
-  *)
+  *}
   "xml_of_term (Code_Evaluation.Free x ty)  = [xml.tagged (STR ''1'') (Some x) (xml_of_typ ty)]"
 by(simp_all add: xml_of_term_def xml_tree_anything)