Zulip Chat Archive
Stream: general
Topic: unique for two elements
Eric Wieser (Mar 24 2022 at 12:14):
In #12671, I state things about indexed families where the indexing family has exactly two elements (and I need to refer explicitly to those elements).
For one element, we can use unique X
and default
.
Whats's the preferred way to refer to this type of thing for two elements?
{i j : ι} (hij : i ≠ j) (h : (set.univ : set ι) = {i, j}) : foo i j
[fintype ι] {i j : ι} (hij : i ≠ j) (h : (finset.univ : set ι) = {i, j}) : foo i j
{i j : ι} (hij : i ≠ j) (h : ∀ k, k = i ∨ k = j) : foo i j
[almost_unique ι] : foo default other_default
Eric Wieser (Mar 24 2022 at 12:15):
Currently I've gone with 1, but 2 has the benefit that h
is often true by rfl
Junyan Xu (Mar 24 2022 at 12:47):
X ≃ bool
or fin 2
? f : bool → X
function.bijective f
?
Eric Rodriguez (Mar 24 2022 at 12:47):
I was thinking that maybe it's better to state the result for fin 2
first and do an equivalence, too
Eric Rodriguez (Mar 24 2022 at 12:48):
fin 2
also has some sort of an API, which is nice (like the fin 3
stuff earlier)
Eric Wieser (Mar 24 2022 at 13:04):
I guess I only really care about zmod 2
and units ℤ
Eric Wieser (Mar 24 2022 at 13:04):
Another one is punit ⊕ punit
Last updated: Dec 20 2023 at 11:08 UTC