src/HOL/Analysis/Tagged_Division.thy
changeset 72569 d56e4eeae967
parent 72548 16345c07bd8c
child 73932 fd21b4a93043
--- a/src/HOL/Analysis/Tagged_Division.thy	Wed Nov 11 11:27:44 2020 +0000
+++ b/src/HOL/Analysis/Tagged_Division.thy	Wed Nov 11 14:27:17 2020 +0000
@@ -2495,8 +2495,8 @@
               (((f j) + 1) / 2 ^ n) * (b \<bullet> j - a \<bullet> j) \<le> (((g j) + 1) / 2 ^ m) * (b \<bullet> j - a \<bullet> j)"
           using that \<open>j \<in> Basis\<close> by (simp add: subset_box field_split_simps aibi)
         then have "((g j) / 2 ^ m) \<le> ((f j) / 2 ^ n) \<and>
-          ((real(f j) + 1) / 2 ^ n) \<le> ((real(g j) + 1) / 2 ^ m)"
-          by (metis bjaj mult.commute of_nat_1 of_nat_add real_mult_le_cancel_iff2)
+                   ((real(f j) + 1) / 2 ^ n) \<le> ((real(g j) + 1) / 2 ^ m)"
+          by (metis bjaj mult.commute of_nat_1 of_nat_add mult_le_cancel_iff2)
         then have "inverse (2^n) \<le> (inverse (2^m) :: real)"
           by (rule dd)
         then have "m \<le> n"