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

Commit c8a43b4

Browse files
committed
feat(order/hom/complete_lattice): inf as an Inf_hom and sup as a Sup_hom (#18023)
Introduces a new definition `inf_Inf_hom` on a complete lattice which is the map `(a, b) ↦ a ⊓ b` as an `Inf_hom`. This is required for #17426. For completeness we also include the equivalent `sup` definition. Co-authored-by: Christopher Hoskin <mans0954@users.noreply.github.com>
1 parent 7ea6047 commit c8a43b4

File tree

1 file changed

+15
-0
lines changed

1 file changed

+15
-0
lines changed

src/order/hom/complete_lattice.lean

Lines changed: 15 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -626,3 +626,18 @@ See also `complete_lattice_hom.set_preimage`. -/
626626
right_inv := λ s, by simp only [← image_comp, equiv.self_comp_symm, id.def, image_id'],
627627
map_rel_iff' :=
628628
λ s t, ⟨λ h, by simpa using @monotone_image _ _ e.symm _ _ h, λ h, monotone_image h⟩ }
629+
630+
section
631+
632+
variables (α) [complete_lattice α]
633+
634+
/-- The map `(a, b) ↦ a ⊓ b` as an `Inf_hom`. -/
635+
@[simps] def inf_Inf_hom : Inf_hom (α × α) α :=
636+
{ to_fun := λ x, x.1 ⊓ x.2,
637+
map_Inf' := λ s, by simp_rw [prod.fst_Inf, prod.snd_Inf, Inf_image, infi_inf_eq], }
638+
639+
/-- The map `(a, b) ↦ a ⊔ b` as a `Sup_hom`. -/
640+
@[simps] def sup_Sup_hom : Sup_hom (α × α) α :=
641+
{ to_fun := λ x, x.1 ⊔ x.2, map_Sup' := (inf_Inf_hom αᵒᵈ).map_Inf' }
642+
643+
end

0 commit comments

Comments
 (0)