src/HOL/Library/Commutative_Ring.thy
changeset 23477 f4b83f03cac9
parent 22742 06165e40e7bd
child 25595 6c48275f9c76
--- a/src/HOL/Library/Commutative_Ring.thy	Fri Jun 22 22:41:17 2007 +0200
+++ b/src/HOL/Library/Commutative_Ring.thy	Sat Jun 23 19:33:22 2007 +0200
@@ -174,11 +174,11 @@
 
 text {* mkPinj preserve semantics *}
 lemma mkPinj_ci: "Ipol l (mkPinj a B) = Ipol l (Pinj a B)"
-  by (induct B) (auto simp add: mkPinj_def ring_eq_simps)
+  by (induct B) (auto simp add: mkPinj_def ring_simps)
 
 text {* mkPX preserves semantics *}
 lemma mkPX_ci: "Ipol l (mkPX A b C) = Ipol l (PX A b C)"
-  by (cases A) (auto simp add: mkPX_def mkPinj_ci power_add ring_eq_simps)
+  by (cases A) (auto simp add: mkPX_def mkPinj_ci power_add ring_simps)
 
 text {* Correctness theorems for the implemented operations *}
 
@@ -193,13 +193,13 @@
   show ?case
   proof (rule linorder_cases)
     assume "x < y"
-    with 6 show ?case by (simp add: mkPinj_ci ring_eq_simps)
+    with 6 show ?case by (simp add: mkPinj_ci ring_simps)
   next
     assume "x = y"
     with 6 show ?case by (simp add: mkPinj_ci)
   next
     assume "x > y"
-    with 6 show ?case by (simp add: mkPinj_ci ring_eq_simps)
+    with 6 show ?case by (simp add: mkPinj_ci ring_simps)
   qed
 next
   case (7 x P Q y R)
@@ -207,7 +207,7 @@
   moreover
   { assume "x = 0" with 7 have ?case by simp }
   moreover
-  { assume "x = 1" with 7 have ?case by (simp add: ring_eq_simps) }
+  { assume "x = 1" with 7 have ?case by (simp add: ring_simps) }
   moreover
   { assume "x > 1" from 7 have ?case by (cases x) simp_all }
   ultimately show ?case by blast
@@ -226,20 +226,20 @@
   show ?case
   proof (rule linorder_cases)
     assume a: "x < y" hence "EX d. d + x = y" by arith
-    with 9 a show ?case by (auto simp add: mkPX_ci power_add ring_eq_simps)
+    with 9 a show ?case by (auto simp add: mkPX_ci power_add ring_simps)
   next
     assume a: "y < x" hence "EX d. d + y = x" by arith
-    with 9 a show ?case by (auto simp add: power_add mkPX_ci ring_eq_simps)
+    with 9 a show ?case by (auto simp add: power_add mkPX_ci ring_simps)
   next
     assume "x = y"
-    with 9 show ?case by (simp add: mkPX_ci ring_eq_simps)
+    with 9 show ?case by (simp add: mkPX_ci ring_simps)
   qed
-qed (auto simp add: ring_eq_simps)
+qed (auto simp add: ring_simps)
 
 text {* Multiplication *}
 lemma mul_ci: "Ipol l (P \<otimes> Q) = Ipol l P * Ipol l Q"
   by (induct P Q arbitrary: l rule: mul.induct)
-    (simp_all add: mkPX_ci mkPinj_ci ring_eq_simps add_ci power_add)
+    (simp_all add: mkPX_ci mkPinj_ci ring_simps add_ci power_add)
 
 text {* Substraction *}
 lemma sub_ci: "Ipol l (P \<ominus> Q) = Ipol l P - Ipol l Q"
@@ -248,7 +248,7 @@
 text {* Square *}
 lemma sqr_ci: "Ipol ls (sqr P) = Ipol ls P * Ipol ls P"
   by (induct P arbitrary: ls)
-    (simp_all add: add_ci mkPinj_ci mkPX_ci mul_ci ring_eq_simps power_add)
+    (simp_all add: add_ci mkPinj_ci mkPX_ci mul_ci ring_simps power_add)
 
 text {* Power *}
 lemma even_pow:"even n \<Longrightarrow> pow n P = pow (n div 2) (sqr P)"