Zulip Chat Archive

Stream: Is there code for X?

Topic: If `Fintype α` then `Fintype (Finset α)`


Jihoon Hyun (Apr 01 2023 at 14:26):

instance {α : Type _} [Fintype α] : Fintype (Finset α) where
  elems := (@Finset.univ α).powerset
  complete x := by simp

I couldn't find such instance. Is there such an instance somewhere, or is this absent?

Yaël Dillies (Apr 01 2023 at 14:26):

Here's the instance in Lean 3: docs#finset.fintype

Jihoon Hyun (Apr 01 2023 at 14:28):

Then there should be one in mathlib4 also.. Thank you.

Yaël Dillies (Apr 01 2023 at 14:29):

docs4#Finset.fintype


Last updated: Dec 20 2023 at 11:08 UTC