Skip to content

Commit

Permalink
chore(ring_theory/*): Eliminate finish (#11100)
Browse files Browse the repository at this point in the history
Removing uses of `finish`, as discussed in this Zulip thread (https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/mathlib.20sat.20solvers)
  • Loading branch information
stuart-presnell committed Dec 28, 2021
1 parent 143fec6 commit 0b80d0c
Show file tree
Hide file tree
Showing 2 changed files with 3 additions and 2 deletions.
2 changes: 1 addition & 1 deletion src/ring_theory/ideal/basic.lean
Expand Up @@ -574,7 +574,7 @@ lemma bot_lt_of_maximal (M : ideal R) [hm : M.is_maximal] (non_field : ¬ is_fie
begin
rcases (ring.not_is_field_iff_exists_ideal_bot_lt_and_lt_top.1 non_field)
with ⟨I, Ibot, Itop⟩,
split, finish,
split, { simp },
intro mle,
apply @irrefl _ (<) _ (⊤ : ideal R),
have : M = ⊥ := eq_bot_iff.mpr mle,
Expand Down
3 changes: 2 additions & 1 deletion src/ring_theory/principal_ideal_domain.lean
Expand Up @@ -168,7 +168,8 @@ instance euclidean_domain.to_principal_ideal_domain : is_principal_ideal_ring R
have (x % (well_founded.min wf {x : R | x ∈ S ∧ x ≠ 0} h) ∉ {x : R | x ∈ S ∧ x ≠ 0}),
from λ h₁, well_founded.not_lt_min wf _ h h₁ (mod_lt x hmin.2),
have x % well_founded.min wf {x : R | x ∈ S ∧ x ≠ 0} h = 0,
by finish [(mod_mem_iff hmin.1).2 hx],
by { simp only [not_and_distrib, set.mem_set_of_eq, not_ne_iff] at this,
cases this, cases this ((mod_mem_iff hmin.1).2 hx), exact this },
by simp *),
λ hx, let ⟨y, hy⟩ := ideal.mem_span_singleton.1 hx in hy.symm ▸ S.mul_mem_right _ hmin.1⟩⟩
else0, submodule.ext $ λ a,
Expand Down

0 comments on commit 0b80d0c

Please sign in to comment.