src/HOL/Ring_and_Field.thy
changeset 23400 a64b39e5809b
parent 23398 0b5a400c7595
child 23406 167b53019d6f
--- a/src/HOL/Ring_and_Field.thy	Fri Jun 15 19:19:23 2007 +0200
+++ b/src/HOL/Ring_and_Field.thy	Sat Jun 16 15:01:54 2007 +0200
@@ -1042,13 +1042,14 @@
 
 subsubsection{*Special Cancellation Simprules for Division*}
 
-lemma mult_divide_cancel_left_if [simp]:
+(* FIXME need not be a simp-rule once "divide_cancel_factor" has been fixed *)
+lemma mult_divide_cancel_left_if[simp]:
   fixes c :: "'a :: {field,division_by_zero}"
   shows "(c*a) / (c*b) = (if c=0 then 0 else a/b)"
 by (simp add: mult_divide_cancel_left)
-(* also used at ML level *)
 
-lemma mult_divide_cancel_right_if [simp]:
+(* Not needed anymore because now subsumed by simproc "divide_cancel_factor"
+lemma mult_divide_cancel_right_if:
   fixes c :: "'a :: {field,division_by_zero}"
   shows "(a*c) / (b*c) = (if c=0 then 0 else a/b)"
 by (simp add: mult_divide_cancel_right)
@@ -1092,7 +1093,7 @@
   fixes a :: "'a :: {field,division_by_zero}"
   shows "(b/a) * a = (if a=0 then 0 else b)"
 by (simp add: times_divide_eq_left)
-
+*)
 
 subsection {* Division and Unary Minus *}