diff -r dbc62f86a1a9 -r de25474ce728 src/HOL/Real.thy --- a/src/HOL/Real.thy Tue Mar 15 14:08:25 2016 +0000 +++ b/src/HOL/Real.thy Wed Mar 16 13:57:06 2016 +0000 @@ -1404,21 +1404,6 @@ lemma real_sum_of_halves: "x/2 + x/2 = (x::real)" by simp -subsection\Absolute Value Function for the Reals\ - -lemma abs_minus_add_cancel: "\x + (- y)\ = \y + (- (x::real))\" - by (simp add: abs_if) - -lemma abs_add_one_gt_zero: "(0::real) < 1 + \x\" - by (simp add: abs_if) - -lemma abs_add_one_not_less_self: "~ \x\ + (1::real) < x" - by simp - -lemma abs_sum_triangle_ineq: "\(x::real) + y + (-l + -m)\ \ \x + -l\ + \y + -m\" - by simp - - subsection\Floor and Ceiling Functions from the Reals to the Integers\ (* FIXME: theorems for negative numerals. Many duplicates, e.g. from Archimedean_Field.thy. *) @@ -1564,7 +1549,7 @@ proof - have "x ^ n = of_int (\x\ ^ n)" using assms by (induct n arbitrary: x) simp_all - then show ?thesis by (metis floor_of_int) + then show ?thesis by (metis floor_of_int) qed lemma floor_numeral_power[simp]: