made destructor-view tactic more robust (by Jan van Brügge)
authortraytel
Tue, 13 Feb 2024 14:31:09 +0100
changeset 79595 3e27ab965a36
parent 79591 6e5f40cfa877
child 79596 1b3770369ee7
made destructor-view tactic more robust (by Jan van Brügge)
src/HOL/Tools/BNF/bnf_gfp_rec_sugar_tactics.ML
--- a/src/HOL/Tools/BNF/bnf_gfp_rec_sugar_tactics.ML	Tue Feb 13 12:23:12 2024 +0100
+++ b/src/HOL/Tools/BNF/bnf_gfp_rec_sugar_tactics.ML	Tue Feb 13 14:31:09 2024 +0100
@@ -139,6 +139,8 @@
     eresolve_tac ctxt (map (fn thm => thm RS neq_eq_eq_contradict) distincts) THEN'
     assume_tac ctxt ORELSE'
     etac ctxt notE THEN' assume_tac ctxt ORELSE'
+    (CHANGED o SELECT_GOAL (unfold_thms_tac ctxt (
+      map (Local_Defs.unfold0 ctxt @{thms id_def[symmetric]}) map_ident0s @ map_comps))) ORELSE'
     (CHANGED o SELECT_GOAL (unfold_thms_tac ctxt (@{thms fst_conv snd_conv id_def comp_def split_def
          sum.case sum.sel sum.distinct[THEN eq_False[THEN iffD2]]} @
        map_ident0s @ map_comps))) ORELSE'