File tree Expand file tree Collapse file tree 1 file changed +9
-0
lines changed Expand file tree Collapse file tree 1 file changed +9
-0
lines changed Original file line number Diff line number Diff line change @@ -529,11 +529,20 @@ theorem PartialOrder.ext {A B : PartialOrder α}
529
529
ext x y
530
530
exact H x y
531
531
532
+ theorem PartialOrder.ext_lt {A B : PartialOrder α}
533
+ (H : ∀ x y : α, (haveI := A; x < y) ↔ x < y) : A = B := by
534
+ ext x y
535
+ rw [le_iff_lt_or_eq, @le_iff_lt_or_eq _ A, H]
536
+
532
537
theorem LinearOrder.ext {A B : LinearOrder α}
533
538
(H : ∀ x y : α, (haveI := A; x ≤ y) ↔ x ≤ y) : A = B := by
534
539
ext x y
535
540
exact H x y
536
541
542
+ theorem LinearOrder.ext_lt {A B : LinearOrder α}
543
+ (H : ∀ x y : α, (haveI := A; x < y) ↔ x < y) : A = B :=
544
+ LinearOrder.toPartialOrder_injective (PartialOrder.ext_lt H)
545
+
537
546
/-- Given a relation `R` on `β` and a function `f : α → β`, the preimage relation on `α` is defined
538
547
by `x ≤ y ↔ f x ≤ f y`. It is the unique relation on `α` making `f` a `RelEmbedding` (assuming `f`
539
548
is injective). -/
You can’t perform that action at this time.
0 commit comments