src/HOL/Library/Code_Real_Approx_By_Float.thy
changeset 82774 2865a6618cba
parent 81706 7beb0cf38292
--- a/src/HOL/Library/Code_Real_Approx_By_Float.thy	Thu Jun 26 17:25:29 2025 +0200
+++ b/src/HOL/Library/Code_Real_Approx_By_Float.thy	Thu Jun 26 17:25:29 2025 +0200
@@ -61,12 +61,6 @@
 
 end
 
-lemma [code]: \<open>Ratreal r = (case quotient_of r of (p, q) \<Rightarrow> real_of_int p / real_of_int q)\<close>
-  by (cases r) (simp add: quotient_of_Fract of_rat_rat)
-
-lemma [code]: \<open>inverse r = 1 / r\<close> for r :: real
-  by (fact inverse_eq_divide)
-
 declare [[code drop: \<open>HOL.equal :: real \<Rightarrow> real \<Rightarrow> bool\<close>
   \<open>(\<le>) :: real \<Rightarrow> real \<Rightarrow> bool\<close>
   \<open>(<) :: real \<Rightarrow> real \<Rightarrow> bool\<close>
@@ -75,6 +69,7 @@
   \<open>uminus :: real \<Rightarrow> real\<close>
   \<open>minus :: real \<Rightarrow> real \<Rightarrow> real\<close>
   \<open>divide :: real \<Rightarrow> real \<Rightarrow> real\<close>
+  \<open>inverse :: real \<Rightarrow> real\<close>
   sqrt
   \<open>ln :: real \<Rightarrow> real\<close>
   pi
@@ -82,6 +77,12 @@
   arccos
   arctan]]
 
+lemma [code]: \<open>Ratreal r = (case quotient_of r of (p, q) \<Rightarrow> real_of_int p / real_of_int q)\<close>
+  by (cases r) (simp add: quotient_of_Fract of_rat_rat)
+
+lemma [code]: \<open>inverse r = 1 / r\<close> for r :: real
+  by (fact inverse_eq_divide)
+
 code_reserved (SML) Real
 
 code_printing