src/HOL/Tools/BNF/bnf_def.ML
changeset 63399 d1742d1b7f0f
parent 63170 eae6549dbea2
child 63714 b62f4f765353
equal deleted inserted replaced
63398:6bf5a8c78175 63399:d1742d1b7f0f
  1733           in
  1733           in
  1734             Goal.prove_sorry lthy [] [] goal (fn {context = ctxt, prems = _} =>
  1734             Goal.prove_sorry lthy [] [] goal (fn {context = ctxt, prems = _} =>
  1735               unfold_thms_tac ctxt [#pred_set axioms] THEN
  1735               unfold_thms_tac ctxt [#pred_set axioms] THEN
  1736               HEADGOAL (EVERY' [REPEAT_DETERM o etac ctxt conjE,
  1736               HEADGOAL (EVERY' [REPEAT_DETERM o etac ctxt conjE,
  1737                 etac ctxt (Lazy.force map_cong) THEN_ALL_NEW
  1737                 etac ctxt (Lazy.force map_cong) THEN_ALL_NEW
  1738                   (etac ctxt bspec THEN' assume_tac ctxt)]))
  1738                   (etac ctxt @{thm bspec} THEN' assume_tac ctxt)]))
  1739             |> Thm.close_derivation
  1739             |> Thm.close_derivation
  1740           end;
  1740           end;
  1741 
  1741 
  1742         val map_cong_pred = Lazy.lazy mk_map_cong_pred;
  1742         val map_cong_pred = Lazy.lazy mk_map_cong_pred;
  1743 
  1743