src/HOL/Word/Word.thy
changeset 46025 64a19ea435fc
parent 46023 fad87bb608fc
parent 46008 c296c75f4cf4
child 46026 83caa4f4bd56
--- a/src/HOL/Word/Word.thy	Wed Dec 28 20:05:52 2011 +0100
+++ b/src/HOL/Word/Word.thy	Wed Dec 28 22:08:44 2011 +0100
@@ -2389,7 +2389,7 @@
   "n = size (w::'a::len0 word) \<Longrightarrow> ofn = set_bits \<Longrightarrow> [w, ofn g] = l \<Longrightarrow> 
     td_ext test_bit ofn {f. ALL i. f i --> i < n} (%h i. h i & i < n)"
   apply (unfold word_size td_ext_def')
-  apply (safe del: subset_antisym)
+  apply safe
      apply (rule_tac [3] ext)
      apply (rule_tac [4] ext)
      apply (unfold word_size of_nth_def test_bit_bl)