Zulip Chat Archive

Stream: mathlib4

Topic: !4#4557 Probability.Indepence.Basic


Xavier Roblot (Jun 01 2023 at 16:59):

The file probability.independence.basic has several definitions or lemmas containing Indep, eg. docs#probability_theory.Indep or docs#probability_theory.Indep.Indep_sets. To deal with those, Mathport has been adding Cat at the end of the names but that is obviously wrong. So what would be the right naming scheme here?

Heather Macbeth (Jun 01 2023 at 17:01):

I think the naming scheme for the various flavours of Union should work.

Rémy Degenne (Jun 01 2023 at 17:01):

To come up with the names Indep/indep, I copied Union/union for sets. So whatever is used for those.

Xavier Roblot (Jun 01 2023 at 17:06):

So that would give iIndep to replace Indep then

Xavier Roblot (Jun 02 2023 at 13:05):

In the same file, the following lemma

@[symm]
theorem IndepFun.symm { : MeasurableSpace β} {f g : Ω  β} (hfg : IndepFun f g μ) :
    IndepFun g f μ := hfg.symm

gives the error

fail to show termination for
  ProbabilityTheory.IndepFun.symm
with errors
structural recursion cannot be used

well-founded recursion cannot be used, 'ProbabilityTheory.IndepFun.symm' does not take any (non-fixed) arguments

In Mathlib3, it was stated as

@[symm] lemma indep_fun.symm { : measurable_space β} {f g : Ω  β} (hfg : indep_fun f g μ) :
  indep_fun g f μ :=
hfg.symm

so essentially the same...

Moritz Doll (Jun 02 2023 at 13:12):

you want to add nonrec in front of you theorem

Moritz Doll (Jun 02 2023 at 13:12):

Lean 4 tries to apply IndepFun.symm for hfg.symm, whereas Lean 3 used something else


Last updated: Dec 20 2023 at 11:08 UTC