src/HOL/Real.thy
changeset 67051 e7e54a0b9197
parent 66912 a99a7cbf0fb5
child 67226 ec32cdaab97b
--- a/src/HOL/Real.thy	Sat Nov 11 18:33:35 2017 +0000
+++ b/src/HOL/Real.thy	Sat Nov 11 18:41:08 2017 +0000
@@ -1245,7 +1245,7 @@
 
 lemma Rats_abs_nat_div_natE:
   assumes "x \<in> \<rat>"
-  obtains m n :: nat where "n \<noteq> 0" and "\<bar>x\<bar> = real m / real n" and "gcd m n = 1"
+  obtains m n :: nat where "n \<noteq> 0" and "\<bar>x\<bar> = real m / real n" and "coprime m n"
 proof -
   from \<open>x \<in> \<rat>\<close> obtain i :: int and n :: nat where "n \<noteq> 0" and "x = real_of_int i / real n"
     by (auto simp add: Rats_eq_int_div_nat)
@@ -1281,6 +1281,8 @@
     with gcd_k gcd_l have "?gcd * ?gcd' = ?gcd" by simp
     with gcd show ?thesis by auto
   qed
+  then have "coprime ?k ?l"
+    by (simp only: coprime_iff_gcd_eq_1)
   ultimately show ?thesis ..
 qed
 
@@ -1415,8 +1417,6 @@
   for m :: nat
   by (metis not_le real_of_nat_less_numeral_iff)
 
-declare of_int_floor_le [simp]  (* FIXME duplicate!? *)
-
 lemma of_int_floor_cancel [simp]: "of_int \<lfloor>x\<rfloor> = x \<longleftrightarrow> (\<exists>n::int. x = of_int n)"
   by (metis floor_of_int)
 
@@ -1424,7 +1424,7 @@
   by linarith
 
 lemma floor_eq2: "real_of_int n \<le> x \<Longrightarrow> x < real_of_int n + 1 \<Longrightarrow> \<lfloor>x\<rfloor> = n"
-  by linarith
+  by (fact floor_unique)
 
 lemma floor_eq3: "real n < x \<Longrightarrow> x < real (Suc n) \<Longrightarrow> nat \<lfloor>x\<rfloor> = n"
   by linarith