Zulip Chat Archive
Stream: Is there code for X?
Topic: Dependent forall_congr
Yaël Dillies (Dec 20 2021 at 20:40):
Could we generalize docs#forall₂_congr and friends to dependent functions? It's very annoying they don't work on bounded quantifiers, as in ∀ a ∈ s, P a ↔ ∀ a ∈ s, Q a
.
Yaël Dillies (Dec 20 2021 at 20:46):
Oh wait, the linkifier breaks because of the ₂
. Anything we can do about that?
Kevin Buzzard (Dec 20 2021 at 22:20):
Right now the workaround is just to post the full URL https://leanprover-community.github.io/mathlib_docs/logic/basic.html#forall%E2%82%82_congr but I'd also be interested in hearing about a workaround (Eric also had a broken linkifier link yesterday for another reason IIRC)
Kevin Buzzard (Dec 20 2021 at 22:21):
Change the def to a dependent theorem and push to a branch to see how much breaks...
Yury G. Kudryashov (Dec 20 2021 at 23:13):
PR?
Last updated: Dec 20 2023 at 11:08 UTC