Zulip Chat Archive
Stream: mathlib4
Topic: Quotient notation on Antisymmetrization
Violeta Hernández (Jan 29 2025 at 07:57):
Currently, we can't use quotient notation ⟦x⟧
on the antisymmetrization of a type. Is this intended/fixable?
import Mathlib.Order.Antisymmetrization
def Foo := Antisymmetrization ℕ (· ≤ ·)
-- failed to synthesize
-- LT (Quotient (AntisymmRel.setoid ℕ fun x1 x2 => x1 ≤ x2))
example (x y : ℕ) : (⟦x⟧ : Foo) < ⟦y⟧ ↔ x < y := Iff.rfl
@Yaël Dillies
Junyan Xu (Jan 29 2025 at 10:39):
I think you need to change docs#Antisymmetrization and Foo to abbrevs. I made docs#DirectLimit an abbrev for this reason.
Yaël Dillies (Jan 29 2025 at 11:40):
Aren't we moving away from global⟦x⟧
notation? cc @Yuyang Zhao
Violeta Hernández (Jan 29 2025 at 21:01):
I wasn't aware of that development. In truth this is something we want to do on the game file anyways (where this issue arose) since we'll soon get a second important quotient.
Last updated: May 02 2025 at 03:31 UTC