Deleted subset_antisym in a few proofs, because it is
authorberghofe
Wed, 07 May 2008 10:59:42 +0200
changeset 26827 a62f8db42f4a
parent 26826 fd8fdf21660f
child 26828 60d1fa8e0831
Deleted subset_antisym in a few proofs, because it is accidentally applied to predicates as well.
src/HOL/Word/BinGeneral.thy
src/HOL/Word/WordBitwise.thy
--- a/src/HOL/Word/BinGeneral.thy	Wed May 07 10:59:41 2008 +0200
+++ b/src/HOL/Word/BinGeneral.thy	Wed May 07 10:59:42 2008 +0200
@@ -272,14 +272,14 @@
     apply safe
     apply (erule rev_mp)
     apply (induct_tac y rule: bin_induct)
-      apply safe
+      apply (safe del: subset_antisym)
       apply (drule_tac x=0 in fun_cong, force)
      apply (erule notE, rule ext, 
             drule_tac x="Suc x" in fun_cong, force)
     apply (drule_tac x=0 in fun_cong, force)
    apply (erule rev_mp)
    apply (induct_tac y rule: bin_induct)
-     apply safe
+     apply (safe del: subset_antisym)
      apply (drule_tac x=0 in fun_cong, force)
     apply (erule notE, rule ext, 
            drule_tac x="Suc x" in fun_cong, force)
--- a/src/HOL/Word/WordBitwise.thy	Wed May 07 10:59:41 2008 +0200
+++ b/src/HOL/Word/WordBitwise.thy	Wed May 07 10:59:42 2008 +0200
@@ -327,7 +327,7 @@
   "n = size (w::'a::len0 word) ==> ofn = set_bits ==> [w, ofn g] = l ==> 
     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
+  apply (safe del: subset_antisym)
      apply (rule_tac [3] ext)
      apply (rule_tac [4] ext)
      apply (unfold word_size of_nth_def test_bit_bl)