src/HOL/Library/Numeral_Type.thy
changeset 62348 9a5f43dac883
parent 61649 268d88ec9087
child 64593 50c715579715
--- a/src/HOL/Library/Numeral_Type.thy	Wed Feb 17 21:51:57 2016 +0100
+++ b/src/HOL/Library/Numeral_Type.thy	Wed Feb 17 21:51:57 2016 +0100
@@ -230,7 +230,7 @@
            "Rep_bit0 :: 'a::finite bit0 \<Rightarrow> int"
            "Abs_bit0 :: int \<Rightarrow> 'a::finite bit0"
 apply (rule mod_type.intro)
-apply (simp add: int_mult type_definition_bit0)
+apply (simp add: of_nat_mult type_definition_bit0)
 apply (rule one_less_int_card)
 apply (rule zero_bit0_def)
 apply (rule one_bit0_def)
@@ -245,7 +245,7 @@
            "Rep_bit1 :: 'a::finite bit1 \<Rightarrow> int"
            "Abs_bit1 :: int \<Rightarrow> 'a::finite bit1"
 apply (rule mod_type.intro)
-apply (simp add: int_mult type_definition_bit1)
+apply (simp add: of_nat_mult type_definition_bit1)
 apply (rule one_less_int_card)
 apply (rule zero_bit1_def)
 apply (rule one_bit1_def)