File tree Expand file tree Collapse file tree 3 files changed +4
-1
lines changed
Expand file tree Collapse file tree 3 files changed +4
-1
lines changed Original file line number Diff line number Diff line change @@ -371,6 +371,7 @@ abbrev getElem?_mkArray := @getElem?_replicate
371371
372372/-! ### mem -/
373373
374+ @[grind ←]
374375theorem not_mem_empty (a : α) : ¬ a ∈ #[] := by simp
375376
376377@[simp, grind =] theorem mem_push {xs : Array α} {x y : α} : x ∈ xs.push y ↔ x ∈ xs ∨ x = y := by
Original file line number Diff line number Diff line change @@ -392,7 +392,7 @@ theorem get!_eq_getElem! [Inhabited α] (l : List α) (i) : l.get! i = l[i]! :=
392392
393393/-! ### mem -/
394394
395- @[simp] theorem not_mem_nil {a : α} : ¬ a ∈ [] := nofun
395+ @[simp, grind ← ] theorem not_mem_nil {a : α} : ¬ a ∈ [] := nofun
396396
397397@[simp, grind =] theorem mem_cons : a ∈ b :: l ↔ a = b ∨ a ∈ l :=
398398 ⟨fun h => by cases h <;> simp [Membership.mem, *],
Original file line number Diff line number Diff line change @@ -907,6 +907,8 @@ theorem getElem?_singleton {a : α} {i : Nat} : #v[a][i]? = if i = 0 then some a
907907
908908grind_pattern getElem_mem => xs[i] ∈ xs
909909
910+
911+ @[grind ←]
910912theorem not_mem_empty (a : α) : ¬ a ∈ #v[] := nofun
911913
912914@[simp, grind =] theorem mem_push {xs : Vector α n} {x y : α} : x ∈ xs.push y ↔ x ∈ xs ∨ x = y := by
You can’t perform that action at this time.
0 commit comments