src/ZF/Epsilon.thy
changeset 76214 0c18df79b1c8
parent 76213 e44d86131648
child 76215 a642599ffdea
--- a/src/ZF/Epsilon.thy	Tue Sep 27 16:51:35 2022 +0100
+++ b/src/ZF/Epsilon.thy	Tue Sep 27 17:03:23 2022 +0100
@@ -359,8 +359,8 @@
 
 lemma def_transrec2:
      "(\<And>x. f(x)\<equiv>transrec2(x,a,b))
-      \<Longrightarrow> f(0) = a &
-          f(succ(i)) = b(i, f(i)) &
+      \<Longrightarrow> f(0) = a \<and>
+          f(succ(i)) = b(i, f(i)) \<and>
           (Limit(K) \<longrightarrow> f(K) = (\<Union>j<K. f(j)))"
 by (simp add: transrec2_Limit)