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

Commit

Permalink
chore(data/polynomial/laurent): remove unused case distinction (#14490)
Browse files Browse the repository at this point in the history
  • Loading branch information
Ruben-VandeVelde committed May 31, 2022
1 parent 26a62b0 commit bdf3e97
Showing 1 changed file with 1 addition and 2 deletions.
3 changes: 1 addition & 2 deletions src/data/polynomial/laurent.lean
Original file line number Diff line number Diff line change
Expand Up @@ -318,8 +318,7 @@ lemma exists_T_pow (f : R[T;T⁻¹]) :
begin
apply f.induction_on' _ (λ n a, _); clear f,
{ rintros f g ⟨m, fn, hf⟩ ⟨n, gn, hg⟩,
by_cases h : m ≤ n;
refine ⟨m + n, fn * X ^ n + gn * X ^ m, _⟩;
refine ⟨m + n, fn * X ^ n + gn * X ^ m, _⟩,
simp only [hf, hg, add_mul, add_comm (n : ℤ), map_add, map_mul, polynomial.to_laurent_X_pow,
mul_T_assoc, int.coe_nat_add] },
{ cases n with n n,
Expand Down

0 comments on commit bdf3e97

Please sign in to comment.