Skip to content

Commit

Permalink
Update Basic.lean
Browse files Browse the repository at this point in the history
  • Loading branch information
vihdzp committed Dec 4, 2024
1 parent ea51583 commit a93cfd3
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions Mathlib/Order/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -534,6 +534,12 @@ theorem LinearOrder.ext {A B : LinearOrder α}
ext x y
exact H x y

theorem LinearOrder.ext_lt {A B : LinearOrder α}
(H : ∀ x y : α, (haveI := A; x < y) ↔ x < y) : A = B := by
ext x y
rw [← not_lt, ← @not_lt _ A, not_iff_not]
exact H y x

/-- Given a relation `R` on `β` and a function `f : α → β`, the preimage relation on `α` is defined
by `x ≤ y ↔ f x ≤ f y`. It is the unique relation on `α` making `f` a `RelEmbedding` (assuming `f`
is injective). -/
Expand Down

0 comments on commit a93cfd3

Please sign in to comment.