Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

Commit

Permalink
chore(algebra/big_operators/part_enat): drop file (#17934)
Browse files Browse the repository at this point in the history
The only lemma in this file is a version of `nat.cast_sum`. Also fix an instance on `part_enat` so that `nat.cast_sum` works for this type.
  • Loading branch information
urkud committed Dec 14, 2022
1 parent 198161d commit a2efed6
Show file tree
Hide file tree
Showing 4 changed files with 2 additions and 26 deletions.
3 changes: 1 addition & 2 deletions archive/imo/imo2019_q4.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,6 @@ Authors: Floris van Doorn
-/
import tactic.interval_cases
import algebra.big_operators.order
import algebra.big_operators.part_enat
import data.nat.multiplicity

/-!
Expand Down Expand Up @@ -36,7 +35,7 @@ begin
{ suffices : multiplicity 2 (k! : ℤ) = (n * (n - 1) / 2 : ℕ),
{ rw [← part_enat.coe_lt_coe, ← this], change multiplicity ((2 : ℕ) : ℤ) _ < _,
simp_rw [int.coe_nat_multiplicity, multiplicity_two_factorial_lt hk.lt.ne.symm] },
rw [h, multiplicity.finset.prod prime_2, ← sum_range_id, ← sum_nat_coe_enat],
rw [h, multiplicity.finset.prod prime_2, ← sum_range_id, nat.cast_sum],
apply sum_congr rfl, intros i hi,
rw [multiplicity_sub_of_gt, multiplicity_pow_self_of_prime prime_2],
rwa [multiplicity_pow_self_of_prime prime_2, multiplicity_pow_self_of_prime prime_2,
Expand Down
1 change: 0 additions & 1 deletion src/algebra/big_operators/default.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,4 +6,3 @@ import algebra.big_operators.ring
import algebra.big_operators.pi
import algebra.big_operators.finsupp
import algebra.big_operators.nat_antidiagonal
import algebra.big_operators.part_enat
22 changes: 0 additions & 22 deletions src/algebra/big_operators/part_enat.lean

This file was deleted.

2 changes: 1 addition & 1 deletion src/data/nat/part_enat.lean
Original file line number Diff line number Diff line change
Expand Up @@ -78,7 +78,7 @@ instance : add_comm_monoid part_enat :=
add_zero := λ x, part.ext' (and_true _) (λ _ _, add_zero _),
add_assoc := λ x y z, part.ext' and.assoc (λ _ _, add_assoc _ _ _) }

instance : add_monoid_with_one part_enat :=
instance : add_comm_monoid_with_one part_enat :=
{ one := 1,
nat_cast := some,
nat_cast_zero := rfl,
Expand Down

0 comments on commit a2efed6

Please sign in to comment.