src/HOL/Binomial.thy
changeset 66311 037aaa0b6daf
parent 65813 bdd17b18e103
child 66806 a4e82b58d833
--- a/src/HOL/Binomial.thy	Thu Aug 03 07:31:25 2017 +0200
+++ b/src/HOL/Binomial.thy	Thu Aug 03 09:30:09 2017 +0200
@@ -1177,10 +1177,10 @@
     using finite_lists_length_eq[OF finite_atLeastLessThan] conj_commute by auto
   have fin_A: "finite ?A" using fin[of _ "N+1"]
     by (intro finite_subset[where ?A = "?A" and ?B = "{xs. size xs = m - 1 \<and> set xs \<subseteq> {0..<N+1}}"])
-      (auto simp: member_le_sum_list_nat less_Suc_eq_le)
+      (auto simp: member_le_sum_list less_Suc_eq_le)
   have fin_B: "finite ?B"
     by (intro finite_subset[where ?A = "?B" and ?B = "{xs. size xs = m \<and> set xs \<subseteq> {0..<N}}"])
-      (auto simp: member_le_sum_list_nat less_Suc_eq_le fin)
+      (auto simp: member_le_sum_list less_Suc_eq_le fin)
   have uni: "?C = ?A' \<union> ?B'"
     by auto
   have disj: "?A' \<inter> ?B' = {}" by blast