# HG changeset patch # User wenzelm # Date 1349814264 -7200 # Node ID 5248806bc7abee4a116b18935f3272502e0acd5d # Parent 444cfaa331c9db09aa162f72a9739c7ed515eb23 removed redundant lemma, cf. class zero_neq_one in HOL/Rings.thy; diff -r 444cfaa331c9 -r 5248806bc7ab src/HOL/Library/Univ_Poly.thy --- 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 \ 0" using zero_neq_one by blast lemma (in comm_ring_1) poly_prime_eq_zero[simp]: "poly [a,1] \ poly []" apply (simp add: fun_eq) apply (rule_tac x = "minus one a" in exI)