Skip to content

Commit

Permalink
chore(category_theory/limits): make fin_category_opposite an instance (
Browse files Browse the repository at this point in the history
  • Loading branch information
TwoFX committed Feb 21, 2022
1 parent b04851f commit d0fa7a8
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 3 deletions.
3 changes: 2 additions & 1 deletion src/category_theory/fin_category.lean
Expand Up @@ -91,7 +91,8 @@ open opposite
/--
The opposite of a finite category is finite.
-/
def fin_category_opposite {J : Type v} [small_category J] [fin_category J] : fin_category Jᵒᵖ :=
instance fin_category_opposite {J : Type v} [small_category J] [fin_category J] :
fin_category Jᵒᵖ :=
{ decidable_eq_obj := equiv.decidable_eq equiv_to_opposite.symm,
fintype_obj := fintype.of_equiv _ equiv_to_opposite,
decidable_eq_hom := λ j j', equiv.decidable_eq (op_equiv j j'),
Expand Down
2 changes: 0 additions & 2 deletions src/category_theory/limits/opposites.lean
Expand Up @@ -162,8 +162,6 @@ begin
apply_instance
end

local attribute [instance] fin_category_opposite

lemma has_finite_colimits_opposite [has_finite_limits C] :
has_finite_colimits Cᵒᵖ :=
{ out := λ J 𝒟 𝒥, by { resetI, apply_instance, }, }
Expand Down

0 comments on commit d0fa7a8

Please sign in to comment.