Zulip Chat Archive

Stream: new members

Topic: Proving trivial identities under expectation


Duncan Skahan (Oct 29 2024 at 00:32):

What tactic should I use for something like this?

import Mathlib

noncomputable section

open MeasureTheory ProbabilityTheory

variable {Ω : Type*} [ : MeasurableSpace Ω] {P : Measure Ω}
variable {X Y Z W : Ω  }

theorem trivial_identity : P[X*Y*Z*W] = P[Z*Y*X*W] := by
  sorry

Derek Rhodes (Oct 29 2024 at 01:35):

this works nicely:

theorem trivial_identity : P[X*Y*Z*W] = P[Z*Y*X*W] := by ring_nf

Last updated: May 02 2025 at 03:31 UTC