File tree Expand file tree Collapse file tree 2 files changed +14
-4
lines changed Expand file tree Collapse file tree 2 files changed +14
-4
lines changed Original file line number Diff line number Diff line change @@ -302,16 +302,24 @@ class IsDiscrete (C : Type*) [Category C] : Prop where
302
302
303
303
attribute [instance] IsDiscrete.subsingleton
304
304
305
- lemma obj_ext_of_isDiscrete {C : Type *} [Category C] [IsDiscrete C]
306
- {X Y : C} (f : X ⟶ Y) : X = Y := IsDiscrete.eq_of_hom f
307
-
308
305
instance Discrete.isDiscrete (C : Type *) : IsDiscrete (Discrete C) where
309
306
eq_of_hom := by rintro ⟨_⟩ ⟨_⟩ ⟨⟨rfl⟩⟩; rfl
310
307
311
- instance (C : Type *) [Category C] [IsDiscrete C] : IsDiscrete Cᵒᵖ where
308
+ section
309
+
310
+ variable {C : Type *} [Category C] [IsDiscrete C]
311
+
312
+ lemma obj_ext_of_isDiscrete {X Y : C} (f : X ⟶ Y) : X = Y := IsDiscrete.eq_of_hom f
313
+
314
+ instance isIso_of_isDiscrete {X Y : C} (f : X ⟶ Y) : IsIso f :=
315
+ ⟨eqToHom (IsDiscrete.eq_of_hom f).symm, by aesop_cat⟩
316
+
317
+ instance : IsDiscrete Cᵒᵖ where
312
318
eq_of_hom := by
313
319
rintro ⟨_⟩ ⟨_⟩ ⟨f⟩
314
320
obtain rfl := obj_ext_of_isDiscrete f
315
321
rfl
316
322
323
+ end
324
+
317
325
end CategoryTheory
Original file line number Diff line number Diff line change @@ -16,4 +16,6 @@ variable {C : Type*}
16
16
17
17
instance : Groupoid (Discrete C) := { inv := fun h ↦ ⟨⟨h.1 .1 .symm⟩⟩ }
18
18
19
+ instance [Category C] [IsDiscrete C] : IsGroupoid C where
20
+
19
21
end CategoryTheory
You can’t perform that action at this time.
0 commit comments