Skip to content

Commit

Permalink
Categories: remove some %type annotations
Browse files Browse the repository at this point in the history
  • Loading branch information
jdchristensen committed Jul 31, 2024
1 parent 1c4250d commit 42647dc
Show file tree
Hide file tree
Showing 6 changed files with 12 additions and 12 deletions.
6 changes: 3 additions & 3 deletions theories/Categories/Category/Prod.v
Original file line number Diff line number Diff line change
Expand Up @@ -17,9 +17,9 @@ Section prod.

Definition prod : PreCategory.
refine (@Build_PreCategory
(C * D)%type
(fun s d => (morphism C (fst s) (fst d)
* morphism D (snd s) (snd d))%type)
(C * D)
(fun s d => morphism C (fst s) (fst d)
* morphism D (snd s) (snd d))
(fun x => (identity (fst x), identity (snd x)))
(fun s d d' m2 m1 => (fst m2 o fst m1, snd m2 o snd m1))
_
Expand Down
8 changes: 4 additions & 4 deletions theories/Categories/Category/Sigma/Univalent.v
Original file line number Diff line number Diff line change
Expand Up @@ -50,7 +50,7 @@ Section onmorphisms.
Variable A : PreCategory.
Variable Pmor : forall s d, morphism A s d -> Type.

Local Notation mor s d := { m : _ | Pmor s d m }%type.
Local Notation mor s d := { m : _ | Pmor s d m }.
Context `(HPmor : forall s d, IsHSet (mor s d)).

Variable Pidentity : forall x, @Pmor x x (@identity A _).
Expand Down Expand Up @@ -148,11 +148,11 @@ Section on_both.
Variable A : PreCategory.
Variable Pobj : A -> Type.

Local Notation obj := { x : _ | Pobj x }%type (only parsing).
Local Notation obj := { x : _ | Pobj x } (only parsing).

Variable Pmor : forall s d : obj, morphism A s.1 d.1 -> Type.

Local Notation mor s d := { m : _ | Pmor s d m }%type (only parsing).
Local Notation mor s d := { m : _ | Pmor s d m } (only parsing).
Context `(HPmor : forall s d, IsHSet (mor s d)).

Variable Pidentity : forall x, @Pmor x x (@identity A _).
Expand Down Expand Up @@ -283,7 +283,7 @@ Section on_both.

Local Definition equiv_iso_A'_eisretr_helper {s d}
(x : {e : @Isomorphic A s.1 d.1
| Pmor_iso_T s d e e^-1 (@left_inverse _ _ _ e e) right_inverse }%type)
| Pmor_iso_T s d e e^-1 (@left_inverse _ _ _ e e) right_inverse })
: transport
(fun e : @Isomorphic A s.1 d.1 =>
Pmor_iso_T s d e e^-1 left_inverse right_inverse)
Expand Down
2 changes: 1 addition & 1 deletion theories/Categories/Category/Sum.v
Original file line number Diff line number Diff line change
Expand Up @@ -43,7 +43,7 @@ End internals.
Definition sum (C D : PreCategory) : PreCategory.
Proof.
refine (@Build_PreCategory
(C + D)%type
(C + D)
(sum_morphism C D)
(sum_identity C D)
(sum_compose C D)
Expand Down
4 changes: 2 additions & 2 deletions theories/Categories/ExponentialLaws/Tactics.v
Original file line number Diff line number Diff line change
Expand Up @@ -21,10 +21,10 @@ Ltac exp_laws_misc_t' :=
Ltac exp_laws_simplify_types' :=
idtac;
match goal with
| [ H : (_ + _)%type |- _ ] => destruct H
| [ H : (_ + _) |- _ ] => destruct H
| [ H : Unit |- _ ] => destruct H
| [ H : Empty |- _ ] => destruct H
| [ H : (_ * _)%type |- _ ] => destruct H
| [ H : (_ * _) |- _ ] => destruct H
| [ |- _ = _ :> Functor _ _ ] => progress path_functor
| [ |- _ = _ :> NaturalTransformation _ _ ] => progress path_natural_transformation
| [ |- _ = _ :> prod _ _ ] => apply path_prod
Expand Down
2 changes: 1 addition & 1 deletion theories/Categories/Functor/Sum.v
Original file line number Diff line number Diff line change
Expand Up @@ -89,7 +89,7 @@ Section swap_functor.
transport_path_forall_hammer.
by repeat match goal with
| [ H : Empty |- _ ] => destruct H
| [ H : (_ + _)%type |- _ ] => destruct H
| [ H : (_ + _) |- _ ] => destruct H
| _ => progress hnf in *
end.
Qed.
Expand Down
2 changes: 1 addition & 1 deletion theories/Categories/NatCategory.v
Original file line number Diff line number Diff line change
Expand Up @@ -18,7 +18,7 @@ Module Export Core.
match n with
| 0 => Empty
| 1 => Unit
| S n' => (CardinalityRepresentative n' + Unit)%type
| S n' => CardinalityRepresentative n' + Unit
end.

Coercion CardinalityRepresentative : nat >-> Sortclass.
Expand Down

0 comments on commit 42647dc

Please sign in to comment.