src/HOL/Tools/record.ML
changeset 46893 d5bb4c212df1
parent 46708 b138dee7bed3
child 46949 94aa7b81bcf6
equal deleted inserted replaced
46892:9920f9a75b51 46893:d5bb4c212df1
  2074     val record_ss = get_simpset defs_thy;
  2074     val record_ss = get_simpset defs_thy;
  2075     val sel_upd_ss = record_ss addsimps (sel_defs @ accessor_thms @ upd_defs @ updator_thms);
  2075     val sel_upd_ss = record_ss addsimps (sel_defs @ accessor_thms @ upd_defs @ updator_thms);
  2076 
  2076 
  2077     val (sel_convs, upd_convs) =
  2077     val (sel_convs, upd_convs) =
  2078       timeit_msg ctxt "record sel_convs/upd_convs proof:" (fn () =>
  2078       timeit_msg ctxt "record sel_convs/upd_convs proof:" (fn () =>
  2079         Par_List.map (fn prop =>
  2079         grouped 10 Par_List.map (fn prop =>
  2080           Skip_Proof.prove_global defs_thy [] [] prop
  2080           Skip_Proof.prove_global defs_thy [] [] prop
  2081             (K (ALLGOALS (asm_full_simp_tac sel_upd_ss)))) (sel_conv_props @ upd_conv_props))
  2081             (K (ALLGOALS (asm_full_simp_tac sel_upd_ss)))) (sel_conv_props @ upd_conv_props))
  2082       |> chop (length sel_conv_props);
  2082       |> chop (length sel_conv_props);
  2083 
  2083 
  2084     val (fold_congs, unfold_congs) = timeit_msg ctxt "record upd fold/unfold congs:" (fn () =>
  2084     val (fold_congs, unfold_congs) = timeit_msg ctxt "record upd fold/unfold congs:" (fn () =>