Skip to content

Commit

Permalink
Merge pull request #226 from m-lindgren/remove-imports
Browse files Browse the repository at this point in the history
Remove some unnecessary imports.
  • Loading branch information
benediktahrens committed Nov 5, 2022
2 parents b507c6f + 53b8c51 commit 71a4afe
Show file tree
Hide file tree
Showing 27 changed files with 85 additions and 46 deletions.
1 change: 1 addition & 0 deletions TypeTheory/Articles/ALV_2017.v
Original file line number Diff line number Diff line change
Expand Up @@ -15,6 +15,7 @@ This file should contain _no substantial formalisation_, and should not be impor

Require Import UniMath.Foundations.Sets.
Require Import TypeTheory.Auxiliary.CategoryTheoryImports.
Require Import UniMath.CategoryTheory.rezk_completion.
Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.

Expand Down
1 change: 1 addition & 0 deletions TypeTheory/Articles/ALV_2018.v
Original file line number Diff line number Diff line change
Expand Up @@ -12,6 +12,7 @@ This file is intended to accompany a sequel article to ALV-2017, currently in (d

Require Import UniMath.Foundations.Sets.
Require Import TypeTheory.Auxiliary.CategoryTheoryImports.
Require Import UniMath.CategoryTheory.rezk_completion.
Require Import UniMath.CategoryTheory.DisplayedCats.Core.
Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Expand Down
3 changes: 2 additions & 1 deletion TypeTheory/Auxiliary/ArrowCategory.v
Original file line number Diff line number Diff line change
Expand Up @@ -2,7 +2,8 @@
Require Import UniMath.Foundations.All.
Require Import UniMath.MoreFoundations.All.

Require Import UniMath.CategoryTheory.All.
Require Import UniMath.CategoryTheory.Core.Prelude.
Require Import UniMath.CategoryTheory.ArrowCategory.

Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Expand Down
10 changes: 8 additions & 2 deletions TypeTheory/Auxiliary/CategoryTheory.v
Original file line number Diff line number Diff line change
@@ -1,18 +1,24 @@
Require Import UniMath.Foundations.All.
Require Import UniMath.MoreFoundations.All.

Require Import UniMath.CategoryTheory.All.
Require Import TypeTheory.Auxiliary.CategoryTheoryImports.
Require Import UniMath.CategoryTheory.CategoryEquality.
Require Import UniMath.CategoryTheory.DisplayedCats.ComprehensionC.

(* a few libraries need to be reloaded after “All”,
to claim precedence on overloaded names *)

Require Import UniMath.CategoryTheory.limits.graphs.limits.
Require Import UniMath.CategoryTheory.limits.pullbacks.
Require Import UniMath.CategoryTheory.limits.graphs.terminal.
Require Import UniMath.CategoryTheory.limits.graphs.initial.

Require Import TypeTheory.Auxiliary.Auxiliary.


(** * General notations and scopes *)

(** We redeclare this notation, along with a new scope . *)
Declare Scope mor_scope.
Notation "ff ;; gg" := (compose ff gg)
(at level 50, left associativity, format "ff ;; gg")
: mor_scope.
Expand Down
2 changes: 1 addition & 1 deletion TypeTheory/Auxiliary/CategoryTheoryImports.v
Original file line number Diff line number Diff line change
Expand Up @@ -14,7 +14,7 @@ Require Export UniMath.CategoryTheory.whiskering.
Require Export UniMath.CategoryTheory.Adjunctions.Core.
Require Export UniMath.CategoryTheory.Equivalences.Core.
Require Export UniMath.CategoryTheory.precomp_fully_faithful.
Require Export UniMath.CategoryTheory.rezk_completion.
(* Require Export UniMath.CategoryTheory.rezk_completion. *)
Require Export UniMath.CategoryTheory.yoneda.
Require Export UniMath.CategoryTheory.categories.HSET.Core.
Require Export UniMath.CategoryTheory.categories.HSET.Univalence.
Expand Down
14 changes: 12 additions & 2 deletions TypeTheory/Auxiliary/DisplayedCategories.v
Original file line number Diff line number Diff line change
Expand Up @@ -2,7 +2,17 @@
Require Import UniMath.Foundations.All.
Require Import UniMath.MoreFoundations.All.

Require Import UniMath.CategoryTheory.All.
Require Import UniMath.CategoryTheory.Core.Prelude.
Require Import UniMath.CategoryTheory.DisplayedCats.Core.
Require Import UniMath.CategoryTheory.DisplayedCats.Functors.
Require Import UniMath.CategoryTheory.DisplayedCats.NaturalTransformations.
Require Import UniMath.CategoryTheory.DisplayedCats.Adjunctions.
Require Import UniMath.CategoryTheory.DisplayedCats.Equivalences.
Require Import UniMath.CategoryTheory.DisplayedCats.Fibrations.
Require Import UniMath.CategoryTheory.DisplayedCats.Total.

Require Import UniMath.CategoryTheory.Adjunctions.Core.
Require Import UniMath.CategoryTheory.Equivalences.Core.

Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Expand Down Expand Up @@ -268,7 +278,7 @@ Section Discrete_Fibrations.
(f : c' --> c) (d : D c) (d' : D c')
: (d' -->[f] d) = (lift_source is_discrete_fibration_D f d = d').
Proof.
apply univalenceweq.
apply univalence.
apply discrete_fibration_mor_weq.
Defined.

Expand Down
2 changes: 1 addition & 1 deletion TypeTheory/Auxiliary/Pullbacks.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
Require Import UniMath.Foundations.All.
Require Import UniMath.MoreFoundations.All.

Require Import UniMath.CategoryTheory.All.
Require Import UniMath.CategoryTheory.Core.Prelude.
(* a few libraries need to be reloaded after “All”,
to claim precedence on overloaded names *)
Require Import UniMath.CategoryTheory.limits.pullbacks.
Expand Down
5 changes: 4 additions & 1 deletion TypeTheory/Auxiliary/SetsAndPresheaves.v
Original file line number Diff line number Diff line change
@@ -1,16 +1,19 @@

Require Import UniMath.Foundations.All.
Require Import UniMath.MoreFoundations.All.
Require Import UniMath.Combinatorics.StandardFiniteSets.

Require Import UniMath.CategoryTheory.All.
(* a few libraries need to be reloaded after “All”,
to claim precedence on overloaded names *)
Require Import UniMath.CategoryTheory.limits.graphs.limits.
Require Import UniMath.CategoryTheory.limits.graphs.pullbacks.
Require Import UniMath.CategoryTheory.limits.pullbacks.
Require Import UniMath.CategoryTheory.categories.HSET.Limits.
Require Import UniMath.CategoryTheory.categories.HSET.Univalence.

Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Require Import TypeTheory.Auxiliary.CategoryTheoryImports.

(** * Presheaf generalities *)

Expand Down
6 changes: 5 additions & 1 deletion TypeTheory/Auxiliary/TypeOfMorphisms.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,11 @@

Require Import UniMath.Foundations.All.
Require Import UniMath.MoreFoundations.All.
Require Import UniMath.CategoryTheory.All.

Require Import UniMath.CategoryTheory.Core.Prelude.
Require Import UniMath.CategoryTheory.Equivalences.Core.
Require Import UniMath.CategoryTheory.Adjunctions.Core.
Require Import UniMath.CategoryTheory.FunctorCategory.

Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Expand Down
4 changes: 0 additions & 4 deletions TypeTheory/Categories/category_FAM.v
Original file line number Diff line number Diff line change
Expand Up @@ -9,10 +9,6 @@

Require Import UniMath.Foundations.All.
Require Import UniMath.MoreFoundations.All.
Require Import UniMath.CategoryTheory.Core.Categories.
Require Import UniMath.CategoryTheory.Core.Functors.
Require Import UniMath.CategoryTheory.yoneda.
Require Import UniMath.CategoryTheory.rezk_completion.

Require Import TypeTheory.Auxiliary.CategoryTheoryImports.
Require Import TypeTheory.Auxiliary.Auxiliary.
Expand Down
7 changes: 5 additions & 2 deletions TypeTheory/CompCats/FullyFaithfulDispFunctor.v
Original file line number Diff line number Diff line change
Expand Up @@ -35,7 +35,10 @@ Accessors for [ff_disp_functor]:

Require Import UniMath.Foundations.All.
Require Import UniMath.MoreFoundations.All.
Require Import UniMath.CategoryTheory.All.
Require Import UniMath.CategoryTheory.Core.Prelude.
Require Import UniMath.CategoryTheory.CategoryEquality.
Require Import UniMath.CategoryTheory.DisplayedCats.Core.
Require Import UniMath.CategoryTheory.DisplayedCats.Functors.

Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Expand Down Expand Up @@ -130,7 +133,7 @@ Section FullyFaithfulDispFunctor.
apply impred_iscontr. intros A'.
apply impred_iscontr. intros f.
use (@iscontrweqf (∑ mord : UU, mord = pr2 D Γ A -->[f] pr2 D Γ' A')).
- use (weqtotal2 (idweq _)). intros mord. apply univalenceweq.
- use (weqtotal2 (idweq _)). intros mord. apply univalence.
- apply iscontrcoconustot.
Defined.

Expand Down
1 change: 1 addition & 0 deletions TypeTheory/CwF/CwF_def.v
Original file line number Diff line number Diff line change
Expand Up @@ -17,6 +17,7 @@ Contents:
Require Import UniMath.Foundations.All.
Require Import UniMath.MoreFoundations.All.
Require Import TypeTheory.Auxiliary.CategoryTheoryImports.
Require Import UniMath.CategoryTheory.rezk_completion.

Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Expand Down
1 change: 1 addition & 0 deletions TypeTheory/CwF/RepMaps.v
Original file line number Diff line number Diff line change
Expand Up @@ -17,6 +17,7 @@ Contents:

Require Import UniMath.Foundations.Sets.
Require Import TypeTheory.Auxiliary.CategoryTheoryImports.
Require Import UniMath.CategoryTheory.rezk_completion.

Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Expand Down
4 changes: 3 additions & 1 deletion TypeTheory/CwF_TypeCat/CwF_SplitTypeCat_Defs.v
Original file line number Diff line number Diff line change
Expand Up @@ -24,7 +24,9 @@ NB: we follow UniMath’s convention that _category_ does not assume saturation/


Require Import UniMath.Foundations.Sets.
Require Import UniMath.CategoryTheory.All. (* TODO: work out what’s actually needed and move into [CategoryTheoryImports]. *)
Require Import UniMath.MoreFoundations.PartA.
Require Import UniMath.CategoryTheory.DisplayedCats.Core.
Require Import UniMath.CategoryTheory.DisplayedCats.Total.
Require Import TypeTheory.Auxiliary.CategoryTheoryImports.

Require Import TypeTheory.Auxiliary.Auxiliary.
Expand Down
5 changes: 4 additions & 1 deletion TypeTheory/CwF_TypeCat/TypeCat_Reassoc.v
Original file line number Diff line number Diff line change
Expand Up @@ -17,7 +17,10 @@ The equivalence is a bit more involved than one might hope; it proceeds in two m

Require Import UniMath.Foundations.All.
Require Import UniMath.MoreFoundations.All.
Require Import UniMath.CategoryTheory.All.
Require Import UniMath.CategoryTheory.Core.Prelude.
Require Import UniMath.CategoryTheory.limits.pullbacks.
Require Import UniMath.CategoryTheory.categories.HSET.All.
Require Import UniMath.CategoryTheory.opp_precat.

Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Expand Down
4 changes: 2 additions & 2 deletions TypeTheory/Initiality/Environments.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@

Require Import UniMath.MoreFoundations.All.
Require Import UniMath.CategoryTheory.All.
Require Import UniMath.CategoryTheory.Core.Prelude.

Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Expand Down Expand Up @@ -66,7 +66,7 @@ Section Environments.

Definition reind_idmap_environment {C : split_typecat}
{Γ : C} {n} (E : environment Γ n)
: reind_environment (id _) E = E.
: reind_environment (identity _) E = E.
Proof.
apply funextfun; intros i; apply reind_idmap_type_with_term.
Qed.
Expand Down
2 changes: 1 addition & 1 deletion TypeTheory/Initiality/Initiality.v
Original file line number Diff line number Diff line change
@@ -1,8 +1,8 @@
Require Import UniMath.MoreFoundations.All.
Require Import UniMath.MoreFoundations.Propositions.
(* [MoreFoundations.Propositions] seems to need individual importing to provide notation [∃!] as [iscontr_hProp] instead of just [iscontr]. TODO: figure out why; perhaps raise issue upstream? *)
Require Import UniMath.CategoryTheory.All.

Require Import UniMath.CategoryTheory.Core.Prelude.

Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Expand Down
2 changes: 1 addition & 1 deletion TypeTheory/Initiality/Interpretation.v
Original file line number Diff line number Diff line change
@@ -1,7 +1,7 @@
(** This file defines the interpretation function, from the syntax of our toy type theory into any split type-cat with suitable structure. *)

Require Import UniMath.MoreFoundations.All.
Require Import UniMath.CategoryTheory.All.
Require Import UniMath.CategoryTheory.Core.Prelude.

(* TODO: raise issue upstream: notation "_ ∘ _" is used for function-order composition of functions, but for diagrammatic-order composition of morphisms in categories! *)

Expand Down
4 changes: 3 additions & 1 deletion TypeTheory/Initiality/SyntacticCategory.v
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,9 @@
As a matter of organisation: all concrete lemmas involving derivations should live upstream in [TypingLemmas]; this file should simply package them up into the appropriate categorical structure. *)

Require Import UniMath.MoreFoundations.All.
Require Import UniMath.CategoryTheory.All.
Require Import UniMath.CategoryTheory.Core.Prelude.
Require Import UniMath.CategoryTheory.limits.pullbacks.
Require Import UniMath.CategoryTheory.limits.graphs.terminal.
Require UniMath.PAdics.lemmas. (* just for [setquotprpathsandR] *)

Require Import TypeTheory.Auxiliary.Auxiliary.
Expand Down
2 changes: 1 addition & 1 deletion TypeTheory/Initiality/SyntacticCategory_Structure.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
Require Import UniMath.MoreFoundations.All.
Require Import UniMath.CategoryTheory.All.
Require Import UniMath.CategoryTheory.Core.Categories.

Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Expand Down
15 changes: 3 additions & 12 deletions TypeTheory/Instances/Presheaves.v
Original file line number Diff line number Diff line change
Expand Up @@ -103,20 +103,11 @@ Written by: Anders Mörtberg, 2017
Require Import UniMath.Foundations.All.
Require Import UniMath.MoreFoundations.All.

Require Import UniMath.CategoryTheory.All.
(*
Require Import UniMath.CategoryTheory.Core.Functors.
Require Import UniMath.CategoryTheory.Adjunctions.Core.
Require Import UniMath.CategoryTheory.opp_precat.
Require Import UniMath.CategoryTheory.whiskering.
Require Import UniMath.CategoryTheory.Equivalences.Core.
Require Import TypeTheory.Auxiliary.CategoryTheoryImports.
Require Import UniMath.CategoryTheory.RightKanExtension.
Require Import UniMath.CategoryTheory.limits.graphs.limits.
Require Import UniMath.CategoryTheory.limits.graphs.eqdiag.
Require Import UniMath.CategoryTheory.limits.pullbacks.
Require Import UniMath.CategoryTheory.Presheaf.
Require Import UniMath.CategoryTheory.categories.HSET.Limits.
Require Import UniMath.CategoryTheory.ElementsOp.
*)

Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Require Import TypeTheory.Auxiliary.Pullbacks.
Expand Down
6 changes: 5 additions & 1 deletion TypeTheory/OtherDefs/CwF_Pitts_completion.v
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,11 @@

Require Import UniMath.Foundations.All.
Require Import UniMath.MoreFoundations.All.
Require Import UniMath.CategoryTheory.All.
Require Import UniMath.CategoryTheory.Core.Prelude.
Require Import UniMath.CategoryTheory.rezk_completion.
Require Import UniMath.CategoryTheory.opp_precat.
Require Import UniMath.CategoryTheory.categories.HSET.Core.
Require Import UniMath.CategoryTheory.categories.HSET.Univalence.

Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Expand Down
14 changes: 8 additions & 6 deletions TypeTheory/RelUniv/RelUnivTransfer.v
Original file line number Diff line number Diff line change
Expand Up @@ -21,6 +21,7 @@ TODO:
Require Import UniMath.Foundations.All.
Require Import UniMath.MoreFoundations.All.
Require Import TypeTheory.Auxiliary.CategoryTheoryImports.
Require Import UniMath.CategoryTheory.rezk_completion.

Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Expand All @@ -33,6 +34,7 @@ Require Import TypeTheory.RelUniv.Transport_along_Equivs.
Require Import TypeTheory.RelUniv.RelUniv_Cat_Simple.
Require Import TypeTheory.RelUniv.RelUniv_Cat.
Require Import UniMath.CategoryTheory.catiso.
Require Import UniMath.CategoryTheory.DisplayedCats.Constructions.

Section RelUniv_Transfer.

Expand Down Expand Up @@ -345,8 +347,8 @@ Section RelUniv_Transfer.
(S_ff : fully_faithful S).

Let E := ((S,, (invS,, (pr1 eta, pr1 eps)))
,, ((λ d, (pr2 (Constructions.pointwise_z_iso_from_nat_z_iso eta d )))
, (λ d', (pr2 (Constructions.pointwise_z_iso_from_nat_z_iso eps d')))))
,, ((λ d, (pr2 (pointwise_z_iso_from_nat_z_iso eta d )))
, (λ d', (pr2 (pointwise_z_iso_from_nat_z_iso eps d')))))
: equivalence_of_cats D D'.

Let AE := adjointificiation E.
Expand All @@ -359,8 +361,8 @@ Section RelUniv_Transfer.
_ (ε',,pr22 (adjointificiation E))
: z_iso (C:=[D', D']) (invS ∙ S) (functor_identity D').

Let ηx := Constructions.pointwise_z_iso_from_nat_z_iso (z_iso_inv_from_z_iso η).
Let αx := Constructions.pointwise_z_iso_from_nat_z_iso (α,,α_is_iso).
Let ηx := pointwise_z_iso_from_nat_z_iso (z_iso_inv_from_z_iso η).
Let αx := pointwise_z_iso_from_nat_z_iso (α,,α_is_iso).

Section Helpers.

Expand Down Expand Up @@ -565,8 +567,8 @@ Section RelUniv_Transfer.
: z_iso u'
(reluniv_functor_with_ess_surj (inv_reluniv_with_ess_surj u')).
Proof.
set (εx := Constructions.pointwise_z_iso_from_nat_z_iso ε).
set (εx' := Constructions.pointwise_z_iso_from_nat_z_iso
set (εx := pointwise_z_iso_from_nat_z_iso ε).
set (εx' := pointwise_z_iso_from_nat_z_iso
(z_iso_inv_from_z_iso ε)).
use make_z_iso.
- use tpair.
Expand Down
1 change: 1 addition & 0 deletions TypeTheory/RelUniv/RelUnivYonedaCompletion.v
Original file line number Diff line number Diff line change
Expand Up @@ -7,6 +7,7 @@
(** This file provides the result: given a universe in [preShv C] relative to the Yoneda embedding [ Yo : C -> preShv C ], this transfers to a similar relative universe in [ preShv (RC C) ]. i.e. on the Rezk-completion of [C]. *)
Require Import UniMath.Foundations.Sets.
Require Import TypeTheory.Auxiliary.CategoryTheoryImports.
Require Import UniMath.CategoryTheory.rezk_completion.

Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Expand Down
5 changes: 4 additions & 1 deletion TypeTheory/RelUniv/Transport_along_Equivs.v
Original file line number Diff line number Diff line change
Expand Up @@ -27,8 +27,11 @@


Require Import UniMath.Foundations.Sets.
Require Import UniMath.CategoryTheory.All.

Require Import UniMath.CategoryTheory.precomp_fully_faithful.
Require Import UniMath.CategoryTheory.precomp_ess_surj.

Require Import TypeTheory.Auxiliary.CategoryTheoryImports.
Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Require Import TypeTheory.Auxiliary.SetsAndPresheaves.
Expand Down
8 changes: 6 additions & 2 deletions TypeTheory/TypeCat/Contextual.v
Original file line number Diff line number Diff line change
Expand Up @@ -2,12 +2,16 @@
(** This file provides a definition (and basic development) of contextual categories as split type-cats/CwA’s in which every object is uniquely expressible as an iterated extension of a chosen terminal object. *)

Require Import UniMath.MoreFoundations.All.
Require Import UniMath.CategoryTheory.All.

Require Import UniMath.CategoryTheory.Core.Prelude.
Require Import UniMath.CategoryTheory.limits.graphs.limits.
Require Import UniMath.CategoryTheory.limits.graphs.terminal.

Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Require Import TypeTheory.Auxiliary.Partial.
Require Import TypeTheory.TypeCat.TypeCat.

Require Import TypeTheory.TypeCat.TypeCat.
Require Import TypeTheory.TypeCat.General.

Section Extensions.
Expand Down
2 changes: 1 addition & 1 deletion TypeTheory/TypeCat/ExtraStructure.v
Original file line number Diff line number Diff line change
Expand Up @@ -2,7 +2,7 @@
not yet integrated into the type theory of [Initiality.Syntax] and the statement/proof of initiality. *)

Require Import UniMath.MoreFoundations.All.
Require Import UniMath.CategoryTheory.All.
Require Import UniMath.CategoryTheory.Core.Categories.

Require Import TypeTheory.Auxiliary.Auxiliary.
Require Import TypeTheory.Auxiliary.CategoryTheory.
Expand Down

0 comments on commit 71a4afe

Please sign in to comment.