Skip to content
Draft
Show file tree
Hide file tree
Changes from all commits
Commits
Show all changes
65 commits
Select commit Hold shift + click to select a range
9f7ceb0
some informal proofs for truncation equivalences
fredrik-bakke Sep 23, 2025
c97413c
edits
fredrik-bakke Sep 23, 2025
1fff72c
edit
fredrik-bakke Sep 23, 2025
e799da9
edits
fredrik-bakke Sep 23, 2025
92788a9
refactor, simplify, and informalize proof of `is-connected-map-is-con…
fredrik-bakke Sep 23, 2025
7b2dcb0
Retractions of `k`-equivalences are `k`-equivalences
fredrik-bakke Sep 23, 2025
004e459
simplify informal proof slightly
fredrik-bakke Sep 23, 2025
5b8442e
edits
fredrik-bakke Sep 25, 2025
ec05b43
edits
fredrik-bakke Sep 25, 2025
9ab3cc4
Merge branch 'master' into informal-proof-truncation-equivs
fredrik-bakke Sep 25, 2025
26a8447
more edits
fredrik-bakke Sep 25, 2025
08301c9
edits `connected-maps`
fredrik-bakke Sep 25, 2025
85b1305
edits
fredrik-bakke Sep 25, 2025
fb3887f
pre-commit
fredrik-bakke Sep 25, 2025
7f2f7cd
`subuniverse-connected-maps`
fredrik-bakke Sep 25, 2025
c0f65ce
`K`-connected maps are closed under cobase change
fredrik-bakke Sep 25, 2025
f00102e
`K`-connected maps are closed under retracts of maps informal proof
fredrik-bakke Sep 26, 2025
8943ae1
edits
fredrik-bakke Sep 28, 2025
3ed7b96
Coproducts of `K`-connected maps
fredrik-bakke Sep 28, 2025
35d57cb
edits
fredrik-bakke Sep 29, 2025
65cf586
lots of edits
fredrik-bakke Sep 29, 2025
a36ebc1
`is-equiv-postcomp-extension`
fredrik-bakke Sep 29, 2025
f1945a4
map-separated types
fredrik-bakke Sep 29, 2025
2140a78
`is-subuniverse-localization-map`
fredrik-bakke Sep 29, 2025
f946d4c
fix indentation
fredrik-bakke Sep 29, 2025
b4fc42d
fix a silly name
fredrik-bakke Sep 30, 2025
d13feda
fix another silly name
fredrik-bakke Sep 30, 2025
68dae00
`is-trunc-map-postcomp-extension`
fredrik-bakke Sep 30, 2025
242d30d
`postcomposition-extensions-maps`
fredrik-bakke Sep 30, 2025
c2e67a9
edits `extensions-maps`
fredrik-bakke Sep 30, 2025
7e76f72
fix import
fredrik-bakke Sep 30, 2025
f8a4c1f
rename files
fredrik-bakke Sep 30, 2025
b3d9701
fix links in `foundation.projective-types`
fredrik-bakke Oct 1, 2025
c31efdc
work separation, subuniverse connected maps and equivalences
fredrik-bakke Oct 2, 2025
d5fc08b
more fiber computation
fredrik-bakke Oct 2, 2025
a6a95fb
`is-subuniverse-equiv-terminal-map-fibers-is-inhabited-family-fiber-Π…
fredrik-bakke Oct 2, 2025
2e104cc
round off conditions subuniverse connected maps
fredrik-bakke Oct 2, 2025
225c8c0
pre-commit
fredrik-bakke Oct 2, 2025
f6b197e
forgot one
fredrik-bakke Oct 2, 2025
5827064
fix a link
fredrik-bakke Oct 3, 2025
d79da3e
modulation!
fredrik-bakke Oct 3, 2025
8cfb546
modulation!
fredrik-bakke Oct 3, 2025
479b9e4
more edits
fredrik-bakke Oct 3, 2025
018c2de
another pushout characterization of smash
fredrik-bakke Oct 22, 2025
62797d1
(𝑛+1)-truncated pointed maps induce 𝑛-truncated maps on loop spaces
fredrik-bakke Oct 23, 2025
261dae1
Merge branch 'master' into informal-proof-truncation-equivs
fredrik-bakke Oct 23, 2025
c999911
edits loop spaces
fredrik-bakke Oct 23, 2025
632bd92
The loop space of a (𝑘+1)-truncated type is 𝑘-truncated
fredrik-bakke Oct 24, 2025
c7347c9
If A is (𝑛+𝑘)-truncated then ΩⁿA is 𝑘-truncated
fredrik-bakke Oct 24, 2025
f15dde7
mildly simplify a proof
fredrik-bakke Oct 24, 2025
da3b38a
add a link
fredrik-bakke Oct 24, 2025
fe3ed62
Computing extension types as a dependent product
fredrik-bakke Oct 25, 2025
dd2a0b7
edits
fredrik-bakke Oct 31, 2025
542c7e0
revert stupid name change
fredrik-bakke Nov 6, 2025
8e8c485
revert stupid name change
fredrik-bakke Nov 6, 2025
282c71d
revert stupid name change
fredrik-bakke Nov 6, 2025
ce1e7fd
fix a renaming mistake
fredrik-bakke Nov 6, 2025
2e972ca
Merge branch 'master' into informal-proof-truncation-equivs
fredrik-bakke Nov 6, 2025
3ed97cc
revert another naming change
fredrik-bakke Nov 6, 2025
e581125
Revert "revert another naming change"
fredrik-bakke Nov 6, 2025
15517ad
fixes
fredrik-bakke Nov 6, 2025
00260e6
Merge branch 'master' into informal-proof-truncation-equivs
fredrik-bakke Nov 6, 2025
0aee02d
Merge branch 'master' into relative-separations
fredrik-bakke Nov 12, 2025
a07e64b
fix merge
fredrik-bakke Nov 12, 2025
540daec
fix merge 2
fredrik-bakke Nov 12, 2025
File filter

Filter by extension

Filter by extension

Conversations
Failed to load comments.
Loading
Jump to
Jump to file
Failed to load files.
Loading
Diff view
Diff view
2 changes: 2 additions & 0 deletions src/orthogonal-factorization-systems.lagda.md
Original file line number Diff line number Diff line change
Expand Up @@ -71,6 +71,8 @@ open import orthogonal-factorization-systems.reflective-global-subuniverses publ
open import orthogonal-factorization-systems.reflective-modalities public
open import orthogonal-factorization-systems.reflective-subuniverses public
open import orthogonal-factorization-systems.regular-cd-structures public
open import orthogonal-factorization-systems.relative-separations-types-global-subuniverses public
open import orthogonal-factorization-systems.relative-separations-types-subuniverses public
open import orthogonal-factorization-systems.sigma-closed-modalities public
open import orthogonal-factorization-systems.sigma-closed-reflective-modalities public
open import orthogonal-factorization-systems.sigma-closed-reflective-subuniverses public
Expand Down
Original file line number Diff line number Diff line change
@@ -0,0 +1,90 @@
# Relative separations of types at global subuniverses

```agda
module orthogonal-factorization-systems.relative-separations-types-global-subuniverses where
```

<details><summary>Imports</summary>

```agda
open import foundation.dependent-pair-types
open import foundation.equivalences
open import foundation.global-subuniverses
open import foundation.universe-levels

open import foundation-core.function-types
open import foundation-core.identity-types
open import foundation-core.propositions

open import orthogonal-factorization-systems.extensions-maps
open import orthogonal-factorization-systems.postcomposition-extensions-maps
```

</details>

## Idea

Consider a [global subuniverse](foundation.global-subuniverses.md) `K` and a map
`δ : X → Y`. A type `A` is said to be
{{#concept "`K`-separated relative to `δ`" Agda=is-rel-separated}} if the type
of extensions of any map `f : X → A` along `δ` is in `K`.

As a special case, a type `A` is _`K`-separated_ if it is `K`-separated relative
to the terminal projection at a two-element type.

## Definitions

### The predicate of being separated

```agda
module _
{α : Level → Level} {l1 l2 l3 : Level} (K : global-subuniverse α)
{X : UU l1} {Y : UU l2} (δ : X → Y)
where

is-rel-separated : (A : UU l3) → UU (α (l1 ⊔ l2 ⊔ l3) ⊔ l1 ⊔ l3)
is-rel-separated A =
(f : X → A) → is-in-global-subuniverse K (extension-map δ f)

is-prop-is-rel-separated :
(A : UU l3) → is-prop (is-rel-separated A)
is-prop-is-rel-separated A =
is-prop-Π (λ f → is-prop-is-in-global-subuniverse K (extension-map δ f))

is-rel-separated-Prop :
(A : UU l3) → Prop (α (l1 ⊔ l2 ⊔ l3) ⊔ l1 ⊔ l3)
is-rel-separated-Prop A =
( is-rel-separated A , is-prop-is-rel-separated A)
```

### The global subuniverse of `K`-separated types relative to `δ`

```agda
module _
{α : Level → Level} {l1 l2 : Level} (K : global-subuniverse α)
{X : UU l1} {Y : UU l2} (δ : X → Y)
where

is-closed-under-equiv-rel-separated-global-subuniverse :
{l4 l5 : Level} →
is-closed-under-equiv-subuniverses
( λ l3 → α (l1 ⊔ l2 ⊔ l3) ⊔ l1 ⊔ l3)
( λ l3 → is-rel-separated-Prop {l3 = l3} K δ)
( l4)
( l5)
is-closed-under-equiv-rel-separated-global-subuniverse A B e H f =
is-closed-under-equiv-global-subuniverse K
( extension-map δ (map-inv-equiv e ∘ f))
( extension-map δ f)
( inv-equiv (equiv-postcomp-extension-map δ f (inv-equiv e)))
( H (map-inv-equiv e ∘ f))

rel-separated-global-subuniverse :
global-subuniverse (λ l3 → α (l1 ⊔ l2 ⊔ l3) ⊔ l1 ⊔ l3)
rel-separated-global-subuniverse =
λ where
.subuniverse-global-subuniverse l3 →
is-rel-separated-Prop K δ
.is-closed-under-equiv-global-subuniverse →
is-closed-under-equiv-rel-separated-global-subuniverse
```
Original file line number Diff line number Diff line change
@@ -0,0 +1,55 @@
# Relative separations of types at subuniverses

```agda
module orthogonal-factorization-systems.relative-separations-types-subuniverses where
```

<details><summary>Imports</summary>

```agda
open import foundation.dependent-pair-types
open import foundation.subuniverses
open import foundation.universe-levels

open import foundation-core.identity-types
open import foundation-core.propositions

open import orthogonal-factorization-systems.extensions-maps
```

</details>

## Idea

Consider a [subuniverse](foundation.subuniverses.md) `K` and a map `δ : X → Y`.
A type `A` is said to be
{{#concept "`K`-separated relative to `δ`" Agda=is-rel-separated'}} if the type
of extensions of any map `f : X → A` along `δ` is in `K`.

## Definitions

### The predicate of being rel-separated

```agda
module _
{l1 l2 l3 : Level} (K : subuniverse l1 l2)
{X : UU l1} {Y : UU l1} (δ : X → Y)
where

is-rel-separated' : (A : UU l1) → UU (l1 ⊔ l2)
is-rel-separated' A = (f : X → A) → is-in-subuniverse K (extension-map δ f)

is-prop-is-rel-separated' :
(A : UU l1) → is-prop (is-rel-separated' A)
is-prop-is-rel-separated' A =
is-prop-Π (λ f → is-prop-is-in-subuniverse K (extension-map δ f))

is-rel-separated'-Prop :
(A : UU l1) → Prop (l1 ⊔ l2)
is-rel-separated'-Prop A =
( is-rel-separated' A , is-prop-is-rel-separated' A)
```

## See also

- [Relative separations of types at global subuniverses](orthogonal-factorization-systems.relative-separations-types-global-subuniverses.md)