diff -r 35a9e1cbb5b3 -r 7f927120b5a2 src/HOL/Number_Theory/Euclidean_Algorithm.thy --- a/src/HOL/Number_Theory/Euclidean_Algorithm.thy Wed Feb 17 21:51:58 2016 +0100 +++ b/src/HOL/Number_Theory/Euclidean_Algorithm.thy Wed Feb 17 21:51:58 2016 +0100 @@ -1064,11 +1064,11 @@ "Lcm {} = 1" by (simp add: Lcm_1_iff) -lemma Lcm_eq_0 [simp]: +lemma Lcm_eq_0_I [simp]: "0 \ A \ Lcm A = 0" by (drule dvd_Lcm) simp -lemma Lcm0_iff': +lemma Lcm_0_iff': "Lcm A = 0 \ \(\l. l \ 0 \ (\a\A. a dvd l))" proof assume "Lcm A = 0" @@ -1092,7 +1092,7 @@ qed qed (simp only: Lcm_Lcm_eucl Lcm_eucl_def if_False) -lemma Lcm0_iff [simp]: +lemma Lcm_0_iff [simp]: "finite A \ Lcm A = 0 \ 0 \ A" proof - assume "finite A" @@ -1108,7 +1108,7 @@ done moreover from \finite A\ have "\a\A. a dvd \A" by blast ultimately have "\l. l \ 0 \ (\a\A. a dvd l)" by blast - with Lcm0_iff' have "Lcm A \ 0" by simp + with Lcm_0_iff' have "Lcm A \ 0" by simp } ultimately show "Lcm A = 0 \ 0 \ A" by blast qed @@ -1210,7 +1210,7 @@ lemma Lcm_Gcd: "Lcm A = Gcd {m. \a\A. a dvd m}" - by (rule LcmI[symmetric]) (auto intro: dvd_Gcd Gcd_greatest) + by (rule LcmI[symmetric]) (auto intro: Gcd_greatest Gcd_greatest) lemma Gcd_1: "1 \ A \ Gcd A = 1"