tuning
authorblanchet
Wed, 17 Dec 2014 16:51:29 +0100
changeset 59145 0e304b1568a5
parent 59144 c9b75c03de3c
child 59146 ba2a326fc271
tuning
src/HOL/Tools/BNF/bnf_lfp_size.ML
src/Pure/Tools/plugin.ML
--- a/src/HOL/Tools/BNF/bnf_lfp_size.ML	Wed Dec 17 16:10:30 2014 +0100
+++ b/src/HOL/Tools/BNF/bnf_lfp_size.ML	Wed Dec 17 16:51:29 2014 +0100
@@ -59,9 +59,6 @@
 fun mk_unabs_def_unused_0 n =
   funpow n (fn thm => thm RS @{thm fun_cong_unused_0} handle THM _ => thm RS fun_cong);
 
-val rec_o_map_simps =
-  @{thms o_def[abs_def] id_def case_prod_app case_sum_map_sum case_prod_map_prod id_bnf_def};
-
 val size_gen_o_map_simps = @{thms prod.inj_map inj_on_id snd_comp_apfst[unfolded apfst_def]};
 
 fun mk_size_gen_o_map_tac ctxt size_def rec_o_map inj_maps size_maps =
@@ -77,8 +74,8 @@
   ALLGOALS (REPEAT_DETERM o (rtac @{thm zero_less_Suc} ORELSE' rtac @{thm trans_less_add2}));
 
 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_maps = ctor_rec_o_maps, ...}, fp_nesting_bnfs,
-      live_nesting_bnfs, ...} : fp_sugar) :: _) lthy0 =
+        fp_res = {bnfs = fp_bnfs, ...}, fp_nesting_bnfs, live_nesting_bnfs, ...} : fp_sugar) :: _)
+      lthy0 =
     let
       val data = Data.get (Context.Proof lthy0);
 
--- a/src/Pure/Tools/plugin.ML	Wed Dec 17 16:10:30 2014 +0100
+++ b/src/Pure/Tools/plugin.ML	Wed Dec 17 16:51:29 2014 +0100
@@ -186,4 +186,3 @@
   #> perhaps consolidate';
 
 end;
-