{-# OPTIONS -vtactic.hlevel:10 #-}
open import 1Lab.Prelude

open import Data.Power
open import Data.Bool
open import Data.Dec
open import Data.Sum
module Data.Power.Complemented where

Complemented subobjects🔗

A subobject of a type is called complemented if there is a subobject such that 1, and Because of lattice structure, these containments suffice to establish equality.

private variable
: Level
  A : Type ℓ
  p q r : ℙ A
is-complemented :  {} {A : Type ℓ} (p : ℙ A)  Type _
is-complemented {A = A} p = Σ[ p⁻¹ ∈ ℙ A ]
  ((p ∩ p⁻¹ ⊆ minimal) × (maximal ⊆ p ∪ p⁻¹))

More conventionally, in constructive mathematics, we may say a subobject is decidable if its associated predicate is pointwise a decidable type. It turns out that these conditions are equivalent: a subobject is decidable if, and only if, it is complemented. It’s immediate that decidable subobjects are complemented: given a decision procedure the fibres and are disjoint and their union is all of

is-decidable :  {} {A : Type ℓ} (p : ℙ A)  Type _
is-decidable {A = A} p = (a : A)  Dec (a ∈ p)

is-decidable→is-complemented : (p : ℙ A)  is-decidable p  is-complemented p
is-decidable→is-complemented {A = A} p dec = inv , intersection , union where
  inv : ℙ A
  inv x = el (¬ (x ∈ p)) (hlevel 1)

  intersection : (p ∩ inv) ⊆ minimal
  intersection x (x∈p , x∉p) = x∉p x∈p

  union : maximal ⊆ (p ∪ inv)
  union x wit with dec x
  ... | yes x∈p = inc (inl x∈p)
  ... | no x∉p = inc (inr x∉p)

For the converse, since decidability of a proposition is itself a proposition, it suffices to assume we have an inhabitant of Assuming that we must show that But by the definition of complemented subobject, the intersection is empty.

is-complemented→is-decidable : (p : ℙ A)  is-complemented p  is-decidable p
is-complemented→is-decidable p (p⁻¹ , intersection , union) elt =
  case union elt tt of λ where
    (inl x∈p)   yes x∈p
    (inr x∈¬p)  no λ x∈p  intersection elt (x∈p , x∈¬p)

Decidable subobject classifiers🔗

In the same way that we have a (large) type of all propositions of size the decidable (complemented) subobjects also have a classifying object: Any two-element type with decidable equality! This can be seen as a local instance of excluded middle: the complemented subobjects are precisely those satisfying and so they are classified by the “classical subobject classifier”

decidable-subobject-classifier
  : {A : Type ℓ}  (A  Bool)(Σ[ p ∈ ℙ A ] (is-decidable p))
decidable-subobject-classifier {A = A} = eqv where

In much the same way that the subobject represented by a map is the fibre over the subobject represented by a map is the fibre over This is a decidable subobject because has decidable equality.

  to : (A  Bool)  (Σ[ p ∈ ℙ A ] (is-decidable p))
  to map .fst x = el (map x ≡ true) (hlevel 1)
  to map .snd p = Bool-elim  p  Dec (p ≡ true))
    (yes refl) (no  p  true≠false (sym p))) (map p)

Conversely, to each decidable subobject and element we associate a boolean such that if and only if Projecting the boolean and forgetting the equivalence gives us a map associated with as desired; The characterisation of serves to smoothen the proof that this process is inverse to taking fibres over

  from : (pr : Σ[ p ∈ ℙ A ] (is-decidable p)) (x : A)
        (Σ[ b ∈ Bool ] ((b ≡ true)(x ∈ pr .fst)))
  from (p , dec) elt = Dec-elim  _  Σ Bool  b  (b ≡ true)(elt ∈ p)))
     y  true , prop-ext!  _  y)  _  refl))
     x∉p  false , prop-ext!
       p  absurd (true≠false (sym p)))
       x  absurd (x∉p x)))
    (dec elt)

  eqv = Iso→Equiv λ where
    .fst  to
    .snd .is-iso.inv p x  from p x .fst
    .snd .is-iso.rinv pred  Σ-prop-path! $ ℙ-ext
       x w  from pred x .snd .fst w)
       x p  Equiv.from (from pred x .snd) p)
    .snd .is-iso.linv pred  funext λ x 
      Bool-elim  p  from (to λ _  p) x .fst ≡ p) refl refl (pred x)

  1. where is regarded as the top element of its own subobject lattice↩︎