Skip to content

Commit

Permalink
Merge pull request #2101 from jdchristensen/small-smallness-fixes
Browse files Browse the repository at this point in the history
Smallness: export in HoTT.v and rename a few things
  • Loading branch information
jdchristensen authored Sep 26, 2024
2 parents b7b3d57 + 8c4a137 commit b008260
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 3 deletions.
1 change: 1 addition & 0 deletions theories/HoTT.v
Original file line number Diff line number Diff line change
Expand Up @@ -26,6 +26,7 @@ Require Export HoTT.Functorish.
Require Export HoTT.Factorization.
Require Export HoTT.Constant.

Require Export HoTT.Universes.Smallness.
Require Export HoTT.Universes.TruncType.
Require Export HoTT.Universes.ObjectClassifier.
Require Export HoTT.Universes.DProp.
Expand Down
6 changes: 3 additions & 3 deletions theories/Universes/Smallness.v
Original file line number Diff line number Diff line change
Expand Up @@ -54,7 +54,7 @@ Proof.
Defined.

(** If a map has small codomain and fibers, then the domain is small. *)
Definition issmall_codomain_issmall_fibers@{i j | } {X Y : Type@{j}}
Definition issmall_issmall_codomain_fibers@{i j | } {X Y : Type@{j}}
(f : X -> Y)
(sY : IsSmall@{i j} Y)
(sF : forall y : Y, IsSmall@{i j} (hfiber f y))
Expand All @@ -77,7 +77,7 @@ Definition issmall_inhabited_issmall@{i j k | i < k, j <= k} `{PropResizing} `{U
: IsSmall@{i j} X.
Proof.
(* Since [IsSmall] is cumulative in the universe [j], it suffices to prove [IsSmall@{i k} X] for [k] the universe that [IsSmall@{i j}] lives in. We think of [k] as max(i+1,j). *)
rapply (issmall_codomain_issmall_fibers@{i k} isX).
rapply (issmall_issmall_codomain_fibers@{i k} isX).
intro sX.
rapply sigma_closed_issmall.
Defined.
Expand Down Expand Up @@ -173,7 +173,7 @@ Proof.
Defined.

(** If a map has n-locally small codomain and fibers, then the domain is n-locally small. *)
Definition islocallysmall_codomain_islocallysmall_fibers@{i j k | i < k, j <= k}
Definition islocallysmall_islocallysmall_codomain_fibers@{i j k | i < k, j <= k}
(n : nat) {X Y : Type@{j}} (f : X -> Y)
(sY : IsLocallySmall@{i j k} n Y)
(sF : forall y : Y, IsLocallySmall@{i j k} n (hfiber f y))
Expand Down

0 comments on commit b008260

Please sign in to comment.