Zulip Chat Archive

Stream: new members

Topic: Proving Countability of linear equivalences


Rahul Soni (Dec 30 2024 at 13:58):

Hello Everyone, any pointers on solving this :-

import Mathlib
variable (h :   )
def isLinearCombination(a1 : )(a2 : ) : Prop :=
     l :  →₀   , a1 - a2 =   i  l.support, l i  h i

instance LinCombEquiv : Equivalence (isLinearCombination h) := sorry

instance SR : Setoid  where
  r := isLinearCombination h
  iseqv := LinCombEquiv h

def E : (Quotient (SR h))  Set  := λ x => {y :  | x = y}

/-We specify that each equivalence class is countable -/
theorem EalphaCountable (α : Quotient (SR h)) : ((E h) α).Countable := by
  rw[E,Set.countable_coe_iff,countable_iff_exists_injective]
  sorry

I am stuck on proving that it's countable.

Kevin Buzzard (Dec 30 2024 at 14:09):

What's the maths proof which you want to formalize?

Rahul Soni (Dec 30 2024 at 14:09):

First, we need to show that there are only countably many Finitely supported functions then every element can be rewritten as the sum of the default element and the evaluation of the finitely supported function on h

Andrew Yang (Dec 30 2024 at 14:37):

I think the more mathliby way to write these definitions is

import Mathlib
variable (h :   )

open Set Submodule

/-We specify that each equivalence class is countable -/
theorem EalphaCountable (α :   span  (range h)) : (Submodule.Quotient.mk ⁻¹' {α}).Countable := by

and you might find more lemmas this way.


Last updated: May 02 2025 at 03:31 UTC