--- a/src/ZF/ex/Ring.thy Tue Sep 27 16:51:35 2022 +0100
+++ b/src/ZF/ex/Ring.thy Tue Sep 27 17:03:23 2022 +0100
@@ -234,9 +234,9 @@
ring_hom :: "[i,i] => i" where
"ring_hom(R,S) \<equiv>
{h \<in> carrier(R) -> carrier(S).
- (\<forall>x y. x \<in> carrier(R) & y \<in> carrier(R) \<longrightarrow>
- h ` (x \<cdot>\<^bsub>R\<^esub> y) = (h ` x) \<cdot>\<^bsub>S\<^esub> (h ` y) &
- h ` (x \<oplus>\<^bsub>R\<^esub> y) = (h ` x) \<oplus>\<^bsub>S\<^esub> (h ` y)) &
+ (\<forall>x y. x \<in> carrier(R) \<and> y \<in> carrier(R) \<longrightarrow>
+ h ` (x \<cdot>\<^bsub>R\<^esub> y) = (h ` x) \<cdot>\<^bsub>S\<^esub> (h ` y) \<and>
+ h ` (x \<oplus>\<^bsub>R\<^esub> y) = (h ` x) \<oplus>\<^bsub>S\<^esub> (h ` y)) \<and>
h ` \<one>\<^bsub>R\<^esub> = \<one>\<^bsub>S\<^esub>}"
lemma ring_hom_memI: