src/HOL/Option.thy
changeset 51703 f2e92fc0c8aa
parent 51096 60e4b75fefe1
child 52435 6646bb548c6b
--- a/src/HOL/Option.thy	Fri Apr 12 17:02:55 2013 +0200
+++ b/src/HOL/Option.thy	Fri Apr 12 17:21:51 2013 +0200
@@ -46,9 +46,7 @@
 lemma ospec [dest]: "(ALL x:set A. P x) ==> A = Some x ==> P x"
   by simp
 
-declaration {* fn _ =>
-  Classical.map_cs (fn cs => cs addSD2 ("ospec", @{thm ospec}))
-*}
+setup {* map_theory_claset (fn ctxt => ctxt addSD2 ("ospec", @{thm ospec})) *}
 
 lemma elem_set [iff]: "(x : set xo) = (xo = Some x)"
   by (cases xo) auto