Skip to content

Commit

Permalink
data/multiset/range): add multiset.coe_range (#15201)
Browse files Browse the repository at this point in the history
  • Loading branch information
Ruben-VandeVelde committed Jul 11, 2022
1 parent 627bd0c commit aae01cd
Showing 1 changed file with 2 additions and 0 deletions.
2 changes: 2 additions & 0 deletions src/data/multiset/range.lean
Expand Up @@ -18,6 +18,8 @@ namespace multiset
that is, the set `{0, 1, ..., n-1}`. -/
def range (n : ℕ) : multiset ℕ := range n

theorem coe_range (n : ℕ) : ↑(list.range n) = range n := rfl

@[simp] theorem range_zero : range 0 = 0 := rfl

@[simp] theorem range_succ (n : ℕ) : range (succ n) = n ::ₘ range n :=
Expand Down

0 comments on commit aae01cd

Please sign in to comment.