Skip to content

Commit

Permalink
Merge pull request #2111 from Alizter/ps/rr/chore__remove_cubical_v_i…
Browse files Browse the repository at this point in the history
…ndexing_file

chore: remove Cubical.v indexing file
  • Loading branch information
Alizter authored Oct 8, 2024
2 parents f14c526 + 75369bb commit 9ed2b66
Show file tree
Hide file tree
Showing 12 changed files with 21 additions and 17 deletions.
2 changes: 1 addition & 1 deletion test/bugs/github1758.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
From HoTT Require Import Basics.Overture HIT.Interval HIT.Flattening Colimits.GraphQuotient
Spaces.Torus.Torus Cubical.
Spaces.Torus.Torus Cubical.DPath.

(* Test that various higher inductive types are defined correctly. If they are defined in the most naive way, two uses of the induction principle that are definitionally equal on the point constructors will be considered definitionally equal, which is inconsistent. There is an idiom that must be used in order to force Coq to regard the supplementary data as being required as well. See, for example, Colimits/GraphQuotient.v for the idiom. *)

Expand Down
2 changes: 1 addition & 1 deletion theories/Algebra/AbGroups/Abelianization.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
Require Import Basics Types Truncations.Core.
Require Import Cubical WildCat.
Require Import Cubical.DPath WildCat.
Require Import Colimits.Coeq.
Require Import Algebra.AbGroups.AbelianGroup.
Require Import Modalities.ReflectiveSubuniverse.
Expand Down
2 changes: 1 addition & 1 deletion theories/Algebra/Groups/FreeProduct.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
Require Import Basics Types.
Require Import Cubical.
Require Import Cubical.DPath.
Require Import Spaces.List.Core Spaces.List.Theory.
Require Import Colimits.Pushout.
Require Import Truncations.Core Truncations.SeparatedTrunc.
Expand Down
5 changes: 0 additions & 5 deletions theories/Cubical.v

This file was deleted.

8 changes: 7 additions & 1 deletion theories/HoTT.v
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,13 @@
Require Export HoTT.Basics.
Require Export HoTT.Types.
Require Export HoTT.WildCat.
Require Export HoTT.Cubical.

Require Export HoTT.Cubical.DPath.
Require Export HoTT.Cubical.PathSquare.
Require Export HoTT.Cubical.DPathSquare.
Require Export HoTT.Cubical.PathCube.
Require Export HoTT.Cubical.DPathCube.

Require Export HoTT.Pointed.
Require Export HoTT.Truncations.

Expand Down
2 changes: 1 addition & 1 deletion theories/Homotopy/CayleyDickson.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
Require Import Classes.interfaces.abstract_algebra.
Require Import Cubical.
Require Import Cubical.DPath Cubical.PathSquare.
Require Import Pointed.Core Pointed.pSusp.
Require Import Homotopy.HSpace.Core.
Require Import Homotopy.Suspension.
Expand Down
3 changes: 2 additions & 1 deletion theories/Homotopy/ClassifyingSpace.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,6 @@
Require Import Basics Types.
Require Import Pointed Cubical WildCat.
Require Import Pointed WildCat.
Require Import Cubical.DPath Cubical.PathSquare Cubical.DPathSquare.
Require Import Algebra.AbGroups.
Require Import Homotopy.HSpace.Core.
Require Import TruncType.
Expand Down
2 changes: 1 addition & 1 deletion theories/Homotopy/HSpaceS1.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
Require Import Classes.interfaces.canonical_names.
Require Import Cubical.
Require Import Cubical.DPath Cubical.PathSquare.
Require Import Homotopy.Suspension.
Require Import Homotopy.HSpace.Core.
Require Import Homotopy.HSpace.Coherent.
Expand Down
3 changes: 2 additions & 1 deletion theories/Homotopy/Join/Core.v
Original file line number Diff line number Diff line change
@@ -1,4 +1,5 @@
Require Import Basics Types Cubical.
Require Import Basics Types.
Require Import Cubical.DPath Cubical.PathSquare.
Require Import NullHomotopy.
Require Import Extensions.
Require Import Colimits.Pushout.
Expand Down
2 changes: 1 addition & 1 deletion theories/Homotopy/Suspension.v
Original file line number Diff line number Diff line change
@@ -1,6 +1,6 @@
Require Import Basics.
Require Import Types.
Require Import Cubical.
Require Import Cubical.DPath Cubical.DPathSquare.
Require Import WildCat.
Require Import Colimits.Pushout.
Require Import NullHomotopy.
Expand Down
4 changes: 2 additions & 2 deletions theories/Spaces/Torus/Torus.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,5 @@
Require Import Basics.
Require Import Cubical.
Require Import Basics.Overture Basics.Equivalences Cubical.DPath
Cubical.PathSquare Cubical.DPathSquare Cubical.PathCube Cubical.DPathCube.

(** In this file we define the Torus as a HIT generated by two loops and a square between them. *)

Expand Down
3 changes: 2 additions & 1 deletion theories/Spaces/Torus/TorusEquivCircles.v
Original file line number Diff line number Diff line change
@@ -1,5 +1,6 @@
Require Import Basics Types.
Require Import Cubical.
Require Import Cubical.DPath Cubical.PathSquare Cubical.DPathSquare
Cubical.PathCube Cubical.DPathCube.
Require Import Spaces.Circle Spaces.Torus.Torus.

(** In this file we prove that the torus is equivalent to the product of two circles. *)
Expand Down

0 comments on commit 9ed2b66

Please sign in to comment.