Skip to content

Commit

Permalink
feat(category_theory): separators and detectors (#11880)
Browse files Browse the repository at this point in the history
  • Loading branch information
TwoFX committed Feb 15, 2022
1 parent ff2c9dc commit d76ac2e
Show file tree
Hide file tree
Showing 4 changed files with 390 additions and 7 deletions.
15 changes: 10 additions & 5 deletions src/category_theory/balanced.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2022 Markus Himmel. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Markus Himmel
-/
import category_theory.isomorphism
import category_theory.epi_mono

/-!
# Balanced categories
Expand All @@ -14,10 +14,6 @@ Balanced categories arise frequently. For example, categories in which every mon
(or epimorphism) is strong are balanced. Examples of this are abelian categories and toposes, such
as the category of types.
## TODO
The opposite of a balanced category is again balanced.
-/

universes v u
Expand All @@ -40,4 +36,13 @@ balanced.is_iso_of_mono_of_epi _
lemma is_iso_iff_mono_and_epi [balanced C] {X Y : C} (f : X ⟶ Y) : is_iso f ↔ mono f ∧ epi f :=
⟨λ _, by exactI ⟨infer_instance, infer_instance⟩, λ ⟨_, _⟩, by exactI is_iso_of_mono_of_epi _⟩

section
local attribute [instance] is_iso_of_mono_of_epi

lemma balanced_opposite [balanced C] : balanced Cᵒᵖ :=
{ is_iso_of_mono_of_epi := λ X Y f fmono fepi,
by { rw ← quiver.hom.op_unop f, exactI is_iso_of_op _ } }

end

end category_theory

0 comments on commit d76ac2e

Please sign in to comment.