src/HOL/RealDef.thy
changeset 38287 796302ca3611
parent 38242 f26d590dce0f
child 38857 97775f3e8722
--- a/src/HOL/RealDef.thy	Mon Aug 09 12:48:40 2010 +0200
+++ b/src/HOL/RealDef.thy	Mon Aug 09 12:53:16 2010 +0200
@@ -1795,8 +1795,8 @@
 fun real_of_int i = (i, 1);
 *}
 
-setup {*
-  Nitpick_HOL.register_frac_type_global @{type_name real}
+declaration {*
+  Nitpick_HOL.register_frac_type @{type_name real}
    [(@{const_name zero_real_inst.zero_real}, @{const_name Nitpick.zero_frac}),
     (@{const_name one_real_inst.one_real}, @{const_name Nitpick.one_frac}),
     (@{const_name plus_real_inst.plus_real}, @{const_name Nitpick.plus_frac}),