src/HOL/Binomial.thy
changeset 73932 fd21b4a93043
parent 72302 d7d90ed4c74e
child 75856 4b507edcf6b5
--- a/src/HOL/Binomial.thy	Fri Jun 18 15:03:12 2021 +0200
+++ b/src/HOL/Binomial.thy	Thu Jul 08 08:42:36 2021 +0200
@@ -933,7 +933,7 @@
   have "?lhs = (\<Sum>k\<le>m. (- a gchoose k) * (- x) ^ k * (x + y) ^ (m - k))"
     by (simp add: gbinomial_partial_sum_poly)
   also have "... = (\<Sum>k\<le>m. (-1) ^ k * (of_nat k - - a - 1 gchoose k) * (- x) ^ k * (x + y) ^ (m - k))"
-    by (metis (no_types, hide_lams) gbinomial_negated_upper)
+    by (metis (no_types, opaque_lifting) gbinomial_negated_upper)
   also have "... = ?rhs"
     by (intro sum.cong) (auto simp flip: power_mult_distrib)
   finally show ?thesis .