src/HOL/Algebra/RingHom.thy
changeset 75963 884dbbc8e1b3
parent 70019 095dce9892e8
--- a/src/HOL/Algebra/RingHom.thy	Wed Aug 24 06:21:06 2022 +0000
+++ b/src/HOL/Algebra/RingHom.thy	Wed Aug 24 08:22:13 2022 +0000
@@ -98,7 +98,7 @@
 
 \<comment> \<open>the kernel of a ring homomorphism is an ideal\<close>
 lemma (in ring_hom_ring) kernel_is_ideal: "ideal (a_kernel R S h) R"
-  apply (rule idealI [OF R.is_ring])
+  apply (rule idealI [OF R.ring_axioms])
     apply (rule additive_subgroup.a_subgroup[OF additive_subgroup_a_kernel])
    apply (auto simp: a_kernel_def')
   done