src/HOL/Rings.thy
changeset 67234 ab10ea1d6fd0
parent 67226 ec32cdaab97b
child 67689 2c38ffd6ec71
--- a/src/HOL/Rings.thy	Wed Dec 20 22:07:05 2017 +0100
+++ b/src/HOL/Rings.thy	Thu Dec 21 08:23:19 2017 +0100
@@ -1263,6 +1263,16 @@
   "coprime (a * c) (b * c) \<longleftrightarrow> is_unit c \<and> coprime a b"
   using coprime_mult_self_left_iff [of c a b] by (simp add: ac_simps)
 
+lemma coprime_absorb_left:
+  assumes "x dvd y"
+  shows   "coprime x y \<longleftrightarrow> is_unit x"
+  using assms coprime_common_divisor is_unit_left_imp_coprime by auto
+
+lemma coprime_absorb_right:
+  assumes "y dvd x"
+  shows   "coprime x y \<longleftrightarrow> is_unit y"
+  using assms coprime_common_divisor is_unit_right_imp_coprime by auto
+
 end
 
 class unit_factor =