Zulip Chat Archive
Stream: mathlib4
Topic: data.finset.lattice mathlib4#1606
Johan Commelin (Jan 17 2023 at 07:09):
I'm working on this PR for a bit
Johan Commelin (Jan 17 2023 at 07:41):
I pushed.
Johan Commelin (Jan 17 2023 at 07:42):
There is some trouble aabout moving back and forth to OrderDual
. We used to convert
a lot of stuff. That no longer works because irreducible, I guess?
Johan Commelin (Jan 17 2023 at 07:42):
Is there a standard way too approach this now?
Kevin Buzzard (Jan 17 2023 at 08:15):
Kevin Buzzard (Jan 17 2023 at 08:15):
It doesn't look irreducible to me?
Johan Commelin (Jan 17 2023 at 08:16):
Huh! Then I don't know what's going on.
Yaël Dillies (Jan 17 2023 at 08:17):
Different order of elaboration is what's happening.
Ruben Van de Velde (Jan 17 2023 at 09:27):
I pushed alternative proofs for some of the OrderDual
issues. Still some errors and name changes needed, if someone wants to pick it up
Johan Commelin (Jan 17 2023 at 10:05):
one error left
Johan Commelin (Jan 17 2023 at 10:05):
Should supr
now always be renamed to sup\i
?
Johan Commelin (Jan 17 2023 at 10:08):
final error fixed
Johan Commelin (Jan 17 2023 at 10:12):
There is one linter complaint.
Johan Commelin (Jan 17 2023 at 10:13):
@[simp]
theorem sup_attach (s : Finset β) (f : β → α) : (s.attach.sup fun x => f x) = s.sup f :=
-- LHS does not simplify
Johan Commelin (Jan 17 2023 at 10:14):
Which I don't understand because
example (s : Finset β) (f : β → α) : (s.attach.sup fun x => f x) = a := by
simp? -- simp only [sup_attach]
-- goal is now `sup s f = a`
Johan Commelin (Jan 17 2023 at 10:22):
I think this one is ready for review
Heather Macbeth (Jan 17 2023 at 16:30):
Johan Commelin said:
There is some trouble aabout moving back and forth to
OrderDual
. We used toconvert
a lot of stuff. That no longer works because irreducible, I guess?
Maybe it's just that convert
is broken generally? Do the issues look like these ones?
https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/convert.20failures
Last updated: Dec 20 2023 at 11:08 UTC