Zulip Chat Archive
Stream: Is there code for X?
Topic: List.ofFn x ~ List.ofFn y
Martin Dvořák (Jan 08 2024 at 12:46):
Is there an existing definition in Mathlib and API for the following concept?
import Mathlib.Data.List.Perm
def ArePerm {T : Type} {n : ℕ} (x y : Fin n → T) : Prop :=
List.ofFn x ~ List.ofFn y
Eric Wieser (Jan 08 2024 at 12:48):
docs#Equiv.Perm.ofFn_comp_perm
Eric Wieser (Jan 08 2024 at 12:48):
Probably you want an iff
version of that
Yury G. Kudryashov (Jan 08 2024 at 14:23):
I guess (not tested) MulAction.orbitRel (DomMulAct (Equiv.Perm (Fin n))
is what you want.
Yury G. Kudryashov (Jan 08 2024 at 14:24):
If you're going to add theory about it, then please do it for α → β
without finiteness assumptions first.
Yury G. Kudryashov (Jan 08 2024 at 14:29):
You can define, e.g.,
def DomConj (f : α → γ) (g : β → γ) : Prop := ∃ e : α ≃ β, f = g ∘ e
Last updated: May 02 2025 at 03:31 UTC