Skip to content

Commit

Permalink
chore(order/galois_connection): upgrade is_glb_l to is_least_l (#…
Browse files Browse the repository at this point in the history
…10606)

* upgrade `galois_connection.is_glb_l` to `galois_connection.is_least_l`;
* upgrade `galois_connection.is_lub_l` to `galois_connection.is_greatest_l`.
  • Loading branch information
urkud committed Dec 4, 2021
1 parent 3479b7f commit 5d0e65a
Showing 1 changed file with 8 additions and 4 deletions.
12 changes: 8 additions & 4 deletions src/order/galois_connection.lean
Expand Up @@ -109,11 +109,15 @@ lemma is_lub_l_image {s : set α} {a : α} (h : is_lub s a) : is_lub (l '' s) (l
lemma is_glb_u_image {s : set β} {b : β} (h : is_glb s b) : is_glb (u '' s) (u b) :=
gc.dual.is_lub_l_image h

lemma is_glb_l {a : α} : is_glb { b | a ≤ u b } (l a) :=
λ b, gc.l_le, λ b h, h $ gc.le_u_l _
lemma is_least_l {a : α} : is_least {b | a ≤ u b} (l a) :=
⟨gc.le_u_l _, λ b hb, gc.l_le hb

lemma is_lub_u {b : β} : is_lub { a | l a ≤ b } (u b) :=
⟨λ b, gc.le_u, λ b h, h $ gc.l_u_le _⟩
lemma is_greatest_u {b : β} : is_greatest {a | l a ≤ b} (u b) :=
gc.dual.is_least_l

lemma is_glb_l {a : α} : is_glb {b | a ≤ u b} (l a) := gc.is_least_l.is_glb

lemma is_lub_u {b : β} : is_lub { a | l a ≤ b } (u b) := gc.is_greatest_u.is_lub

end

Expand Down

0 comments on commit 5d0e65a

Please sign in to comment.