src/HOL/Algebra/UnivPoly.thy
changeset 75963 884dbbc8e1b3
parent 69597 ff784d5a5bfb
child 76987 4c275405faae
--- a/src/HOL/Algebra/UnivPoly.thy	Wed Aug 24 06:21:06 2022 +0000
+++ b/src/HOL/Algebra/UnivPoly.thy	Wed Aug 24 08:22:13 2022 +0000
@@ -501,11 +501,8 @@
   Interpretation of lemmas from \<^term>\<open>algebra\<close>.
 \<close>
 
-lemma (in cring) cring:
-  "cring R" ..
-
 lemma (in UP_cring) UP_algebra:
-  "algebra R P" by (auto intro!: algebraI R.cring UP_cring UP_smult_l_distr UP_smult_r_distr
+  "algebra R P" by (auto intro!: algebraI R.cring_axioms UP_cring UP_smult_l_distr UP_smult_r_distr
     UP_smult_assoc1 UP_smult_assoc2)
 
 sublocale UP_cring < algebra R P using UP_algebra .