src/ZF/Constructible/AC_in_L.thy
changeset 71417 89d05db6dd1f
parent 69593 3dda49e08b9d
child 71568 1005c50b2750
--- a/src/ZF/Constructible/AC_in_L.thy	Tue Feb 04 16:36:49 2020 +0100
+++ b/src/ZF/Constructible/AC_in_L.thy	Tue Feb 04 16:19:15 2020 +0000
@@ -311,7 +311,7 @@
     "well_ord(A,r) ==> well_ord(DPow(A), DPow_r(fn,r,A))"
 apply (simp add: DPow_r_def)
 apply (rule well_ord_measure)
- apply (simp add: DPow_least_def Ord_Least)
+ apply (simp add: DPow_least_def)
 apply (drule DPow_imp_DPow_least, assumption)+
 apply simp
 apply (blast intro: DPow_ord_unique)
@@ -357,7 +357,7 @@
                       Ord_mem_iff_lt)
  apply (blast intro: lt_trans)
 apply (rule_tac x = "succ(lrank(x))" in bexI)
- apply (simp add: Lset_succ_lrank_iff)
+ apply (simp)
 apply (blast intro: Limit_has_succ ltD)
 done