src/HOL/Int.thy
changeset 47192 0c0501cb6da6
parent 47108 2a1953f0d20d
child 47207 9368aa814518
--- a/src/HOL/Int.thy	Thu Mar 29 11:47:30 2012 +0200
+++ b/src/HOL/Int.thy	Thu Mar 29 14:09:10 2012 +0200
@@ -857,14 +857,6 @@
   "abs(-1 ^ n) = (1::'a::linordered_idom)"
 by (simp add: power_abs)
 
-text{*Lemmas for specialist use, NOT as default simprules*}
-(* TODO: see if semiring duplication can be removed without breaking proofs *)
-lemma mult_2: "2 * z = (z+z::'a::semiring_1)"
-unfolding one_add_one [symmetric] left_distrib by simp
-
-lemma mult_2_right: "z * 2 = (z+z::'a::semiring_1)"
-unfolding one_add_one [symmetric] right_distrib by simp
-
 
 subsection{*More Inequality Reasoning*}