src/HOL/Decision_Procs/Approximation.thy
changeset 36531 19f6e3b0d9b6
parent 36526 353041483b9b
child 36778 739a9379e29b
--- a/src/HOL/Decision_Procs/Approximation.thy	Thu Apr 29 15:00:39 2010 +0200
+++ b/src/HOL/Decision_Procs/Approximation.thy	Thu Apr 29 15:00:40 2010 +0200
@@ -3209,13 +3209,12 @@
   interpret_floatarith_divide interpret_floatarith_diff interpret_floatarith_tan interpret_floatarith_powr interpret_floatarith_log
   interpret_floatarith_sin
 
-code_reflect
+code_reflect Float_Arith
   datatypes float = Float
   and floatarith = Add | Minus | Mult | Inverse | Cos | Arctan
     | Abs | Max | Min | Pi | Sqrt | Exp | Ln | Power | Var | Num
   and form = Bound | Assign | Less | LessEqual | AtLeastAtMost
   functions approx_form approx_tse_form approx' approx_form_eval
-  module_name Float_Arith
 
 ML {*
   fun reorder_bounds_tac prems i =