Skip to content

Commit

Permalink
Trigger CI for leanprover/lean4#3718
Browse files Browse the repository at this point in the history
  • Loading branch information
leanprover-community-mathlib4-bot committed Sep 23, 2024
2 parents b03e617 + f51886e commit 21c475d
Showing 1 changed file with 0 additions and 7 deletions.
7 changes: 0 additions & 7 deletions Batteries/Lean/HashSet.lean
Original file line number Diff line number Diff line change
Expand Up @@ -59,10 +59,3 @@ def insert' (s : HashSet α) (a : α) : HashSet α × Bool :=
let oldSize := s.size
let s := s.insert a
(s, s.size == oldSize)

/--
`O(n)`. Obtain a `HashSet` from an array.
-/
@[inline]
protected def ofArray [BEq α] [Hashable α] (as : Array α) : HashSet α :=
HashSet.empty.insertMany as

0 comments on commit 21c475d

Please sign in to comment.