Zulip Chat Archive

Stream: mathlib4

Topic: missing attributes


Patrick Massot (Oct 16 2022 at 19:36):

During the port, what should we do when Lean complains an attribute doesn't exist?

Patrick Massot (Oct 16 2022 at 19:36):

Specifically, what about refl and trans?

Scott Morrison (Oct 16 2022 at 22:11):

For refl:

import Mathlib.Tactic.Relation.Rfl

@[refl]
theorem foo : 1 = 1 := rfl

Scott Morrison (Oct 16 2022 at 22:12):

For trans, for now use import Mathlib.Mathport.Attributes, I guess.

Scott Morrison (Oct 16 2022 at 22:14):

If you run into other attributes, hopefully you will find them noted as needing porting in Mathlib/Mathport/Syntax.lean (which you can freely import if needed, I guess), or they should already be implemented somewhere, and searching for register.*attr should help you locate it.

Patrick Massot (Oct 17 2022 at 07:23):

@Mario Carneiro do you agree with all this?


Last updated: Dec 20 2023 at 11:08 UTC