bookshelf/Common/Finset.lean

17 lines
323 B
Plaintext
Raw Normal View History

import Mathlib.Data.Finset.Basic
/-! # Common.Finset
Additional theorems and definitions useful in the context of `Finset`s.
-/
namespace Finset
/--
An alternative `Finset.range` function that returns `Fin` indices instead of ``
indices.
-/
def finRange (n : ) : Finset (Fin n) :=
⟨sorry, sorry⟩
end Finset