Zulip Chat Archive

Stream: mathlib4

Topic: doc comment of `himp_bot`


Asei Inoue (Sep 07 2024 at 20:14):

This is correct? (copy-paste mistake?)

/-- A Heyting algebra is a bounded lattice with an additional binary operation `⇨` called Heyting
implication such that `a ⇨` is right adjoint to `a ⊓`. -/
class HeytingAlgebra (α : Type*) extends GeneralizedHeytingAlgebra α, OrderBot α, HasCompl α where
  /-- `a ⇨` is right adjoint to `a ⊓` -/
  himp_bot (a : α) : a   = a

Asei Inoue (Sep 07 2024 at 20:14):

https://github.com/leanprover-community/mathlib4/blob/2969d0119259fdf37a81cca002481be932cc8953/Mathlib/Order/Heyting/Basic.lean#L144

Yaël Dillies (Sep 07 2024 at 20:21):

Yes, copy-paste error. Feel free to open a PR and request my review!

Asei Inoue (Sep 07 2024 at 20:30):

done

https://github.com/leanprover-community/mathlib4/pull/16587

Yury G. Kudryashov (Sep 08 2024 at 04:21):

@Yaël Dillies maintainer merge would be more visible. Delegated.

Yaël Dillies (Sep 08 2024 at 06:30):

What do you mean? I didn't yet have time to review it

Yury G. Kudryashov (Sep 08 2024 at 13:17):

Sorry, I misinterpreted your :praise:.


Last updated: May 02 2025 at 03:31 UTC