diff -r a80ad0ac0837 -r 4a327c061870 src/HOL/Real.thy --- a/src/HOL/Real.thy Sat Jun 22 06:25:34 2019 +0000 +++ b/src/HOL/Real.thy Sat Jun 22 07:18:55 2019 +0000 @@ -1253,16 +1253,7 @@ subsection \Numerals and Arithmetic\ declaration \ - K (Lin_Arith.add_inj_thms [@{thm of_nat_le_iff} RS iffD2, @{thm of_nat_eq_iff} RS iffD2] - (* not needed because x < (y::nat) can be rewritten as Suc x <= y: of_nat_less_iff RS iffD2 *) - #> Lin_Arith.add_inj_thms [@{thm of_int_le_iff} RS iffD2, @{thm of_nat_eq_iff} RS iffD2] - (* not needed because x < (y::int) can be rewritten as x + 1 <= y: of_int_less_iff RS iffD2 *) - #> Lin_Arith.add_simps [@{thm of_nat_0}, @{thm of_nat_Suc}, @{thm of_nat_add}, - @{thm of_nat_mult}, @{thm of_int_0}, @{thm of_int_1}, - @{thm of_int_add}, @{thm of_int_minus}, @{thm of_int_diff}, - @{thm of_int_mult}, @{thm of_int_of_nat_eq}, - @{thm of_nat_numeral}, @{thm of_int_numeral}, @{thm of_int_neg_numeral}] - #> Lin_Arith.add_inj_const (\<^const_name>\of_nat\, \<^typ>\nat \ real\) + K (Lin_Arith.add_inj_const (\<^const_name>\of_nat\, \<^typ>\nat \ real\) #> Lin_Arith.add_inj_const (\<^const_name>\of_int\, \<^typ>\int \ real\)) \