Skip to content

Commit

Permalink
feat(Order/CompleteLattice): instances for CompleteSemilatticeInf / C…
Browse files Browse the repository at this point in the history
…ompleteSemilatticeSup for Dual types (#20246)
  • Loading branch information
Bergschaf committed Jan 2, 2025
1 parent 45302a8 commit 0673d5a
Showing 1 changed file with 9 additions and 0 deletions.
9 changes: 9 additions & 0 deletions Mathlib/Order/CompleteLattice.lean
Original file line number Diff line number Diff line change
Expand Up @@ -173,6 +173,15 @@ theorem sInf_singleton {a : α} : sInf {a} = a :=

end

instance {α : Type*} [CompleteSemilatticeInf α] : CompleteSemilatticeSup αᵒᵈ where
le_sSup := @CompleteSemilatticeInf.sInf_le α _
sSup_le := @CompleteSemilatticeInf.le_sInf α _

instance {α : Type*} [CompleteSemilatticeSup α] : CompleteSemilatticeInf αᵒᵈ where
le_sInf := @CompleteSemilatticeSup.sSup_le α _
sInf_le := @CompleteSemilatticeSup.le_sSup α _


/-- A complete lattice is a bounded lattice which has suprema and infima for every subset. -/
class CompleteLattice (α : Type*) extends Lattice α, CompleteSemilatticeSup α,
CompleteSemilatticeInf α, Top α, Bot α where
Expand Down

0 comments on commit 0673d5a

Please sign in to comment.