Zulip Chat Archive
Stream: general
Topic: le_min_of_mem
Kenny Lau (Jul 28 2018 at 20:06):
theorem le_min_of_mem {s : finset α} {a b : α} (h₁ : b ∈ s) (h₂ : a ∈ s.min) : a ≤ b := by rcases @inf_le (with_top α) _ _ _ _ _ _ _ h₁ _ rfl with ⟨b', hb, ab⟩; cases h₂.symm.trans hb; assumption
Kenny Lau (Jul 28 2018 at 20:06):
looks like min_le_of_mem
to me
Chris Hughes (Jul 28 2018 at 20:09):
PR it.
Chris Hughes (Jul 28 2018 at 20:10):
my guess is someone copied the name le_max_of_mem
and didn't notice the word order needed changing
Last updated: Dec 20 2023 at 11:08 UTC