Skip to content

Commit

Permalink
feat(control/equiv_functor): fintype instance (#3783)
Browse files Browse the repository at this point in the history
  • Loading branch information
semorrison and semorrison committed Aug 15, 2020
1 parent b670212 commit 67dad7f
Showing 1 changed file with 4 additions and 1 deletion.
5 changes: 4 additions & 1 deletion src/control/equiv_functor/instances.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2020 Scott Morrison. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Author: Scott Morrison
-/
import data.finset.basic
import data.fintype.basic
import control.equiv_functor

/-!
Expand All @@ -24,3 +24,6 @@ instance equiv_functor_perm : equiv_functor perm :=
-- but we provide this computable alternative separately.
instance equiv_functor_finset : equiv_functor finset :=
{ map := λ α β e s, s.map e.to_embedding, }

instance equiv_functor_fintype : equiv_functor fintype :=
{ map := λ α β e s, by exactI fintype.of_bijective e e.bijective, }

0 comments on commit 67dad7f

Please sign in to comment.