Skip to content

Commit c481a1e

Browse files
committed
Renamed CoqSet to SET, CoqSetoid to SETOID and CatCat to CAT.
1 parent 0752837 commit c481a1e

18 files changed

+267
-267
lines changed

Cat.v

+7-7
Original file line numberDiff line numberDiff line change
@@ -684,7 +684,7 @@ Defined.
684684

685685
(** ** The category of setoids *)
686686

687-
(** [CoqSetoid] corresponds to what most category theory textbooks call Set,
687+
(** [SETOID] corresponds to what most category theory textbooks call Set,
688688
the category of sets and functions.
689689
690690
We need to use setoids instead of sets, because our categories have a
@@ -785,7 +785,7 @@ Proof. now setoid. Defined.
785785

786786
#[refine]
787787
#[global]
788-
Instance CoqSetoid : Cat :=
788+
Instance SETOID : Cat :=
789789
{|
790790
Ob := Setoid';
791791
Hom := SetoidHom;
@@ -952,7 +952,7 @@ Defined.
952952

953953
#[refine]
954954
#[export]
955-
Instance HomFunctor (C : Cat) (X : Ob C) : Functor C CoqSetoid :=
955+
Instance HomFunctor (C : Cat) (X : Ob C) : Functor C SETOID :=
956956
{
957957
fob := fun Y : Ob C => {| carrier := Hom X Y; setoid := HomSetoid X Y |}
958958
}.
@@ -991,7 +991,7 @@ Defined.
991991

992992
#[refine]
993993
#[export]
994-
Instance HomContravariant (C : Cat) (X : Ob C) : Contravariant C CoqSetoid :=
994+
Instance HomContravariant (C : Cat) (X : Ob C) : Contravariant C SETOID :=
995995
{
996996
coob := fun Y : Ob C => {| carrier := Hom Y X; setoid := HomSetoid Y X |}
997997
}.
@@ -1157,7 +1157,7 @@ Defined.
11571157

11581158
#[refine]
11591159
#[export]
1160-
Instance HomProfunctor (C : Cat) : Profunctor C C CoqSetoid :=
1160+
Instance HomProfunctor (C : Cat) : Profunctor C C SETOID :=
11611161
{
11621162
diob := fun X Y : Ob C => {| carrier := Hom X Y; setoid := HomSetoid X Y |};
11631163
}.
@@ -1371,8 +1371,8 @@ Proof.
13711371
now exists (component β X).
13721372
Qed.
13731373

1374-
Definition representable {C : Cat} (X : Ob C) (F : Functor C CoqSetoid) : Type :=
1374+
Definition representable {C : Cat} (X : Ob C) (F : Functor C SETOID) : Type :=
13751375
{α : NatTrans F (HomFunctor C X) & natural_isomorphism α}.
13761376

1377-
Definition corepresentable {C : Cat} (X : Ob C) (F : Functor (Dual C) CoqSetoid) : Type :=
1377+
Definition corepresentable {C : Cat} (X : Ob C) (F : Functor (Dual C) SETOID) : Type :=
13781378
{α : NatTrans F (HomFunctor (Dual C) X) & natural_isomorphism α}.

Category/Enriched.v

+4-4
Original file line numberDiff line numberDiff line change
@@ -1,7 +1,7 @@
11
From Cat Require Import Cat.
22
From Cat.Category Require Import CartesianClosed Monoidal.
33
From Cat.Universal Require Import Initial Terminal Product Coproduct.
4-
From Cat Require Import Instances.Setoids.
4+
From Cat Require Import Instances.SETOID.
55

66
Class Enriched (V : Monoidal) : Type :=
77
{
@@ -23,10 +23,10 @@ Class Enriched (V : Monoidal) : Type :=
2323

2424
#[refine]
2525
#[export]
26-
Instance Enriched_CoqSetoid
27-
: Enriched (Monoidal_HasTerm_HasProducts HasTerm_CoqSetoid HasProducts_CoqSetoid) :=
26+
Instance Enriched_SETOID
27+
: Enriched (Monoidal_HasTerm_HasProducts HasTerm_SETOID HasProducts_SETOID) :=
2828
{
29-
EOb := Ob CoqSetoid;
29+
EOb := Ob SETOID;
3030
EHom := fun X Y =>
3131
{|
3232
carrier := @Hom _ X Y;

Instances/AbGrp.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,6 @@
11
From Cat Require Export Cat.
22
From Cat.Universal Require Import Initial Terminal Zero Product Coproduct.
3-
From Cat.Instances Require Import Setoids Mon CMon Grp.
3+
From Cat.Instances Require Import SETOID Mon CMon Grp.
44

55
Set Implicit Arguments.
66

File renamed without changes.

Instances/Graph.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,6 @@
11
From Cat Require Export Cat.
22
From Cat.Universal Require Import Initial Terminal Product Coproduct.
3-
From Cat Require Export Instances.Setoids.
3+
From Cat Require Export Instances.SETOID.
44

55
Set Implicit Arguments.
66

Instances/Grp.v

+1-1
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,6 @@
11
From Cat Require Export Cat.
22
From Cat.Universal Require Import Initial Terminal Zero Product Coproduct.
3-
From Cat.Instances Require Import Setoids Mon.
3+
From Cat.Instances Require Import SETOID Mon.
44

55
Set Implicit Arguments.
66

Instances/Lin.v

+2-2
Original file line numberDiff line numberDiff line change
@@ -98,7 +98,7 @@ Proof. now lin. Defined.
9898
#[export]
9999
Instance Lin_Pros_product (X Y : Lin) : Pros :=
100100
{
101-
carrier := CoqSetoid_product X Y;
101+
carrier := SETOID_product X Y;
102102
leq := fun p1 p2 : X * Y =>
103103
fst p1 ≤ fst p2 /\ ~ fst p1 == fst p2
104104
\/
@@ -140,7 +140,7 @@ Defined.
140140
#[export]
141141
Instance Lin_Pros_coproduct (X Y : Lin) : Pros :=
142142
{
143-
carrier := CoqSetoid_coproduct X Y;
143+
carrier := SETOID_coproduct X Y;
144144
leq := fun p1 p2 : X + Y =>
145145
match p1, p2 with
146146
| inl x, inl x' => leq x x'

Instances/Mon.v

+7-7
Original file line numberDiff line numberDiff line change
@@ -454,7 +454,7 @@ Defined.
454454

455455
#[refine]
456456
#[export]
457-
Instance forgetful : Functor MonCat CoqSetoid :=
457+
Instance forgetful : Functor MonCat SETOID :=
458458
{
459459
fob := fun X : Mon => @setoid (sgr X);
460460
fmap := fun (A B : Mon) (f : Hom A B) => f;
@@ -468,7 +468,7 @@ Defined.
468468
Notation "'U'" := forgetful.
469469

470470
Definition free_monoid
471-
(X : Ob CoqSetoid) (M : Mon) (p : Hom X (fob U M)) : Prop :=
471+
(X : Ob SETOID) (M : Mon) (p : Hom X (fob U M)) : Prop :=
472472
forall (N : Mon) (q : SetoidHom X (fob U N)),
473473
exists!! h : MonHom M N, q == p .> fmap U h.
474474

@@ -494,7 +494,7 @@ Proof.
494494
all: now cbn; intros; lia.
495495
Defined.
496496

497-
Definition MonListUnit_p : SetoidHom CoqSetoid_term MonListUnit.
497+
Definition MonListUnit_p : SetoidHom SETOID_term MonListUnit.
498498
Proof.
499499
exists (fun _ => 1).
500500
now proper.
@@ -503,10 +503,10 @@ Defined.
503503
Set Nested Proofs Allowed.
504504

505505
Lemma free_monoid_MonListUnit :
506-
@free_monoid CoqSetoid_term MonListUnit MonListUnit_p.
506+
@free_monoid SETOID_term MonListUnit MonListUnit_p.
507507
Proof.
508508
unfold free_monoid. intros.
509-
Definition f1 (N : Mon) (q : SetoidHom CoqSetoid_term (fob U N))
509+
Definition f1 (N : Mon) (q : SetoidHom SETOID_term (fob U N))
510510
: SetoidHom MonListUnit N.
511511
Proof.
512512
exists (fix f (n : nat) : N :=
@@ -516,15 +516,15 @@ Proof.
516516
end).
517517
now proper; subst.
518518
Defined.
519-
Definition f2 (N : Mon) (q : SetoidHom CoqSetoid_term (fob U N))
519+
Definition f2 (N : Mon) (q : SetoidHom SETOID_term (fob U N))
520520
: SgrHom MonListUnit N.
521521
Proof.
522522
exists (f1 N q).
523523
induction x as [| x']; intros.
524524
- now cbn; rewrite neutr_l.
525525
- now cbn; rewrite <- assoc, -> IHx'.
526526
Defined.
527-
Definition f3 (N : Mon) (q : SetoidHom CoqSetoid_term (fob U N))
527+
Definition f3 (N : Mon) (q : SetoidHom SETOID_term (fob U N))
528528
: MonHom MonListUnit N.
529529
Proof.
530530
now exists (f2 N q).

Instances/Pros.v

+13-13
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,6 @@
11
From Cat Require Export Cat.
22
From Cat.Universal Require Export Initial Terminal Product Coproduct.
3-
From Cat Require Export Instances.Setoids.
3+
From Cat Require Export Instances.SETOID.
44

55
Set Implicit Arguments.
66

@@ -123,14 +123,14 @@ Abort.
123123
#[export]
124124
Instance Pros_init : Pros :=
125125
{
126-
carrier := CoqSetoid_init;
126+
carrier := SETOID_init;
127127
leq := fun (x y : Empty_set) => match x with end
128128
}.
129129
Proof. all: easy. Defined.
130130

131131
Definition Pros_create (X : Pros) : ProsHom Pros_init X.
132132
Proof.
133-
now exists (CoqSetoid_create X).
133+
now exists (SETOID_create X).
134134
Defined.
135135

136136
#[refine]
@@ -155,14 +155,14 @@ Defined.
155155
#[export]
156156
Instance Pros_term : Pros :=
157157
{
158-
carrier := CoqSetoid_term;
158+
carrier := SETOID_term;
159159
leq := fun _ _ => True
160160
}.
161161
Proof. all: easy. Defined.
162162

163163
Definition Pros_delete (X : Pros) : ProsHom X Pros_term.
164164
Proof.
165-
now exists (CoqSetoid_delete X).
165+
now exists (SETOID_delete X).
166166
Defined.
167167

168168
#[refine]
@@ -178,7 +178,7 @@ Proof. easy. Defined.
178178
#[export]
179179
Instance Pros_product (X Y : Pros) : Pros :=
180180
{
181-
carrier := CoqSetoid_product X Y;
181+
carrier := SETOID_product X Y;
182182
leq := fun x y : X * Y => leq (fst x) (fst y) /\ leq (snd x) (snd y)
183183
}.
184184
Proof.
@@ -190,18 +190,18 @@ Defined.
190190

191191
Definition Pros_outl (X Y : Pros) : ProsHom (Pros_product X Y) X.
192192
Proof.
193-
now exists (CoqSetoid_outl X Y); cbn.
193+
now exists (SETOID_outl X Y); cbn.
194194
Defined.
195195

196196
Definition Pros_outr (X Y : Pros) : ProsHom (Pros_product X Y) Y.
197197
Proof.
198-
now exists (CoqSetoid_outr X Y); cbn.
198+
now exists (SETOID_outr X Y); cbn.
199199
Defined.
200200

201201
Definition Pros_fpair
202202
{A B X : Pros} (f : ProsHom X A) (g : ProsHom X B) : ProsHom X (Pros_product A B).
203203
Proof.
204-
exists (CoqSetoid_fpair f g).
204+
exists (SETOID_fpair f g).
205205
now pros.
206206
Defined.
207207

@@ -225,7 +225,7 @@ Defined.
225225
#[export]
226226
Instance Pros_coproduct (X Y : Pros) : Pros :=
227227
{
228-
carrier := CoqSetoid_coproduct X Y;
228+
carrier := SETOID_coproduct X Y;
229229
leq := fun a b : X + Y =>
230230
match a, b with
231231
| inl x, inl x' => x ≤ x'
@@ -242,18 +242,18 @@ Defined.
242242

243243
Definition Pros_finl (X Y : Pros) : ProsHom X (Pros_coproduct X Y).
244244
Proof.
245-
now exists (CoqSetoid_finl X Y).
245+
now exists (SETOID_finl X Y).
246246
Defined.
247247

248248
Definition Pros_finr (X Y : Pros) : ProsHom Y (Pros_coproduct X Y).
249249
Proof.
250-
now exists (CoqSetoid_finr X Y).
250+
now exists (SETOID_finr X Y).
251251
Defined.
252252

253253
Definition Pros_copair
254254
(A B X : Pros) (f : ProsHom A X) (g : ProsHom B X) : ProsHom (Pros_coproduct A B) X.
255255
Proof.
256-
exists (CoqSetoid_copair f g).
256+
exists (SETOID_copair f g).
257257
now intros [] []; pros.
258258
Defined.
259259

Instances/RelMor.v

+3-3
Original file line numberDiff line numberDiff line change
@@ -1,6 +1,6 @@
11
From Cat Require Export Cat.
22
From Cat.Universal Require Import Initial Terminal Zero Product Coproduct.
3-
From Cat Require Export Instances.Setoids.
3+
From Cat Require Export Instances.SETOID.
44

55
Class SetoidRel (X Y : Setoid') : Type :=
66
{
@@ -81,7 +81,7 @@ Proof. all: now rel. Defined.
8181
#[export]
8282
Program Instance HasInit_SetoidRel : HasInit SetoidRelCat :=
8383
{
84-
init := CoqSetoid_init;
84+
init := SETOID_init;
8585
create := fun X : Setoid' => {| rel := fun (e : Empty_set) _ => match e with end |}
8686
}.
8787
Next Obligation. easy. Defined.
@@ -90,7 +90,7 @@ Next Obligation. easy. Defined.
9090
#[export]
9191
Program Instance HasTerm_SetoidRel : HasTerm SetoidRelCat :=
9292
{
93-
term := CoqSetoid_init;
93+
term := SETOID_init;
9494
delete := fun X : Setoid' => {| rel := fun _ (e : Empty_set) => match e with end |}
9595
}.
9696
Next Obligation. easy. Defined.

0 commit comments

Comments
 (0)