src/HOL/Rat.thy
changeset 43732 6b2bdc57155b
parent 42311 eb32a8474a57
child 43733 a6ca7b83612f
--- a/src/HOL/Rat.thy	Fri Jul 08 22:00:53 2011 +0200
+++ b/src/HOL/Rat.thy	Sat Jul 09 13:41:58 2011 +0200
@@ -739,6 +739,20 @@
   qed
 qed
 
+instantiation rat :: floor_ceiling
+begin
+
+definition [code del]:
+  "floor (x::rat) = (THE z. of_int z \<le> x \<and> x < of_int (z + 1))"
+
+instance proof
+  fix x :: rat
+  show "of_int (floor x) \<le> x \<and> x < of_int (floor x + 1)"
+    unfolding floor_rat_def using floor_exists1 by (rule theI')
+qed
+
+end
+
 lemma floor_Fract: "floor (Fract a b) = a div b"
   using rat_floor_lemma [of a b]
   by (simp add: floor_unique)