src/HOL/Library/Log_Nat.thy
changeset 80732 3eda814762fc
parent 75455 91c16c5ad3e9
child 81410 da3bf4a755b3
--- a/src/HOL/Library/Log_Nat.thy	Thu Aug 08 18:56:14 2024 +0100
+++ b/src/HOL/Library/Log_Nat.thy	Fri Aug 09 20:45:31 2024 +0100
@@ -22,7 +22,7 @@
   then have "real (x div b) + real (x mod b) / real b - real (x div b) < 1"
     by (simp add: field_simps)
   then show ?thesis
-    by (simp add: real_of_nat_div_aux [symmetric])
+    by (metis of_nat_of_nat_div_aux)
 qed
 
 
@@ -108,7 +108,7 @@
   also have "\<dots> = \<lfloor>log b (x / b)\<rfloor> + 1" using that by simp
   also have "\<lfloor>log b (x / b)\<rfloor> = \<lfloor>log b (x div b + (x / b - x div b))\<rfloor>" by simp
   also have "\<dots> = \<lfloor>log b (x div b)\<rfloor>"
-    using that real_of_nat_div4 divide_nat_diff_div_nat_less_one
+    using that of_nat_div_le_of_nat divide_nat_diff_div_nat_less_one
     by (intro floor_log_add_eqI) auto
   finally show ?thesis .
 qed