src/HOL/Library/Nat_Bijection.thy
changeset 39302 d7728f65b353
parent 37591 d3daea901123
child 41959 b460124855b8
--- a/src/HOL/Library/Nat_Bijection.thy	Mon Sep 13 08:43:48 2010 +0200
+++ b/src/HOL/Library/Nat_Bijection.thy	Mon Sep 13 11:13:15 2010 +0200
@@ -333,8 +333,8 @@
 lemma set_decode_plus_power_2:
   "n \<notin> set_decode z \<Longrightarrow> set_decode (2 ^ n + z) = insert n (set_decode z)"
  apply (induct n arbitrary: z, simp_all)
-  apply (rule set_ext, induct_tac x, simp, simp add: even_nat_Suc_div_2)
- apply (rule set_ext, induct_tac x, simp, simp add: add_commute)
+  apply (rule set_eqI, induct_tac x, simp, simp add: even_nat_Suc_div_2)
+ apply (rule set_eqI, induct_tac x, simp, simp add: add_commute)
 done
 
 lemma finite_set_decode [simp]: "finite (set_decode n)"