Zulip Chat Archive

Stream: general

Topic: Happy new year!


Adam Topaz (Jan 01 2024 at 04:23):

import Mathlib

open Padic in
theorem HappyNewYear (p : ) [Fact p.Prime] :
    Nat.card ((ZMod 7 × ZMod 7) ≃+ (ZMod 7 × ZMod 7)) +
    Nat.card ((Fin 3  Fin 3) ≃* (Fin 3  Fin 3)) +
    Nat.card ( ≃+* ) +
    Nat.card (ℚ_[p] ≃+* ℚ_[p]) =
    2024 :=
  sorry

Adam Topaz (Jan 01 2024 at 04:44):

(Sorry for the edits, it should be doable now :))

Frederick Pu (Jan 01 2024 at 14:41):

Adam Topaz said:

import Mathlib

open Padic in
theorem HappyNewYear (p : ) [Fact p.Prime] :
    Nat.card ((ZMod 7 × ZMod 7) ≃+ (ZMod 7 × ZMod 7)) +
    Nat.card ((Fin 3  Fin 3) ≃* (Fin 3  Fin 3)) +
    Nat.card ( ≃+* ) +
    Nat.card (ℚ_[p] ≃+* ℚ_[p]) =
    2024 :=
  sorry

Sorry if this is a stupid question but how are you able to chain equivalence together like that. What does it mean?

Mauricio Collares (Jan 01 2024 at 14:43):

The code snippet sums cardinalities of different sets of equivalences/isomorphisms

Edit: having read Yaël's answer I now understand the question

Yaël Dillies (Jan 01 2024 at 14:44):

Fin 3 ≃ Fin 3 is a group, namely the symmetric group on three elements. In particular, we can talk about endomorphisms of it.

Frederick Pu (Jan 02 2024 at 02:07):

Yaël Dillies said:

Fin 3 ≃ Fin 3 is a group, namely the symmetric group on three elements. In particular, we can talk about endomorphisms of it.

Is there a coercion from equivalence to endomorphism to group?

Junyan Xu (Jan 02 2024 at 02:59):

It's just a Group isntance docs#Equiv.Perm.permGroup on Equiv.perm α which is defined to be α ≃ α reducibly.


Last updated: May 02 2025 at 03:31 UTC