Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit f6c8aff

Browse files
committed
feat(order/zorn) : chain_univ (#9162)
`univ` is a `r`-chain iff `r` is trichotomous
1 parent 5b702ec commit f6c8aff

File tree

1 file changed

+18
-0
lines changed

1 file changed

+18
-0
lines changed

src/order/zorn.lean

Lines changed: 18 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -92,6 +92,24 @@ lemma chain.mono {c c'} :
9292
c' ⊆ c → chain c → chain c' :=
9393
pairwise_on.mono
9494

95+
lemma chain_of_trichotomous [is_trichotomous α r] (s : set α) :
96+
chain s :=
97+
begin
98+
intros a _ b _ hab,
99+
obtain h | h | h := @trichotomous _ r _ a b,
100+
{ exact or.inl h },
101+
{ exact (hab h).elim },
102+
{ exact or.inr h }
103+
end
104+
105+
lemma chain_univ_iff :
106+
chain (univ : set α) ↔ is_trichotomous α r :=
107+
begin
108+
refine ⟨λ h, ⟨λ a b , _⟩, λ h, @chain_of_trichotomous _ _ h univ⟩,
109+
rw [or.left_comm, or_iff_not_imp_left],
110+
exact h a trivial b trivial,
111+
end
112+
95113
lemma chain.directed_on [is_refl α r] {c} (H : chain c) :
96114
directed_on (≺) c :=
97115
λ x hx y hy,

0 commit comments

Comments
 (0)