The category of Heyting algebras #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file defines HeytAlg
, the category of Heyting algebras.
The category of Heyting algebras.
Equations
@[protected, instance]
@[protected, instance]
Equations
- X.heyting_algebra = X.str
Construct a bundled HeytAlg
from a heyting_algebra
.
Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
- HeytAlg.bundled_hom = {to_fun := λ (α β : Type u_1) [_inst_1 : heyting_algebra α] [_inst_2 : heyting_algebra β], coe_fn, id := heyting_hom.id, comp := heyting_hom.comp, hom_ext := HeytAlg.bundled_hom._proof_1, id_to_fun := HeytAlg.bundled_hom._proof_2, comp_to_fun := HeytAlg.bundled_hom._proof_3}
@[protected, instance]
@[simp]
@[simp]
@[protected, instance]
@[simp]
Constructs an isomorphism of Heyting algebras from an order isomorphism between them.
Equations
- HeytAlg.iso.mk e = {hom := ↑e, inv := ↑(e.symm), hom_inv_id' := _, inv_hom_id' := _}