merged
authortraytel
Thu, 06 Oct 2016 13:34:00 +0200
changeset 64068 3a506cb576d3
parent 64067 6855c2f7aa6a (diff)
parent 64064 f3ac9153bc0d (current diff)
child 64069 800174511cc3
merged
--- a/src/HOL/Tools/BNF/bnf_fp_def_sugar.ML	Thu Oct 06 11:27:28 2016 +0200
+++ b/src/HOL/Tools/BNF/bnf_fp_def_sugar.ML	Thu Oct 06 13:34:00 2016 +0200
@@ -847,7 +847,7 @@
           in
             Goal.prove_sorry lthy vars [] goal (fn {context = ctxt, prems = _} =>
               mk_map_tac ctxt abs_inverses pre_map_def dtor_ctor fp_map_thm'
-                live_nesting_map_ident0s ctr_defs' extra_unfolds_map)
+                live_nesting_map_id0s ctr_defs' extra_unfolds_map)
             |> Thm.close_derivation
             |> Conjunction.elim_balanced (length goals)
           end;
--- a/src/HOL/Tools/BNF/bnf_fp_def_sugar_tactics.ML	Thu Oct 06 11:27:28 2016 +0200
+++ b/src/HOL/Tools/BNF/bnf_fp_def_sugar_tactics.ML	Thu Oct 06 13:34:00 2016 +0200
@@ -392,12 +392,12 @@
       (1 upto nn) ns pre_rel_defs fp_abs_inverses abs_inverses dtor_ctors exhausts ctr_defss discsss
       selsss));
 
-fun mk_map_tac ctxt abs_inverses pre_map_def dtor_ctor fp_map' live_nesting_map_ident0s ctr_defs'
+fun mk_map_tac ctxt abs_inverses pre_map_def dtor_ctor fp_map' live_nesting_map_id0s ctr_defs'
     extra_unfolds =
   TRYALL Goal.conjunction_tac THEN
   unfold_thms_tac ctxt (pre_map_def :: dtor_ctor :: fp_map' :: abs_inverses @
-    live_nesting_map_ident0s @ ctr_defs' @ extra_unfolds @ sumprod_thms_map @
-    @{thms o_def[abs_def] id_def}) THEN
+    live_nesting_map_id0s @ ctr_defs' @ extra_unfolds @ sumprod_thms_map @
+    @{thms o_apply id_apply id_o o_id}) THEN
   ALLGOALS (rtac ctxt refl);
 
 fun mk_map_disc_iff_tac ctxt ct exhaust discs maps =