src/ZF/Constructible/Reflection.thy
changeset 71417 89d05db6dd1f
parent 69593 3dda49e08b9d
child 76213 e44d86131648
--- a/src/ZF/Constructible/Reflection.thy	Tue Feb 04 16:36:49 2020 +0100
+++ b/src/ZF/Constructible/Reflection.thy	Tue Feb 04 16:19:15 2020 +0000
@@ -121,7 +121,7 @@
      "[| M(z); y\<in>Mset(a); P(<y,z>); Ord(a) |] ==> \<exists>z\<in>Mset(FF(P,a)). P(<y,z>)"
 apply (simp add: FF_def)
 apply (simp_all add: cont_Ord_Union [of concl: Mset]
-                     Mset_cont Mset_mono_le not_emptyI Ord_F0)
+                     Mset_cont Mset_mono_le not_emptyI)
 apply (blast intro: F0_works)
 done