Skip to content
New issue

Have a question about this project? Sign up for a free GitHub account to open an issue and contact its maintainers and the community.

By clicking “Sign up for GitHub”, you agree to our terms of service and privacy statement. We’ll occasionally send you account related emails.

Already on GitHub? Sign in to your account

[Merged by Bors] - feat(probability_theory/independence): prove equivalences for indep_set #6242

Closed
wants to merge 40 commits into from

Conversation

RemyDegenne
Copy link
Collaborator

@RemyDegenne RemyDegenne commented Feb 15, 2021

Prove the following equivalences on indep_set, for measurable sets s,t and a probability measure µ :

  • indep_set s t μ ↔ μ (s ∩ t) = μ s * μ t,
  • indep_set s t μ ↔ indep_sets {s} {t} μ.

In indep_sets.indep_set_of_mem, we use those equivalences to obtain indep_set s t µ from indep_sets S T µ and s ∈ S, t ∈ T.


@RemyDegenne RemyDegenne added the awaiting-review The author would like community review of the PR label Feb 15, 2021
@sgouezel
Copy link
Collaborator

I think a more principled approach to generate_from_set might make sense. Something like the following, maybe:

@[simp] lemma union_univ {s : set α} : s ∪ univ = univ := sorry

@[simp] lemma univ_union {s : set α} : univ ∪ s = univ := sorry

lemma generate_from_of_finite
  (S : set (set α)) (hcompl : ∀ s ∈ S, sᶜ ∈ S) (hempty : ∅ ∈ S) (hfin : finite S)
  (hun : ∀ s ∈ S, ∀ t ∈ S, s ∪ t ∈ S) :
  generate_measurable S = S :=
let m : measurable_space α :=
{ measurable_set' := S,
  measurable_set_empty := hempty,
  measurable_set_compl := hcompl,
  measurable_set_Union := sorry } in
le_antisymm (generate_from_le (λ t ht, ht) : generate_from S ≤ m)
  (λ t ht, measurable_set_generate_from ht)

lemma generate_from_set (s : set α) :
  generate_measurable ({∅, set.univ, s, sᶜ} : set (set α)) = ({∅, set.univ, s, sᶜ} : set (set α)) :=
generate_from_of_finite _ (by simp) (by simp) (by simp) (by simp)

Note that union_univ and univ_union have just been merged in master. So, there is only one sorry left (which is nontrivial, but probably more interesting than a case by case analysis).

@RemyDegenne RemyDegenne added awaiting-author A reviewer has asked the author a question or requested changes and removed awaiting-review The author would like community review of the PR labels Feb 16, 2021
@RemyDegenne
Copy link
Collaborator Author

Thanks for the better approach.
After experimenting a bit, I think this will be easier if we have lemmas about (finite) union-closed sets of sets. In fact, this is the third independent piece of code I have in which union-closed sets of sets appear and I need some of their properties. I will define sup-closed sets (and finsets) in a complete lattice and prove a bunch of lemmas on them before coming back to this PR.

@sgouezel sgouezel added the WIP Work in progress label Feb 16, 2021
@RemyDegenne
Copy link
Collaborator Author

I changed the proof to use a much simpler approach, using the fact that {s} is a pi-system, as done by @mzinkevi in #6466.

All statements about generate_from_set have been removed. I plan on doing two new related PRs: one with the properties of sup-closed sets I was talking about in my last comment (which will also be useful for the proof of the zero-one law), a second one with the generate_from_of_finite and generate_from_set lemmas discussed above.

@RemyDegenne RemyDegenne removed WIP Work in progress awaiting-author A reviewer has asked the author a question or requested changes labels Feb 28, 2021
@github-actions github-actions bot added merge-conflict Please `git merge origin/master` then a bot will remove this label. and removed blocked-by-other-PR This PR depends on another PR which is still in the queue. A bot manages this label via PR comment. labels Mar 11, 2021
@github-actions
Copy link

🎉 Great news! Looks like all the dependencies have been resolved:

💡 To add or remove a dependency please update this issue/PR description.

Brought to you by Dependent Issues (:robot: ). Happy coding!

@RemyDegenne RemyDegenne added the awaiting-author A reviewer has asked the author a question or requested changes label Mar 11, 2021
@github-actions github-actions bot removed the merge-conflict Please `git merge origin/master` then a bot will remove this label. label Mar 11, 2021
@RemyDegenne RemyDegenne added awaiting-review The author would like community review of the PR and removed awaiting-author A reviewer has asked the author a question or requested changes labels Mar 11, 2021
@sgouezel
Copy link
Collaborator

bors r+

@github-actions github-actions bot added ready-to-merge All that is left is for bors to build and merge this PR. (Remember you need to say `bors r+`.) and removed awaiting-review The author would like community review of the PR labels Mar 13, 2021
bors bot pushed a commit that referenced this pull request Mar 13, 2021
…et (#6242)

Prove the following equivalences on `indep_set`, for measurable sets `s,t` and a probability measure `µ` :
* `indep_set s t μ ↔ μ (s ∩ t) = μ s * μ t`,
* `indep_set s t μ ↔ indep_sets {s} {t} μ`.

In `indep_sets.indep_set_of_mem`, we use those equivalences to obtain `indep_set s t µ` from `indep_sets S T µ` and `s ∈ S`, `t ∈ T`.



Co-authored-by: mzinkevi <martinz@google.com>
Co-authored-by: mzinkevi <41597957+mzinkevi@users.noreply.github.com>
@bors
Copy link

bors bot commented Mar 13, 2021

Build failed (retrying...):

bors bot pushed a commit that referenced this pull request Mar 14, 2021
…et (#6242)

Prove the following equivalences on `indep_set`, for measurable sets `s,t` and a probability measure `µ` :
* `indep_set s t μ ↔ μ (s ∩ t) = μ s * μ t`,
* `indep_set s t μ ↔ indep_sets {s} {t} μ`.

In `indep_sets.indep_set_of_mem`, we use those equivalences to obtain `indep_set s t µ` from `indep_sets S T µ` and `s ∈ S`, `t ∈ T`.



Co-authored-by: mzinkevi <martinz@google.com>
Co-authored-by: mzinkevi <41597957+mzinkevi@users.noreply.github.com>
@bors
Copy link

bors bot commented Mar 14, 2021

Pull request successfully merged into master.

Build succeeded:

@bors bors bot changed the title feat(probability_theory/independence): prove equivalences for indep_set [Merged by Bors] - feat(probability_theory/independence): prove equivalences for indep_set Mar 14, 2021
@bors bors bot closed this Mar 14, 2021
@bors bors bot deleted the indep_set branch March 14, 2021 03:21
b-mehta pushed a commit that referenced this pull request Apr 2, 2021
…et (#6242)

Prove the following equivalences on `indep_set`, for measurable sets `s,t` and a probability measure `µ` :
* `indep_set s t μ ↔ μ (s ∩ t) = μ s * μ t`,
* `indep_set s t μ ↔ indep_sets {s} {t} μ`.

In `indep_sets.indep_set_of_mem`, we use those equivalences to obtain `indep_set s t µ` from `indep_sets S T µ` and `s ∈ S`, `t ∈ T`.



Co-authored-by: mzinkevi <martinz@google.com>
Co-authored-by: mzinkevi <41597957+mzinkevi@users.noreply.github.com>
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment
Labels
ready-to-merge All that is left is for bors to build and merge this PR. (Remember you need to say `bors r+`.)
Projects
None yet
Development

Successfully merging this pull request may close these issues.

None yet

3 participants