Skip to content

Commit

Permalink
chore(data/set/basic): add set.compl_eq_compl (#7641)
Browse files Browse the repository at this point in the history
  • Loading branch information
ericrbg committed May 18, 2021
1 parent c2114d4 commit e275604
Showing 1 changed file with 1 addition and 0 deletions.
1 change: 1 addition & 0 deletions src/data/set/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -105,6 +105,7 @@ instance {α : Type*} : boolean_algebra (set α) :=
@[simp] lemma inf_eq_inter : ((⊓) : set α → set α → set α) = (∩) := rfl
@[simp] lemma le_eq_subset : ((≤) : set α → set α → Prop) = (⊆) := rfl
/-! `set.lt_eq_ssubset` is defined further down -/
@[simp] lemma compl_eq_compl : set.compl = (has_compl.compl : set α → set α) := rfl

/-- Coercion from a set to the corresponding subtype. -/
instance {α : Type*} : has_coe_to_sort (set α) := ⟨_, λ s, {x // x ∈ s}⟩
Expand Down

0 comments on commit e275604

Please sign in to comment.