Skip to content

Commit

Permalink
Update src/algebra/big_operators.lean
Browse files Browse the repository at this point in the history
Co-Authored-By: Chris Hughes <33847686+ChrisHughes24@users.noreply.github.com>
  • Loading branch information
urkud and ChrisHughes24 committed Jan 25, 2020
1 parent 9f05140 commit 17c89a8
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/algebra/big_operators.lean
Original file line number Diff line number Diff line change
Expand Up @@ -180,7 +180,7 @@ by rw [←prod_sdiff h]; simp only [this, prod_const_one, one_mul]
-- If we use `decidable_eq β` here, some rewrites fail because they find a wrong `decidable`
-- instance first
@[to_additive]
lemma prod_filter_ne_one [∀ x, decidable (f x ≠ 1)] : (s.filter $ λx, f x ≠ 1).prod f = s.prod f :=
lemma prod_filter_ne_one {h : ∀ x, decidable (f x ≠ 1)} : (s.filter $ λx, f x ≠ 1).prod f = s.prod f :=
prod_subset (filter_subset _) $ λ x,
by { classical, rw [not_imp_comm, mem_filter], exact and.intro }

Expand Down

0 comments on commit 17c89a8

Please sign in to comment.