src/HOL/Int.thy
changeset 32272 cc1bf9077167
parent 32069 6d28bbd33e2c
child 32437 66f1a0dfe7d9
equal deleted inserted replaced
32269:b642e4813e53 32272:cc1bf9077167
   998 
   998 
   999 text {*
   999 text {*
  1000   Converting numerals 0 and 1 to their abstract versions.
  1000   Converting numerals 0 and 1 to their abstract versions.
  1001 *}
  1001 *}
  1002 
  1002 
  1003 lemma numeral_0_eq_0 [simp]:
  1003 lemma numeral_0_eq_0 [simp, code_post]:
  1004   "Numeral0 = (0::'a::number_ring)"
  1004   "Numeral0 = (0::'a::number_ring)"
  1005   unfolding number_of_eq numeral_simps by simp
  1005   unfolding number_of_eq numeral_simps by simp
  1006 
  1006 
  1007 lemma numeral_1_eq_1 [simp]:
  1007 lemma numeral_1_eq_1 [simp, code_post]:
  1008   "Numeral1 = (1::'a::number_ring)"
  1008   "Numeral1 = (1::'a::number_ring)"
  1009   unfolding number_of_eq numeral_simps by simp
  1009   unfolding number_of_eq numeral_simps by simp
  1010 
  1010 
  1011 text {*
  1011 text {*
  1012   Special-case simplification for small constants.
  1012   Special-case simplification for small constants.