Skip to content

Commit

Permalink
feat: port Mathlib.Data.List.Range (#1463)
Browse files Browse the repository at this point in the history
  • Loading branch information
jcommelin committed Jan 10, 2023
1 parent daa535f commit cbea84f
Show file tree
Hide file tree
Showing 2 changed files with 330 additions and 38 deletions.
2 changes: 1 addition & 1 deletion Mathlib/Data/Fintype/Basic.lean
Expand Up @@ -44,6 +44,6 @@ end Finset
namespace Fintype

instance (n : ℕ) : Fintype (Fin n) :=
⟨⟨List.finRange n, List.nodup_fin_range n⟩, List.mem_fin_range
⟨⟨List.finRange n, List.nodup_finRange n⟩, List.mem_finRange

end Fintype

0 comments on commit cbea84f

Please sign in to comment.