Zulip Chat Archive

Stream: general

Topic: induction while keeping track of a hypothesis


Mantas Baksys (Dec 15 2021 at 21:38):

Hey, I've run into the following problem. I can't seem to be able to find out how to induct over permutations satisfying a specific hypothesis. Here's an MWE :

import tactic group_theory.perm.support group_theory.perm.sign

open finset equiv
open_locale classical big_operators

theorem induction {ι : Type*} [fintype ι] (s : finset ι) (σ : perm ι) ( : σ.support  s) :
  false :=
begin
  cases (perm.trunc_swap_factors σ).out with l hl,
  induction l with g l generalizing σ ,
  sorry,
  sorry,
end

The problem is that as a hypothesis is true only for the current σ and I'd like to have it as a hypothesis also for the previous one. Initially, I wanted to use swap_induction_on but that turned out to be set up in a way, where this hypothesis tracking is not supported. Thanks!

Riccardo Brasca (Dec 15 2021 at 21:46):

This was nonsense, sorry

Alex J. Best (Dec 15 2021 at 21:47):

I don't think this is mathematically possible for an arbitrary hypothesis right? Like if the hypothesis is sigma.support = s there's no way to get there with only transpositions. So you are really doing something special to the situation that I don't think there are tools for. You'd have to write an induction principle saying that every perm with restricted support is attainable via compositing transpositions with that support, likely the existing proof already does this under the hood?
In your case seeing as your condition is that the perm lies in a subgroup it might be more effective to pass to that subgroup (perm s) and use induction on that subgroup.

Mantas Baksys (Dec 15 2021 at 21:51):

Alex J. Best said:

I don't think this is mathematically possible for an arbitrary hypothesis right? Like if the hypothesis is sigma.support = s there's no way to get there with only transpositions. So you are really doing something special to the situation that I don't think there are tools for. You'd have to write an induction principle saying that every perm with restricted support is attainable via compositing transpositions with that support, likely the existing proof already does this under the hood?
In your case seeing as your condition is that the perm lies in a subgroup it might be more effective to pass to that subgroup (perm s) and use induction on that subgroup.

You're right, I'll need to write something specific in that case.

Yakov Pechersky (Dec 16 2021 at 03:48):

Does cases h : (perm.trunc_swap_factors σ).out with l hl, help, at least conceptually, with what you wanted?


Last updated: Dec 20 2023 at 11:08 UTC