Skip to content

Commit

Permalink
add IsBot.isMin_iff
Browse files Browse the repository at this point in the history
  • Loading branch information
pitmonticone committed Nov 20, 2024
1 parent 08e5232 commit 432124e
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions Mathlib/Order/Max.lean
Original file line number Diff line number Diff line change
Expand Up @@ -204,6 +204,10 @@ theorem IsTop.isMax_iff {α} [PartialOrder α] {i j : α} (h : IsTop i) : IsMax
simp_rw [le_antisymm_iff, h j, true_and]
exact ⟨(· (h j)), Function.swap (fun _ ↦ h · |>.trans ·)⟩

theorem IsBot.isMin_iff {α} [PartialOrder α] {i j : α} (h : IsBot i) : IsMin j ↔ j = i := by
simp_rw [le_antisymm_iff, h j, and_true]
exact ⟨fun a ↦ a (h j), fun a h' ↦ fun _ ↦ Preorder.le_trans j i h' a (h h')⟩

@[simp]
theorem isBot_toDual_iff : IsBot (toDual a) ↔ IsTop a :=
Iff.rfl
Expand Down

0 comments on commit 432124e

Please sign in to comment.