Documentation

Mathlib.MeasureTheory.SetSemiring

Semirings and rings of sets #

A semi-ring of sets C (in the sense of measure theory) is a family of sets containing , stable by intersection and such that for all s, t ∈ C, t \ s is equal to a disjoint union of finitely many sets in C. Note that a semi-ring of sets may not contain unions.

An important example of a semi-ring of sets is intervals in . The intersection of two intervals is an interval (possibly empty). The union of two intervals may not be an interval. The set difference of two intervals may not be an interval, but it will be a disjoint union of two intervals.

A ring of sets is a set of sets containing , stable by union, set difference and intersection.

Main definitions #

Main statements #

structure MeasureTheory.IsSetSemiring {α : Type u_1} (C : Set (Set α)) :

A semi-ring of sets C is a family of sets containing , stable by intersection and such that for all s, t ∈ C, s \ t is equal to a disjoint union of finitely many sets in C.

Instances For
    noncomputable def MeasureTheory.IsSetSemiring.diffFinset {α : Type u_1} {C : Set (Set α)} {s : Set α} {t : Set α} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (ht : t C) :
    Finset (Set α)

    In a semi-ring of sets C, for all sets s, t ∈ C, s \ t is equal to a disjoint union of finitely many sets in C. The finite set of sets in the union is not unique, but this definition gives an arbitrary Finset (Set α) that satisfies the equality.

    We remove the empty set to ensure that t ∉ hC.diffFinset hs ht even if t = ∅.

    Equations
    Instances For
      theorem MeasureTheory.IsSetSemiring.empty_not_mem_diffFinset {α : Type u_1} {C : Set (Set α)} {s : Set α} {t : Set α} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (ht : t C) :
      theorem MeasureTheory.IsSetSemiring.diffFinset_subset {α : Type u_1} {C : Set (Set α)} {s : Set α} {t : Set α} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (ht : t C) :
      theorem MeasureTheory.IsSetSemiring.sUnion_diffFinset {α : Type u_1} {C : Set (Set α)} {s : Set α} {t : Set α} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (ht : t C) :
      theorem MeasureTheory.IsSetSemiring.not_mem_diffFinset {α : Type u_1} {C : Set (Set α)} {s : Set α} {t : Set α} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (ht : t C) :
      theorem MeasureTheory.IsSetSemiring.sUnion_insert_diffFinset {α : Type u_1} {C : Set (Set α)} {s : Set α} {t : Set α} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (ht : t C) (hst : t s) :
      theorem MeasureTheory.IsSetSemiring.disjoint_sUnion_diffFinset {α : Type u_1} {C : Set (Set α)} {s : Set α} {t : Set α} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (ht : t C) :
      theorem MeasureTheory.IsSetSemiring.exists_disjoint_finset_diff_eq {α : Type u_1} {C : Set (Set α)} {s : Set α} {I : Finset (Set α)} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (hI : I C) :
      ∃ (J : Finset (Set α)), J C Set.PairwiseDisjoint (J) id s \ ⋃₀ I = ⋃₀ J

      In a semiring of sets C, for all set s ∈ C and finite set of sets I ⊆ C, there is a finite set of sets in C whose union is s \ ⋃₀ I. See IsSetSemiring.diffFinset₀ for a definition that gives such a set.

      noncomputable def MeasureTheory.IsSetSemiring.diffFinset₀ {α : Type u_1} {C : Set (Set α)} {s : Set α} {I : Finset (Set α)} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (hI : I C) :
      Finset (Set α)

      In a semiring of sets C, for all set s ∈ C and finite set of sets I ⊆ C, diffFinset₀ is a finite set of sets in C such that s \ ⋃₀ I = ⋃₀ (hC.diffFinset₀ hs I hI). diffFinset is a special case of diffFinset₀ where I is a singleton.

      Equations
      Instances For
        theorem MeasureTheory.IsSetSemiring.empty_not_mem_diffFinset₀ {α : Type u_1} {C : Set (Set α)} {s : Set α} {I : Finset (Set α)} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (hI : I C) :
        theorem MeasureTheory.IsSetSemiring.diffFinset₀_subset {α : Type u_1} {C : Set (Set α)} {s : Set α} {I : Finset (Set α)} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (hI : I C) :
        theorem MeasureTheory.IsSetSemiring.diff_sUnion_eq_sUnion_diffFinset₀ {α : Type u_1} {C : Set (Set α)} {s : Set α} {I : Finset (Set α)} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (hI : I C) :
        theorem MeasureTheory.IsSetSemiring.sUnion_diffFinset₀_subset {α : Type u_1} {C : Set (Set α)} {s : Set α} {I : Finset (Set α)} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (hI : I C) :
        theorem MeasureTheory.IsSetSemiring.disjoint_sUnion_diffFinset₀ {α : Type u_1} {C : Set (Set α)} {s : Set α} {I : Finset (Set α)} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (hI : I C) :
        theorem MeasureTheory.IsSetSemiring.disjoint_diffFinset₀ {α : Type u_1} {C : Set (Set α)} {s : Set α} {I : Finset (Set α)} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (hI : I C) :
        theorem MeasureTheory.IsSetSemiring.pairwiseDisjoint_union_diffFinset₀ {α : Type u_1} {C : Set (Set α)} {s : Set α} {I : Finset (Set α)} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (hI : I C) (h_dis : Set.PairwiseDisjoint (I) id) :
        theorem MeasureTheory.IsSetSemiring.sUnion_union_sUnion_diffFinset₀_of_subset {α : Type u_1} {C : Set (Set α)} {s : Set α} {I : Finset (Set α)} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (hI : I C) (hI_ss : tI, t s) :
        theorem MeasureTheory.IsSetSemiring.sUnion_union_diffFinset₀_of_subset {α : Type u_1} {C : Set (Set α)} {s : Set α} {I : Finset (Set α)} (hC : MeasureTheory.IsSetSemiring C) (hs : s C) (hI : I C) (hI_ss : tI, t s) [DecidableEq (Set α)] :
        structure MeasureTheory.IsSetRing {α : Type u_1} (C : Set (Set α)) :

        A ring of sets C is a family of sets containing , stable by union and set difference. It is then also stable by intersection (see IsSetRing.inter_mem).

        Instances For
          theorem MeasureTheory.IsSetRing.inter_mem {α : Type u_1} {C : Set (Set α)} {s : Set α} {t : Set α} (hC : MeasureTheory.IsSetRing C) (hs : s C) (ht : t C) :
          s t C
          theorem MeasureTheory.IsSetRing.biUnion_mem {α : Type u_1} {C : Set (Set α)} {ι : Type u_2} (hC : MeasureTheory.IsSetRing C) {s : ιSet α} (S : Finset ι) (hs : nS, s n C) :
          ⋃ i ∈ S, s i C
          theorem MeasureTheory.IsSetRing.biInter_mem {α : Type u_1} {C : Set (Set α)} {ι : Type u_2} (hC : MeasureTheory.IsSetRing C) {s : ιSet α} (S : Finset ι) (hS : S.Nonempty) (hs : nS, s n C) :
          ⋂ i ∈ S, s i C