src/HOL/Rat.thy
changeset 38287 796302ca3611
parent 38242 f26d590dce0f
child 38857 97775f3e8722
--- a/src/HOL/Rat.thy	Mon Aug 09 12:48:40 2010 +0200
+++ b/src/HOL/Rat.thy	Mon Aug 09 12:53:16 2010 +0200
@@ -1173,8 +1173,8 @@
 fun rat_of_int i = (i, 1);
 *}
 
-setup {*
-  Nitpick_HOL.register_frac_type_global @{type_name rat}
+declaration {*
+  Nitpick_HOL.register_frac_type @{type_name rat}
    [(@{const_name zero_rat_inst.zero_rat}, @{const_name Nitpick.zero_frac}),
     (@{const_name one_rat_inst.one_rat}, @{const_name Nitpick.one_frac}),
     (@{const_name plus_rat_inst.plus_rat}, @{const_name Nitpick.plus_frac}),