src/HOL/Rat.thy
changeset 41920 d4fb7a418152
parent 41792 ff3cb0c418b7
child 42311 eb32a8474a57
--- a/src/HOL/Rat.thy	Fri Mar 11 15:21:13 2011 +0100
+++ b/src/HOL/Rat.thy	Fri Mar 11 15:21:13 2011 +0100
@@ -1132,11 +1132,11 @@
 no_notation fcomp (infixl "\<circ>>" 60)
 no_notation scomp (infixl "\<circ>\<rightarrow>" 60)
 
-instantiation rat :: full_small
+instantiation rat :: exhaustive
 begin
 
 definition
-  "full_small f d = full_small (%(k, kt). full_small (%(l, lt).
+  "exhaustive f d = exhaustive (%(k, kt). exhaustive (%(l, lt).
      f (valterm_fract (Code_Numeral.int_of k, %_. Code_Evaluation.term_of (Code_Numeral.int_of k)) (Code_Numeral.int_of l, %_. Code_Evaluation.term_of (Code_Numeral.int_of l)))) d) d"
 
 instance ..