Zulip Chat Archive

Stream: mathlib4

Topic: how does one get a `higher_order` annotation in Lean 4?


Arien Malec (Dec 01 2022 at 02:52):

I see the Mathport.Syntax definition and tried to import that, but got nothing...

Arien Malec (Dec 01 2022 at 03:11):

Also tried to follow the breadcrumbs up from Mathport.Syntax & get unknown attribute [higherOrder]

Mario Carneiro (Dec 01 2022 at 07:53):

things in Mathport.Syntax represent syntax for tactics and annotations that have not yet been implemented

Arien Malec (Dec 01 2022 at 16:12):

OK -- so control.bifunctor is blocked, or I can hand-roll what's needed.

If I understood the Lean 3 implementation, the goal is to take theorem foo ∀ x, f (g x) = h xand reason over theorem foo_f_g: f ∘ g = h...


Last updated: Dec 20 2023 at 11:08 UTC