Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit ba87647

Browse files
committed
feat(data/set/finite): add lemma about to_finset of complement of set (#5881)
Add lemma stating that taking to_finset of the complement of a set is the same thing as taking the complement of to_finset of the set. Co-authored-by: agusakov <39916842+agusakov@users.noreply.github.com>
1 parent 7188d80 commit ba87647

File tree

1 file changed

+4
-0
lines changed

1 file changed

+4
-0
lines changed

src/data/set/finite.lean

Lines changed: 4 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -573,6 +573,10 @@ section
573573

574574
local attribute [instance, priority 1] classical.prop_decidable
575575

576+
lemma to_finset_compl {α : Type*} [fintype α] (s : set α) :
577+
sᶜ.to_finset = (s.to_finset)ᶜ :=
578+
by ext; simp
579+
576580
lemma to_finset_inter {α : Type*} [fintype α] (s t : set α) :
577581
(s ∩ t).to_finset = s.to_finset ∩ t.to_finset :=
578582
by ext; simp

0 commit comments

Comments
 (0)