src/HOL/Tools/Function/size.ML
changeset 35021 c839a4c670c6
parent 34974 18b41bba42b5
child 35047 1b2bae06c796
--- a/src/HOL/Tools/Function/size.ML	Sun Feb 07 19:31:55 2010 +0100
+++ b/src/HOL/Tools/Function/size.ML	Sun Feb 07 19:33:34 2010 +0100
@@ -197,7 +197,7 @@
 
     fun prove_size_eqs p size_fns size_ofp simpset =
       maps (fn (((_, (_, _, constrs)), size_const), T) =>
-        map (fn constr => Drule.standard (Skip_Proof.prove ctxt [] []
+        map (fn constr => Drule.export_without_context (Skip_Proof.prove ctxt [] []
           (gen_mk_size_eq p (AList.lookup op = (new_type_names ~~ size_fns))
              size_ofp size_const T constr)
           (fn _ => simp_tac simpset 1))) constrs)