Documentation

Mathlib.Combinatorics.SetFamily.Compression.Down

Down-compressions #

This file defines down-compression.

Down-compressing π’œ : Finset (Finset Ξ±) along a : Ξ± means removing a from the elements of π’œ, when the resulting set is not already in π’œ.

Main declarations #

Notation #

𝓓 a π’œ is notation for Down.compress a π’œ in locale SetFamily.

References #

Tags #

compression, down-compression

def Finset.nonMemberSubfamily {Ξ± : Type u_1} [DecidableEq Ξ±] (a : Ξ±) (π’œ : Finset (Finset Ξ±)) :
Finset (Finset Ξ±)

Elements of π’œ that do not contain a.

Equations
Instances For
    def Finset.memberSubfamily {Ξ± : Type u_1} [DecidableEq Ξ±] (a : Ξ±) (π’œ : Finset (Finset Ξ±)) :
    Finset (Finset Ξ±)

    Image of the elements of π’œ which contain a under removing a. Finsets that do not contain a such that insert a s ∈ π’œ.

    Equations
    Instances For
      @[simp]
      theorem Finset.mem_nonMemberSubfamily {Ξ± : Type u_1} [DecidableEq Ξ±] {π’œ : Finset (Finset Ξ±)} {s : Finset Ξ±} {a : Ξ±} :
      s ∈ Finset.nonMemberSubfamily a π’œ ↔ s ∈ π’œ ∧ a βˆ‰ s
      @[simp]
      theorem Finset.mem_memberSubfamily {Ξ± : Type u_1} [DecidableEq Ξ±] {π’œ : Finset (Finset Ξ±)} {s : Finset Ξ±} {a : Ξ±} :
      s ∈ Finset.memberSubfamily a π’œ ↔ insert a s ∈ π’œ ∧ a βˆ‰ s
      theorem Finset.nonMemberSubfamily_inter {Ξ± : Type u_1} [DecidableEq Ξ±] (a : Ξ±) (π’œ : Finset (Finset Ξ±)) (ℬ : Finset (Finset Ξ±)) :
      theorem Finset.memberSubfamily_inter {Ξ± : Type u_1} [DecidableEq Ξ±] (a : Ξ±) (π’œ : Finset (Finset Ξ±)) (ℬ : Finset (Finset Ξ±)) :
      theorem Finset.nonMemberSubfamily_union {Ξ± : Type u_1} [DecidableEq Ξ±] (a : Ξ±) (π’œ : Finset (Finset Ξ±)) (ℬ : Finset (Finset Ξ±)) :
      theorem Finset.memberSubfamily_union {Ξ± : Type u_1} [DecidableEq Ξ±] (a : Ξ±) (π’œ : Finset (Finset Ξ±)) (ℬ : Finset (Finset Ξ±)) :
      theorem Finset.card_memberSubfamily_add_card_nonMemberSubfamily {Ξ± : Type u_1} [DecidableEq Ξ±] (a : Ξ±) (π’œ : Finset (Finset Ξ±)) :
      (Finset.memberSubfamily a π’œ).card + (Finset.nonMemberSubfamily a π’œ).card = π’œ.card
      theorem Finset.memberSubfamily_union_nonMemberSubfamily {Ξ± : Type u_1} [DecidableEq Ξ±] (a : Ξ±) (π’œ : Finset (Finset Ξ±)) :
      Finset.memberSubfamily a π’œ βˆͺ Finset.nonMemberSubfamily a π’œ = Finset.image (fun (s : Finset Ξ±) => Finset.erase s a) π’œ
      @[simp]
      theorem Finset.memberSubfamily_memberSubfamily {Ξ± : Type u_1} [DecidableEq Ξ±] {π’œ : Finset (Finset Ξ±)} {a : Ξ±} :
      @[simp]
      theorem Finset.memberSubfamily_nonMemberSubfamily {Ξ± : Type u_1} [DecidableEq Ξ±] {π’œ : Finset (Finset Ξ±)} {a : Ξ±} :
      @[simp]
      theorem Finset.nonMemberSubfamily_memberSubfamily {Ξ± : Type u_1} [DecidableEq Ξ±] {π’œ : Finset (Finset Ξ±)} {a : Ξ±} :
      @[simp]
      theorem Finset.memberSubfamily_image_insert {Ξ± : Type u_1} [DecidableEq Ξ±] {π’œ : Finset (Finset Ξ±)} {a : Ξ±} (hπ’œ : βˆ€ s ∈ π’œ, a βˆ‰ s) :
      Finset.memberSubfamily a (Finset.image (insert a) π’œ) = π’œ
      @[simp]
      theorem Finset.nonMemberSubfamily_image_insert {Ξ± : Type u_1} [DecidableEq Ξ±] {π’œ : Finset (Finset Ξ±)} {a : Ξ±} :
      @[simp]
      theorem Finset.memberSubfamily_image_erase {Ξ± : Type u_1} [DecidableEq Ξ±] {π’œ : Finset (Finset Ξ±)} {a : Ξ±} :
      Finset.memberSubfamily a (Finset.image (fun (x : Finset Ξ±) => Finset.erase x a) π’œ) = βˆ…
      theorem Finset.image_insert_memberSubfamily {Ξ± : Type u_1} [DecidableEq Ξ±] (π’œ : Finset (Finset Ξ±)) (a : Ξ±) :
      Finset.image (insert a) (Finset.memberSubfamily a π’œ) = Finset.filter (fun (x : Finset Ξ±) => a ∈ x) π’œ
      theorem Finset.memberFamily_induction_on {Ξ± : Type u_1} [DecidableEq Ξ±] {p : Finset (Finset Ξ±) β†’ Prop} (π’œ : Finset (Finset Ξ±)) (empty : p βˆ…) (singleton_empty : p {βˆ…}) (subfamily : βˆ€ (a : Ξ±) β¦ƒπ’œ : Finset (Finset Ξ±)⦄, p (Finset.nonMemberSubfamily a π’œ) β†’ p (Finset.memberSubfamily a π’œ) β†’ p π’œ) :
      p π’œ

      Induction principle for finset families. To prove a statement for every finset family, it suffices to prove it for

      • the empty finset family.
      • the finset family which only contains the empty finset.
      • ℬ βˆͺ {s βˆͺ {a} | s ∈ π’ž} assuming the property for ℬ and π’ž, where a is an element of the ground type and π’œ and ℬ are families of finsets not containing a. Note that instead of giving ℬ and π’ž, the subfamily case gives you π’œ = ℬ βˆͺ {s βˆͺ {a} | s ∈ π’ž}, so that ℬ = π’œ.nonMemberSubfamily and π’ž = π’œ.memberSubfamily.

      This is a way of formalising induction on n where π’œ is a finset family on n elements.

      See also Finset.family_induction_on.

      theorem Finset.family_induction_on {Ξ± : Type u_1} [DecidableEq Ξ±] {p : Finset (Finset Ξ±) β†’ Prop} (π’œ : Finset (Finset Ξ±)) (empty : p βˆ…) (singleton_empty : p {βˆ…}) (image_insert : βˆ€ (a : Ξ±) β¦ƒπ’œ : Finset (Finset Ξ±)⦄, (βˆ€ s ∈ π’œ, a βˆ‰ s) β†’ p π’œ β†’ p (Finset.image (insert a) π’œ)) (subfamily : βˆ€ (a : Ξ±) β¦ƒπ’œ : Finset (Finset Ξ±)⦄, p (Finset.filter (fun (x : Finset Ξ±) => a βˆ‰ x) π’œ) β†’ p (Finset.filter (fun (x : Finset Ξ±) => a ∈ x) π’œ) β†’ p π’œ) :
      p π’œ

      Induction principle for finset families. To prove a statement for every finset family, it suffices to prove it for

      • the empty finset family.
      • the finset family which only contains the empty finset.
      • {s βˆͺ {a} | s ∈ π’œ} assuming the property for π’œ a family of finsets not containing a.
      • ℬ βˆͺ π’ž assuming the property for ℬ and π’ž, where a is an element of the ground type and ℬis a family of finsets not containing a and π’ž a family of finsets containing a. Note that instead of giving ℬ and π’ž, the subfamily case gives you π’œ = ℬ βˆͺ π’ž, so that ℬ = π’œ.filter (a βˆ‰ Β·) and π’ž = π’œ.filter (a ∈ Β·).

      This is a way of formalising induction on n where π’œ is a finset family on n elements.

      See also Finset.memberFamily_induction_on.

      def Down.compression {Ξ± : Type u_1} [DecidableEq Ξ±] (a : Ξ±) (π’œ : Finset (Finset Ξ±)) :
      Finset (Finset Ξ±)

      a-down-compressing π’œ means removing a from the elements of π’œ that contain it, when the resulting Finset is not already in π’œ.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For

        a-down-compressing π’œ means removing a from the elements of π’œ that contain it, when the resulting Finset is not already in π’œ.

        Equations
        Instances For
          theorem Down.mem_compression {Ξ± : Type u_1} [DecidableEq Ξ±] {π’œ : Finset (Finset Ξ±)} {s : Finset Ξ±} {a : Ξ±} :
          s ∈ Down.compression a π’œ ↔ s ∈ π’œ ∧ Finset.erase s a ∈ π’œ ∨ s βˆ‰ π’œ ∧ insert a s ∈ π’œ

          a is in the down-compressed family iff it's in the original and its compression is in the original, or it's not in the original but it's the compression of something in the original.

          theorem Down.erase_mem_compression {Ξ± : Type u_1} [DecidableEq Ξ±] {π’œ : Finset (Finset Ξ±)} {s : Finset Ξ±} {a : Ξ±} (hs : s ∈ π’œ) :
          theorem Down.erase_mem_compression_of_mem_compression {Ξ± : Type u_1} [DecidableEq Ξ±] {π’œ : Finset (Finset Ξ±)} {s : Finset Ξ±} {a : Ξ±} :
          s ∈ Down.compression a π’œ β†’ Finset.erase s a ∈ Down.compression a π’œ
          theorem Down.mem_compression_of_insert_mem_compression {Ξ± : Type u_1} [DecidableEq Ξ±] {π’œ : Finset (Finset Ξ±)} {s : Finset Ξ±} {a : Ξ±} (h : insert a s ∈ Down.compression a π’œ) :
          @[simp]
          theorem Down.compression_idem {Ξ± : Type u_1} [DecidableEq Ξ±] (a : Ξ±) (π’œ : Finset (Finset Ξ±)) :

          Down-compressing a family is idempotent.

          @[simp]
          theorem Down.card_compression {Ξ± : Type u_1} [DecidableEq Ξ±] (a : Ξ±) (π’œ : Finset (Finset Ξ±)) :
          (Down.compression a π’œ).card = π’œ.card

          Down-compressing a family doesn't change its size.