src/HOL/Bali/AxSem.thy
changeset 51703 f2e92fc0c8aa
parent 45605 a89b4bc311a5
child 51717 9e7d1c139569
--- a/src/HOL/Bali/AxSem.thy	Fri Apr 12 17:02:55 2013 +0200
+++ b/src/HOL/Bali/AxSem.thy	Fri Apr 12 17:21:51 2013 +0200
@@ -465,7 +465,7 @@
 declare split_if     [split del] split_if_asm     [split del] 
         option.split [split del] option.split_asm [split del]
 declaration {* K (Simplifier.map_ss (fn ss => ss delloop "split_all_tac")) *}
-declaration {* K (Classical.map_cs (fn cs => cs delSWrapper "split_all_tac")) *}
+setup {* map_theory_claset (fn ctxt => ctxt delSWrapper "split_all_tac") *}
 
 inductive
   ax_derivs :: "prog \<Rightarrow> 'a triples \<Rightarrow> 'a triples \<Rightarrow> bool" ("_,_|\<turnstile>_" [61,58,58] 57)