author | haftmann |
Sun, 08 Oct 2017 22:28:19 +0200 | |
changeset 66798 | 39bb2462e681 |
parent 66797 | 9c9baae29217 |
child 66799 | 7ba45c30250c |
--- a/src/HOL/Euclidean_Division.thy Sun Oct 08 22:28:19 2017 +0200 +++ b/src/HOL/Euclidean_Division.thy Sun Oct 08 22:28:19 2017 +0200 @@ -192,6 +192,10 @@ by (auto intro!: euclidean_size_times_nonunit) qed +lemma unit_imp_mod_eq_0: + "a mod b = 0" if "is_unit b" + using that by (simp add: mod_eq_0_iff_dvd unit_imp_dvd) + end class euclidean_ring = idom_modulo + euclidean_semiring