Skip to content
Draft
Show file tree
Hide file tree
Changes from all commits
Commits
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: 0 additions & 2 deletions theories/Algebra/AbGroups/AbelianGroup.v
Original file line number Diff line number Diff line change
Expand Up @@ -6,8 +6,6 @@ Require Export Algebra.Groups.Subgroup.
Require Import Algebra.Groups.QuotientGroup.
Require Import WildCat.

Local Set Polymorphic Inductive Cumulativity.

Local Open Scope mc_scope.
Local Open Scope mc_add_scope.

Expand Down
2 changes: 0 additions & 2 deletions theories/Algebra/Groups/Group.v
Original file line number Diff line number Diff line change
Expand Up @@ -20,8 +20,6 @@ Require Import WildCat.
Require Import Spaces.Nat.Core.
Require Import Truncations.Core.

Local Set Polymorphic Inductive Cumulativity.

Generalizable Variables G H A B C f g.

Declare Scope group_scope.
Expand Down
3 changes: 2 additions & 1 deletion theories/Algebra/Universal/Homomorphism.v
Original file line number Diff line number Diff line change
Expand Up @@ -36,7 +36,8 @@ Section is_homomorphism.
Qed.
End is_homomorphism.

Record Homomorphism {σ} {A B : Algebra σ} : Type := Build_Homomorphism
(* We make this NonCumulative so that the proof of [homomorphism_id] goes through smoothly. TODO: remove this. *)
NonCumulative Record Homomorphism {σ} {A B : Algebra σ} : Type := Build_Homomorphism
{ def_homomorphism : forall (s : Sort σ), A s -> B s
; is_homomorphism : IsHomomorphism def_homomorphism }.

Expand Down
2 changes: 0 additions & 2 deletions theories/Basics/Datatypes.v
Original file line number Diff line number Diff line change
Expand Up @@ -18,8 +18,6 @@ Global Set Primitive Projections.
Global Set Nonrecursive Elimination Schemes.
Local Unset Elimination Schemes.

Local Set Polymorphic Inductive Cumulativity.

(** [option A] is the extension of [A] with an extra element [None] *)

Inductive option (A : Type) : Type :=
Expand Down
1 change: 1 addition & 0 deletions theories/Basics/Logic.v
Original file line number Diff line number Diff line change
Expand Up @@ -15,6 +15,7 @@ Set Implicit Arguments.
Require Export Basics.Notations.

Global Set Universe Polymorphism.
Global Set Polymorphic Inductive Cumulativity.
Global Set Asymmetric Patterns.

Notation "A -> B" := (forall (_ : A), B) : type_scope.
Expand Down
2 changes: 0 additions & 2 deletions theories/Basics/Overture.v
Original file line number Diff line number Diff line change
Expand Up @@ -13,8 +13,6 @@ Create HintDb rewrite discriminated.
#[export] Hint Variables Opaque : rewrite.
Create HintDb typeclass_instances discriminated.

Local Set Polymorphic Inductive Cumulativity.

(** ** Type classes *)

(** This command prevents Coq from trying to guess the values of existential variables while doing typeclass resolution. If you don't know what that means, ignore it. *)
Expand Down
2 changes: 0 additions & 2 deletions theories/Classes/interfaces/abstract_algebra.v
Original file line number Diff line number Diff line change
Expand Up @@ -2,8 +2,6 @@ Require Import Spaces.Nat.Core.
Require Export HoTT.Classes.interfaces.canonical_names.
Require Import Modalities.ReflectiveSubuniverse.

Local Set Polymorphic Inductive Cumulativity.

Generalizable Variables A B f g x y.

(*
Expand Down
2 changes: 1 addition & 1 deletion theories/Cubical/PathCube.v
Original file line number Diff line number Diff line change
Expand Up @@ -40,7 +40,7 @@ x011 | | x011----pi11----x111 |

(* Homogeneous cubes *)
(* PathCube left right top bottom front back *)
Cumulative Inductive PathCube {A}
Inductive PathCube {A}
: forall x000 {x010 x100 x110 x001 x011 x101 x111 : A}
{p0i0 : x000 = x010} {p1i0 : x100 = x110} {pi00 : x000 = x100}
{pi10 : x010 = x110} {p0i1 : x001 = x011} {p1i1 : x101 = x111}
Expand Down
2 changes: 1 addition & 1 deletion theories/Cubical/PathSquare.v
Original file line number Diff line number Diff line change
Expand Up @@ -36,7 +36,7 @@ Local Unset Elimination Schemes.

(* Definition of PathSquare *)
(* PathSquare left right up down *)
Cumulative Inductive PathSquare {A} : forall a00 {a10 a01 a11 : A},
Inductive PathSquare {A} : forall a00 {a10 a01 a11 : A},
a00 = a10 -> a01 = a11 -> a00 = a01 -> a10 = a11 -> Type
:= sq_id : forall {x : A},
PathSquare x 1 1 1 1.
Expand Down
1 change: 1 addition & 0 deletions theories/HIT/quotient.v
Original file line number Diff line number Diff line change
Expand Up @@ -84,6 +84,7 @@ Section Equiv.
intros. eapply concat;[apply transport_const|].
apply path_forall. intro z. apply path_hprop; simpl.
apply @equiv_iff_hprop; eauto.
(** Some universe annotations needed above for typeclass instance istrunc_trunctype. *)
Defined.

Context {Hrefl : Reflexive R}.
Expand Down
3 changes: 2 additions & 1 deletion theories/Modalities/Accessible.v
Original file line number Diff line number Diff line change
Expand Up @@ -27,7 +27,8 @@ Coercion lgenerator : LocalGenerators >-> Funclass.

(** We put this definition in a module so that no one outside of this file will use it accidentally. It will be redefined in [Localization] to refer to the localization reflective subuniverse, which is judgmentally the same but will also pick up typeclass inference for [In]. *)
Module Import IsLocal_Internal.
Definition IsLocal f X :=
(* TODO: reorder these universe variables; make it land in v. Currently done this way for backwards compatibility, to keep diff small. *)
Definition IsLocal@{u v a | u <= v, a <= v} (f : LocalGenerators@{a}) (X : Type@{u}) :=
(forall (i : lgen_indices f), ooExtendableAlong (f i) (fun _ => X)).
End IsLocal_Internal.

Expand Down
2 changes: 2 additions & 0 deletions theories/Modalities/Descent.v
Original file line number Diff line number Diff line change
Expand Up @@ -142,6 +142,8 @@ Proof.
Defined.

(** We can also state it in terms of belonging to a subuniverse if we lift [O'] accessibly (an analogue of Theorem 3.11(iii) of RSS). *)
(* *** TODO: With Cumulativity turned on globally, this produces a universe error.
It doesn't help to make the two Classes defined in this file NonCumulative. *)
Global Instance inO_TypeO_lex_leq `{Univalence} `{IsAccRSU O'}
: In (lift_accrsu O') (Type_ O)
:= fun i => ooextendable_TypeO_lex_leq (acc_lgen O' i).
Expand Down
6 changes: 3 additions & 3 deletions theories/Modalities/Localization.v
Original file line number Diff line number Diff line change
Expand Up @@ -267,7 +267,7 @@ Defined.

Module Export LocalizationHIT.

Cumulative Private Inductive Localize (f : LocalGenerators@{a}) (X : Type@{i})
Private Inductive Localize (f : LocalGenerators@{a}) (X : Type@{i})
: Type@{max(a,i)} :=
| loc : X -> Localize f X.

Expand Down Expand Up @@ -337,7 +337,7 @@ Section Localization.

End Localization.

Definition Loc@{a i} (f : LocalGenerators@{a}) : ReflectiveSubuniverse@{i}.
Definition Loc@{a i | a <= i} (f : LocalGenerators@{a}) : ReflectiveSubuniverse@{i}.
Proof.
snrefine (Build_ReflectiveSubuniverse
(Build_Subuniverse (IsLocal f) _ _)
Expand Down Expand Up @@ -422,7 +422,7 @@ Proof.
Defined.

(** Conversely, if a subuniverse is accessible, then the corresponding localization subuniverse is equivalent to it, and moreover exists at every universe level and satisfies its computation rules judgmentally. This is called [lift_accrsu] but in fact it works equally well to *lower* the universe level, as long as both levels are no smaller than the size [a] of the generators. *)
Definition lift_accrsu@{a i j} (O : Subuniverse@{i}) `{IsAccRSU@{a i} O}
Definition lift_accrsu@{a i j | a <= i, a <= j} (O : Subuniverse@{i}) `{IsAccRSU@{a i} O}
: ReflectiveSubuniverse@{j}
:= Loc@{a j} (acc_lgen O).

Expand Down
2 changes: 0 additions & 2 deletions theories/Pointed/Core.v
Original file line number Diff line number Diff line change
Expand Up @@ -6,8 +6,6 @@ Require Import Truncations.Core.
Require Import ReflectiveSubuniverse.
Require Import Extensions.

Local Set Polymorphic Inductive Cumulativity.

Declare Scope pointed_scope.

Local Open Scope pointed_scope.
Expand Down
9 changes: 5 additions & 4 deletions theories/TruncType.v
Original file line number Diff line number Diff line change
Expand Up @@ -38,9 +38,9 @@ Section TruncType.
: (A <~> B) <~> (A = B :> TruncType n)
:= equiv_path_trunctype' _ _ oE equiv_path_universe _ _.

Definition path_trunctype@{a b} {n : trunc_index} {A B : TruncType n}
Definition path_trunctype {n : trunc_index} {A B : TruncType n}
: A <~> B -> (A = B :> TruncType n)
:= equiv_path_trunctype@{a b} A B.
:= equiv_path_trunctype A B.

Global Instance isequiv_path_trunctype {n : trunc_index} {A B : TruncType n}
: IsEquiv (@path_trunctype n A B) := _.
Expand Down Expand Up @@ -99,7 +99,7 @@ Section TruncType.
Proof.
apply istrunc_S.
intros A B.
refine (istrunc_equiv_istrunc _ (equiv_path_trunctype@{i j} A B)).
refine (istrunc_equiv_istrunc _ (equiv_path_trunctype A B)).
case n as [ | n'].
- apply contr_equiv_contr_contr. (* The reason is different in this case. *)
- apply istrunc_equiv.
Expand All @@ -110,7 +110,8 @@ Section TruncType.
Global Instance istrunc_sig_istrunc : forall n, IsTrunc n.+1 { A : Type & IsTrunc n A } | 0.
Proof.
intro n.
apply (istrunc_equiv_istrunc _ issig_trunctype^-1).
nrefine (istrunc_equiv_istrunc _ issig_trunctype^-1).
exact istrunc_trunctype. (* To get universe variables to match, we do this as a separate step. *)
Defined.

(** ** Some standard inhabitants *)
Expand Down
2 changes: 1 addition & 1 deletion theories/Truncations/Core.v
Original file line number Diff line number Diff line change
Expand Up @@ -27,7 +27,7 @@ However, while we are faking our higher-inductives anyway, we can take some shor
Module Export Trunc.
Delimit Scope trunc_scope with trunc.

Cumulative Private Inductive Trunc (n : trunc_index) (A :Type) : Type :=
Private Inductive Trunc (n : trunc_index) (A :Type) : Type :=
tr : A -> Trunc n A.
Bind Scope trunc_scope with Trunc.
Arguments tr {n A} a.
Expand Down