mathlib3 documentation

order.category.HeytAlg

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.

@[protected, instance]
Equations
def HeytAlg.of (α : Type u_1) [heyting_algebra α] :

Construct a bundled HeytAlg from a heyting_algebra.

Equations
@[simp]
theorem HeytAlg.coe_of (α : Type u_1) [heyting_algebra α] :
@[protected, instance]
Equations
@[protected, instance]
Equations
@[simp]
theorem HeytAlg.iso.mk_hom {α β : HeytAlg} (e : α ≃o β) :
@[simp]
theorem HeytAlg.iso.mk_inv {α β : HeytAlg} (e : α ≃o β) :
def HeytAlg.iso.mk {α β : HeytAlg} (e : α ≃o β) :
α β

Constructs an isomorphism of Heyting algebras from an order isomorphism between them.

Equations