Skip to content

Commit

Permalink
fix(data/set/basic): fix name of has_mem.mem.out (#13721)
Browse files Browse the repository at this point in the history
  • Loading branch information
fpvandoorn committed Apr 26, 2022
1 parent b00a7f8 commit 48997d7
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/data/set/basic.lean
Expand Up @@ -192,7 +192,7 @@ lemma mem_set_of {a : α} {p : α → Prop} : a ∈ {x | p x} ↔ p a := iff.rfl
/-- If `h : a ∈ {x | p x}` then `h.out : p x`. These are definitionally equal, but this can
nevertheless be useful for various reasons, e.g. to apply further projection notation or in an
argument to `simp`. -/
lemma has_mem.mem.out {p : α → Prop} {a : α} (h : a ∈ {x | p x}) : p a := h
lemma _root_.has_mem.mem.out {p : α → Prop} {a : α} (h : a ∈ {x | p x}) : p a := h

theorem nmem_set_of_eq {a : α} {p : α → Prop} : a ∉ {x | p x} = ¬ p a := rfl

Expand Down

0 comments on commit 48997d7

Please sign in to comment.