Zulip Chat Archive

Stream: new members

Topic: permutations


vxctyxeha (May 14 2025 at 16:59):

Do these two sides represent different sets?

({σ : Perm (Fin 4) | σ.cycleType = {4}} : Finset (Perm (Fin 4))) = ((univ : Finset (Perm (Fin 4))).filter (fun σ => σ.cycleType = {4}) : Finset (Perm (Fin 4)))

Aaron Liu (May 14 2025 at 17:05):

no, they are "syntactically" equal

vxctyxeha (May 14 2025 at 17:09):

"Is the code below equivalent to proving what all the 4-cycles in S4 are?

import Mathlib
open Equiv Equiv.Perm Finset

theorem S4 :  ({ c[0,1,2,3], c[0,1,3,2], c[0,2,1,3], c[0,2,3,1], c[0,3,2,1], c[0,3,1,2] } : Finset (Perm (Fin 4))) = ((univ : Finset (Perm (Fin 4))).filter (fun σ => σ.cycleType = {4}) : Finset (Perm (Fin 4))) --
    := by

      native_decide

vxctyxeha (May 14 2025 at 17:44):

import Mathlib

open Equiv Equiv.Perm Finset

theorem per :

  ({ 1,  c[0, 1, 2], (c[0, 1, 2])^2, c[0, 1], c[0, 1, 2] * c[0, 1], ((c[0, 1, 2])^2) * c[0, 1] } : Finset (Perm (Fin 3))) = (univ : Finset (Perm (Fin 3))) :=

by
-

  decide

Last updated: Dec 20 2025 at 21:32 UTC