Skip to content

Commit

Permalink
generalize facts from ordinals to all injective types
Browse files Browse the repository at this point in the history
Co-authored-by: Tom de Jong <[email protected]>
  • Loading branch information
martinescardo and tomdjong committed Jul 18, 2024
1 parent e31bb20 commit 5757337
Showing 1 changed file with 36 additions and 5 deletions.
41 changes: 36 additions & 5 deletions source/Taboos/Decomposability.lagda
Original file line number Diff line number Diff line change
Expand Up @@ -394,11 +394,12 @@ of them if we are given a proof of decomposability.

Added 9th September 2022 by Tom de Jong.

After a discussion with Martín on 8th September 2022, we noticed that the
decomposability theorem can be generalised from Ord 𝓤 to any locally small
𝓤-sup-lattice with two distinct points. (This is indeed a generalisation because
Ord 𝓤 is a locally small 𝓤-sup-lattice, at least in the presence of small set
quotients or set replacement, see Ordinals.OrdinalOfOrdinalsSuprema.)
After a discussion with Martín on 8th September 2022, we noticed that
the decomposability theorem can be generalised from Ord 𝓤 to any
locally small 𝓤-sup-lattice with two distinct points. (This is indeed
a generalisation because Ord 𝓤 is a locally small 𝓤-sup-lattice, at
least in the presence of small set quotients or set replacement, see
Ordinals.OrdinalOfOrdinalsSuprema.)

One direction is still given by the lemma above:
WEM-gives-decomposition-of-two-pointed-types⁺ :
Expand Down Expand Up @@ -558,6 +559,36 @@ decomposition-of-ordinals-type-gives-WEM-bis {𝓤} =

\end{code}

Added by Martin Escardo and Tom de Jong 18th July 2024. We generalize
a fact given above from ordinals to injective types.

\begin{code}

module decomposability-bis (pt : propositional-truncations-exist) where

open PropositionalTruncation pt
open decomposability pt

ainjective-type-decomposable-iff-WEM
: (D : 𝓤 ̇ )
→ ainjective-type D 𝓤 𝓥
→ has-two-distinct-points D
→ decomposable D ↔ WEM 𝓤
ainjective-type-decomposable-iff-WEM D D-ainj htdp =
∥∥-rec (WEM-is-prop fe) (decomposition-of-ainjective-type-gives-WEM D D-ainj) ,
(λ wem → ∣ WEM-gives-decomposition-of-two-pointed-types wem D htdp ∣)

ainjective-type-decomposability-gives-decomposition
: (D : 𝓤 ̇ )
→ ainjective-type D 𝓤 𝓥
→ has-two-distinct-points D
→ decomposable D
→ decomposition D
ainjective-type-decomposability-gives-decomposition {𝓤} D D-ainj htdp δ =
WEM-gives-decomposition-of-two-pointed-types (lr-implication (ainjective-type-decomposable-iff-WEM D D-ainj htdp) δ) D htdp

\end{code}

Added by Martin Escardo 10th June 2024. From any non-trivial,
totally separated, injective type we get the double negation of the
principle of weak excluded middle. Here by non-trivial we mean that
Expand Down

0 comments on commit 5757337

Please sign in to comment.