src/HOL/Fields.thy
changeset 54230 b1d955791529
parent 54147 97a8ff4e4ac9
child 55718 34618f031ba9
--- a/src/HOL/Fields.thy	Thu Oct 31 16:54:22 2013 +0100
+++ b/src/HOL/Fields.thy	Fri Nov 01 18:51:14 2013 +0100
@@ -156,7 +156,7 @@
   by (simp add: divide_inverse)
 
 lemma diff_divide_distrib: "(a - b) / c = a / c - b / c"
-  by (simp add: diff_minus add_divide_distrib)
+  using add_divide_distrib [of a "- b" c] by simp
 
 lemma nonzero_eq_divide_eq [field_simps]: "c \<noteq> 0 \<Longrightarrow> a = b / c \<longleftrightarrow> a * c = b"
 proof -
@@ -845,7 +845,7 @@
   fix x y :: 'a
   from less_add_one show "\<exists>y. x < y" .. 
   from less_add_one have "x + (- 1) < (x + 1) + (- 1)" by (rule add_strict_right_mono)
-  then have "x - 1 < x + 1 - 1" by (simp only: diff_minus [symmetric])
+  then have "x - 1 < x + 1 - 1" by simp
   then have "x - 1 < x" by (simp add: algebra_simps)
   then show "\<exists>y. y < x" ..
   show "x < y \<Longrightarrow> \<exists>z>x. z < y" by (blast intro!: less_half_sum gt_half_sum)