Documentation

Mathlib.Order.Heyting.Boundary

Co-Heyting boundary #

The boundary of an element of a co-Heyting algebra is the intersection of its Heyting negation with itself. The boundary in the co-Heyting algebra of closed sets coincides with the topological boundary.

Main declarations #

Notation #

∂ a is notation for Coheyting.boundary a in locale Heyting.

def Coheyting.boundary {α : Type u_1} [CoheytingAlgebra α] (a : α) :
α

The boundary of an element of a co-Heyting algebra is the intersection of its Heyting negation with itself. Note that this is always for a boolean algebra.

Equations
Instances For

    The boundary of an element of a co-Heyting algebra.

    Equations
    Instances For
      theorem Coheyting.inf_hnot_self {α : Type u_1} [CoheytingAlgebra α] (a : α) :
      theorem Coheyting.boundary_le {α : Type u_1} [CoheytingAlgebra α] {a : α} :
      @[simp]
      @[simp]
      theorem Coheyting.hnot_boundary {α : Type u_1} [CoheytingAlgebra α] (a : α) :
      theorem Coheyting.boundary_inf {α : Type u_1} [CoheytingAlgebra α] (a b : α) :

      Leibniz rule for the co-Heyting boundary.

      @[simp]
      theorem Coheyting.boundary_idem {α : Type u_1} [CoheytingAlgebra α] (a : α) :
      theorem Coheyting.hnot_eq_top_iff_exists_boundary {α : Type u_1} [CoheytingAlgebra α] {a : α} :
      a = ∃ (b : α), boundary b = a
      @[simp]
      theorem Coheyting.boundary_eq_bot {α : Type u_1} [BooleanAlgebra α] (a : α) :