src/HOL/Tools/BNF/bnf_lfp_size.ML
changeset 58578 9ff8ca957c02
parent 58461 75ee8d49c724
child 58634 9f10d82e8188
--- a/src/HOL/Tools/BNF/bnf_lfp_size.ML	Mon Oct 06 13:36:48 2014 +0200
+++ b/src/HOL/Tools/BNF/bnf_lfp_size.ML	Mon Oct 06 13:37:38 2014 +0200
@@ -82,7 +82,7 @@
   IF_UNSOLVED (unfold_thms_tac ctxt @{thms o_def} THEN HEADGOAL (rtac refl));
 
 fun generate_datatype_size (fp_sugars as ({T = Type (_, As), BT = Type (_, Bs), fp = Least_FP,
-      fp_res = {bnfs = fp_bnfs, xtor_co_rec_o_map_thms = ctor_rec_o_maps, ...}, fp_nesting_bnfs,
+      fp_res = {bnfs = fp_bnfs, xtor_co_rec_o_maps = ctor_rec_o_maps, ...}, fp_nesting_bnfs,
       live_nesting_bnfs, ...} : fp_sugar) :: _) lthy0 =
     let
       val data = Data.get (Context.Proof lthy0);