src/HOL/Library/Univ_Poly.thy
changeset 49751 5248806bc7ab
parent 46730 e3b99d0231bc
child 49962 a8cc904a6820
--- a/src/HOL/Library/Univ_Poly.thy	Tue Oct 09 21:33:12 2012 +0200
+++ b/src/HOL/Library/Univ_Poly.thy	Tue Oct 09 22:24:24 2012 +0200
@@ -414,7 +414,6 @@
 apply (auto simp add: poly_exp poly_mult)
 done
 
-lemma (in semiring_1) one_neq_zero[simp]: "1 \<noteq> 0" using zero_neq_one by blast
 lemma (in comm_ring_1) poly_prime_eq_zero[simp]: "poly [a,1] \<noteq> poly []"
 apply (simp add: fun_eq)
 apply (rule_tac x = "minus one a" in exI)