src/HOL/HOLCF/IOA/meta_theory/Abstraction.thy
changeset 42795 66fcc9882784
parent 42793 88bee9f6eec7
child 42814 5af15f1e2ef6
equal deleted inserted replaced
42794:07155da3b2f4 42795:66fcc9882784
   604 
   604 
   605 ML {*
   605 ML {*
   606 fun abstraction_tac ctxt =
   606 fun abstraction_tac ctxt =
   607   SELECT_GOAL (auto_tac
   607   SELECT_GOAL (auto_tac
   608     (ctxt addSIs @{thms weak_strength_lemmas}
   608     (ctxt addSIs @{thms weak_strength_lemmas}
   609       |> map_simpset_local (fn ss =>
   609       |> map_simpset (fn ss =>
   610         ss addsimps [@{thm state_strengthening_def}, @{thm state_weakening_def}])))
   610         ss addsimps [@{thm state_strengthening_def}, @{thm state_weakening_def}])))
   611 *}
   611 *}
   612 
   612 
   613 method_setup abstraction = {* Scan.succeed (SIMPLE_METHOD' o abstraction_tac) *} ""
   613 method_setup abstraction = {* Scan.succeed (SIMPLE_METHOD' o abstraction_tac) *} ""
   614 
   614