One useful lemma/simprule
authorpaulson <lp15@cam.ac.uk>
Fri, 08 Jan 2021 16:07:34 +0000
changeset 73103 b69fd6e19662
parent 73102 87067698ae53
child 73104 6520d59fbdd7
One useful lemma/simprule
src/HOL/Computational_Algebra/Factorial_Ring.thy
--- a/src/HOL/Computational_Algebra/Factorial_Ring.thy	Fri Jan 08 15:13:23 2021 +0100
+++ b/src/HOL/Computational_Algebra/Factorial_Ring.thy	Fri Jan 08 16:07:34 2021 +0000
@@ -1606,6 +1606,9 @@
   thus ?thesis by simp
 qed
 
+lemma multiplicity_zero_1 [simp]: "multiplicity 0 x = 0"
+  by (metis (mono_tags) local.dvd_0_left multiplicity_zero not_dvd_imp_multiplicity_0)
+
 lemma inj_on_Prod_primes:
   assumes "\<And>P p. P \<in> A \<Longrightarrow> p \<in> P \<Longrightarrow> prime p"
   assumes "\<And>P. P \<in> A \<Longrightarrow> finite P"