src/HOL/HOLCF/IOA/meta_theory/Abstraction.thy
changeset 42795 66fcc9882784
parent 42793 88bee9f6eec7
child 42814 5af15f1e2ef6
--- a/src/HOL/HOLCF/IOA/meta_theory/Abstraction.thy	Fri May 13 23:24:06 2011 +0200
+++ b/src/HOL/HOLCF/IOA/meta_theory/Abstraction.thy	Fri May 13 23:58:40 2011 +0200
@@ -606,7 +606,7 @@
 fun abstraction_tac ctxt =
   SELECT_GOAL (auto_tac
     (ctxt addSIs @{thms weak_strength_lemmas}
-      |> map_simpset_local (fn ss =>
+      |> map_simpset (fn ss =>
         ss addsimps [@{thm state_strengthening_def}, @{thm state_weakening_def}])))
 *}