Skip to content

Commit

Permalink
chore(probability_theory/*): Rename folder (#11989)
Browse files Browse the repository at this point in the history
Rename `probability_theory` to `probability`.
  • Loading branch information
YaelDillies committed Feb 15, 2022
1 parent 430faa9 commit 4c76eac
Show file tree
Hide file tree
Showing 6 changed files with 4 additions and 5 deletions.
File renamed without changes.
File renamed without changes.
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Martin Zinkevich
-/
import measure_theory.integral.lebesgue
import probability_theory.independence
import probability.independence

/-!
# Integration in Probability Theory
Expand Down
Expand Up @@ -3,9 +3,8 @@ Copyright (c) 2021 Rémy Degenne. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Rémy Degenne, Kexing Ying
-/

import probability_theory.stopping
import probability_theory.notation
import probability.notation
import probability.stopping

/-!
# Martingales
Expand All @@ -18,7 +17,7 @@ and for all `i ≤ j`, `μ[f j | ℱ.le i] ≤ᵐ[μ] f i`. Finally, `f : ι →
submartingale with respect to the filtration `ℱ` if `f i` is integrable, `f` is adapted with
resepct to `ℱ` and for all `i ≤ j`, `f i ≤ᵐ[μ] μ[f j | ℱ.le i]`.
The definitions of filtration and adapted can be found in `probability_theory.stopping`.
The definitions of filtration and adapted can be found in `probability.stopping`.
### Definitions
Expand Down
File renamed without changes.
File renamed without changes.

0 comments on commit 4c76eac

Please sign in to comment.