src/Pure/codegen.ML
changeset 20548 8ef25fe585a8
parent 20286 4cf8e86a2d29
child 20599 65bd267ae23f
--- a/src/Pure/codegen.ML	Fri Sep 15 22:56:08 2006 +0200
+++ b/src/Pure/codegen.ML	Fri Sep 15 22:56:13 2006 +0200
@@ -1010,7 +1010,7 @@
       | strip t = t;
     val (gi, frees) = Logic.goal_params
       (prop_of (snd (snd (Proof.get_goal (Toplevel.proof_of st))))) i;
-    val gi' = ObjectLogic.atomize_term thy (map_term_types
+    val gi' = ObjectLogic.atomize_term thy (map_types
       (map_type_tfree (fn p as (s, _) =>
         the_default (the_default (TFree p) default_type)
           (AList.lookup (op =) tvinsts s))) (subst_bounds (frees, strip gi)));