Zulip Chat Archive
Stream: mathlib4
Topic: Finset.le_eq_subset
Yury G. Kudryashov (Apr 13 2024 at 23:04):
Here is an #mwe:
import Mathlib.Data.Finset.Basic
example (s : Finset ℕ) : Finset.coeEmb s = s := by simp -- works
example (s : Finset ℕ) : Finset.coeEmb.1 s = s := by simp -- fails
Yury G. Kudryashov (Apr 13 2024 at 23:07):
Why it fails
Yury G. Kudryashov (Apr 13 2024 at 23:08):
What should we do about it?
Yury G. Kudryashov (Apr 14 2024 at 05:38):
I would prefer to get rid of ⊆
for sets and finsets but I was told that it's bad for pedagogical reasons.
Antoine Chambert-Loir (Apr 14 2024 at 07:21):
I agree that it is a burden to have to rewrite subset as le or the other way round. Is it possible to have subset be just notation for le?
Yaël Dillies (Apr 14 2024 at 07:22):
Yes, Kyle and I have some work towards it
Yaël Dillies (Apr 14 2024 at 07:22):
but I won't have time to finish it before this summer
Antoine Chambert-Loir (Apr 14 2024 at 07:29):
Can't you delegate some things from the big plate you seem to have? Nobody's too young to suffer burn out, but still...
Yaël Dillies (Apr 14 2024 at 07:30):
Go wild :smile: :point_down:
Kyle Miller said:
Here's an experiment with what we talked about in Bonn regarding Set using lattice operations but pretty printing using set notation: https://github.com/leanprover-community/mathlib4/tree/kmill_set_use_lattice
Last updated: May 02 2025 at 03:31 UTC