Skip to content

Commit f7e96f4

Browse files
committed
chore: fix the lemma name condIndepFun_iff_condDistrib_prod_ae_eq_prodMkRight (#30545)
There is a `prodMkRight` in the statement, not a `prodMkLeft`. Co-authored-by: Remy Degenne <remydegenne@gmail.com>
1 parent 4c1ded9 commit f7e96f4

File tree

1 file changed

+4
-1
lines changed

1 file changed

+4
-1
lines changed

Mathlib/Probability/Independence/Conditional.lean

Lines changed: 4 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -863,7 +863,7 @@ theorem condIndepFun_iff_map_prod_eq_prod_condDistrib_prod_condDistrib
863863
/-- Two random variables `f, g` are conditionally independent given a third `k` iff the
864864
conditional distribution of `f` given `k` and `g` is equal to the conditional distribution of `f`
865865
given `k`. -/
866-
theorem condIndepFun_iff_condDistrib_prod_ae_eq_prodMkLeft
866+
theorem condIndepFun_iff_condDistrib_prod_ae_eq_prodMkRight
867867
{γ : Type*} {mγ : MeasurableSpace γ} {mβ : MeasurableSpace β} {mβ' : MeasurableSpace β'}
868868
[StandardBorelSpace β] [Nonempty β] [StandardBorelSpace β'] [Nonempty β']
869869
(hf : Measurable f) (hg : Measurable g) {k : Ω → γ} (hk : Measurable k) :
@@ -907,6 +907,9 @@ theorem condIndepFun_iff_condDistrib_prod_ae_eq_prodMkLeft
907907
rw [h1, h2]
908908
exact ⟨fun h ↦ by rw [h], fun h ↦ by rw [h1_symm, h1, h2_symm, h2, h]⟩
909909

910+
@[deprecated (since := "2025-10-14")] alias condIndepFun_iff_condDistrib_prod_ae_eq_prodMkLeft :=
911+
condIndepFun_iff_condDistrib_prod_ae_eq_prodMkRight
912+
910913
section iCondIndepFun
911914
variable {β : ι → Type*} {m : ∀ i, MeasurableSpace (β i)} {f : ∀ i, Ω → β i}
912915

0 commit comments

Comments
 (0)