Skip to content

Commit

Permalink
chore(category_theory/Fintype): remove redundant lemmas (#7531)
Browse files Browse the repository at this point in the history
These lemmas exist for arbitrary concrete categories.


- [x] depends on: #7530
  • Loading branch information
jcommelin committed May 10, 2021
1 parent b9f4420 commit 41c7b1e
Showing 1 changed file with 0 additions and 10 deletions.
10 changes: 0 additions & 10 deletions src/category_theory/Fintype.lean
Expand Up @@ -45,16 +45,6 @@ def incl : Fintype ⥤ Type* := induced_functor _

instance : concrete_category Fintype := ⟨incl⟩

@[simp] lemma coe_id {A : Fintype} : (𝟙 A : A → A) = id := rfl

@[simp] lemma coe_comp {A B C : Fintype} (f : A ⟶ B) (g : B ⟶ C) :
(f ≫ g : A → C) = g ∘ f := rfl

lemma id_apply {A : Fintype} (a : A) : (𝟙 A : A → A) a = a := rfl

lemma comp_apply {A B C : Fintype} (f : A ⟶ B) (g : B ⟶ C) (a : A) :
(f ≫ g) a = g (f a) := rfl

/--
The "standard" skeleton for `Fintype`. This is the full subcategory of `Fintype` spanned by objects
of the form `fin n` for `n : ℕ`. We parameterize the objects of `Fintype.skeleton` directly as `ℕ`,
Expand Down

0 comments on commit 41c7b1e

Please sign in to comment.