Skip to content

Commit

Permalink
chore(ring_theory/unique_factorization_domain): Eliminate finish (#…
Browse files Browse the repository at this point in the history
  • Loading branch information
stuart-presnell committed Dec 27, 2021
1 parent d67c469 commit de6f57d
Showing 1 changed file with 2 additions and 1 deletion.
3 changes: 2 additions & 1 deletion src/ring_theory/unique_factorization_domain.lean
Expand Up @@ -101,7 +101,8 @@ wf_dvd_monoid.induction_on_irreducible a
(λ u hu _, ⟨0, ⟨by simp [hu], associated.symm (by simp [hu, associated_one_iff_is_unit])⟩⟩)
(λ a i ha0 hii ih hia0,
let ⟨s, hs⟩ := ih ha0 in
⟨i ::ₘ s, ⟨by clear _let_match; finish,
⟨i ::ₘ s, ⟨by clear _let_match;
{ intros b H, cases (multiset.mem_cons.mp H), { convert hii }, { exact hs.1 b h } },
by { rw multiset.prod_cons,
exact hs.2.mul_left _ }⟩⟩)

Expand Down

0 comments on commit de6f57d

Please sign in to comment.