src/HOL/Complex/CLim.thy
changeset 14738 83f1a514dcb4
parent 14469 c7674b7034f5
child 15013 34264f5e4691
--- a/src/HOL/Complex/CLim.thy	Tue May 11 14:00:02 2004 +0200
+++ b/src/HOL/Complex/CLim.thy	Tue May 11 20:11:08 2004 +0200
@@ -17,7 +17,7 @@
 by (simp add: numeral_2_eq_2)
 
 text{*Changing the quantified variable. Install earlier?*}
-lemma all_shift: "(\<forall>x::'a::ring. P x) = (\<forall>x. P (x-a))";
+lemma all_shift: "(\<forall>x::'a::comm_ring_1. P x) = (\<forall>x. P (x-a))";
 apply auto 
 apply (drule_tac x="x+a" in spec) 
 apply (simp add: diff_minus add_assoc)