src/Pure/codegen.ML
changeset 43324 2b47822868e4
parent 42427 5611f178a747
child 43955 efc6f0a81c36
--- a/src/Pure/codegen.ML	Thu Jun 09 15:38:49 2011 +0200
+++ b/src/Pure/codegen.ML	Thu Jun 09 16:34:49 2011 +0200
@@ -273,7 +273,7 @@
 
 fun preprocess_term thy t =
   let
-    val x = Free (Name.variant (OldTerm.add_term_names (t, [])) "x", fastype_of t);
+    val x = Free (singleton (Name.variant_list (OldTerm.add_term_names (t, []))) "x", fastype_of t);
     (* fake definition *)
     val eq = Skip_Proof.make_thm thy (Logic.mk_equals (x, t));
     fun err () = error "preprocess_term: bad preprocessor"