Documentation

Mathlib.Topology.Category.Profinite.Nobeling

Nöbeling's theorem #

This file proves Nöbeling's theorem.

Main result #

Proof idea #

We follow the proof of theorem 5.4 in [scholze2019condensed], in which the idea is to embed S in a product of I copies of Bool for some sufficiently large I, and then to choose a well-ordering on I and use ordinal induction over that well-order. Here we can let I be the set of clopen subsets of S since S is totally separated.

The above means it suffices to prove the following statement: For a closed subset C of I → Bool, the -module LocallyConstant C ℤ is free.

For i : I, let e C i : LocallyConstant C ℤ denote the map fun f ↦ (if f.val i then 1 else 0).

The basis will consist of products e C iᵣ * ⋯ * e C i₁ with iᵣ > ⋯ > i₁ which cannot be written as linear combinations of lexicographically smaller products. We call this set GoodProducts C

What is proved by ordinal induction is that this set is linearly independent. The fact that it spans can be proved directly.

References #

Projection maps #

The purpose of this section is twofold.

Firstly, in the proof that the set GoodProducts C spans the whole module LocallyConstant C ℤ, we need to project C down to finite discrete subsets and write C as a cofiltered limit of those.

Secondly, in the inductive argument, we need to project C down to "smaller" sets satisfying the inductive hypothesis.

In this section we define the relevant projection maps and prove some compatibility results.

Main definitions #

def Profinite.NobelingProof.Proj {I : Type u} (J : IProp) [(i : I) → Decidable (J i)] :
(IBool)IBool

The projection mapping everything that satisfies J i to itself, and everything else to false

Equations
Instances For
    def Profinite.NobelingProof.π {I : Type u} (C : Set (IBool)) (J : IProp) [(i : I) → Decidable (J i)] :
    Set (IBool)

    The image of Proj π J

    Equations
    Instances For
      @[simp]
      theorem Profinite.NobelingProof.ProjRestrict_coe {I : Type u} (C : Set (IBool)) (J : IProp) [(i : I) → Decidable (J i)] :
      ∀ (a : C) (a_1 : I), (Profinite.NobelingProof.ProjRestrict C J a) a_1 = Profinite.NobelingProof.Proj J (a) a_1
      def Profinite.NobelingProof.ProjRestrict {I : Type u} (C : Set (IBool)) (J : IProp) [(i : I) → Decidable (J i)] :
      C(Profinite.NobelingProof.π C J)

      The restriction of Proj π J to a subset, mapping to its image.

      Equations
      Instances For
        @[simp]
        theorem Profinite.NobelingProof.proj_eq_self {I : Type u} (J : IProp) [(i : I) → Decidable (J i)] {x : IBool} (h : ∀ (i : I), x i falseJ i) :
        theorem Profinite.NobelingProof.proj_prop_eq_self {I : Type u} (C : Set (IBool)) (J : IProp) [(i : I) → Decidable (J i)] (hh : ∀ (i : I), xC, x i falseJ i) :
        theorem Profinite.NobelingProof.proj_comp_of_subset {I : Type u} (J : IProp) (K : IProp) [(i : I) → Decidable (J i)] [(i : I) → Decidable (K i)] (h : ∀ (i : I), J iK i) :
        theorem Profinite.NobelingProof.proj_eq_of_subset {I : Type u} (C : Set (IBool)) (J : IProp) (K : IProp) [(i : I) → Decidable (J i)] [(i : I) → Decidable (K i)] (h : ∀ (i : I), J iK i) :
        @[simp]
        theorem Profinite.NobelingProof.ProjRestricts_coe {I : Type u} (C : Set (IBool)) {J : IProp} {K : IProp} [(i : I) → Decidable (J i)] [(i : I) → Decidable (K i)] (h : ∀ (i : I), J iK i) :
        def Profinite.NobelingProof.ProjRestricts {I : Type u} (C : Set (IBool)) {J : IProp} {K : IProp} [(i : I) → Decidable (J i)] [(i : I) → Decidable (K i)] (h : ∀ (i : I), J iK i) :

        A variant of ProjRestrict with domain of the form π C K

        Equations
        Instances For
          @[simp]
          theorem Profinite.NobelingProof.continuous_projRestricts {I : Type u} (C : Set (IBool)) {J : IProp} {K : IProp} [(i : I) → Decidable (J i)] [(i : I) → Decidable (K i)] (h : ∀ (i : I), J iK i) :
          theorem Profinite.NobelingProof.surjective_projRestricts {I : Type u} (C : Set (IBool)) {J : IProp} {K : IProp} [(i : I) → Decidable (J i)] [(i : I) → Decidable (K i)] (h : ∀ (i : I), J iK i) :
          theorem Profinite.NobelingProof.projRestricts_eq_id {I : Type u} (C : Set (IBool)) (J : IProp) [(i : I) → Decidable (J i)] :
          theorem Profinite.NobelingProof.projRestricts_eq_comp {I : Type u} (C : Set (IBool)) {J : IProp} {K : IProp} {L : IProp} [(i : I) → Decidable (J i)] [(i : I) → Decidable (K i)] [(i : I) → Decidable (L i)] (hJK : ∀ (i : I), J iK i) (hKL : ∀ (i : I), K iL i) :
          theorem Profinite.NobelingProof.projRestricts_comp_projRestrict {I : Type u} (C : Set (IBool)) {J : IProp} {K : IProp} [(i : I) → Decidable (J i)] [(i : I) → Decidable (K i)] (h : ∀ (i : I), J iK i) :
          def Profinite.NobelingProof.iso_map {I : Type u} (C : Set (IBool)) (J : IProp) [(i : I) → Decidable (J i)] :

          The objectwise map in the isomorphism spanFunctorProfinite.indexFunctor

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            noncomputable def Profinite.NobelingProof.spanFunctor {I : Type u} {C : Set (IBool)} (hC : IsCompact C) [(s : Finset I) → (i : I) → Decidable (i s)] :

            For a given compact subset C of I → Bool, spanFunctor is the functor from the poset of finsets of I to Profinite, sending a finite subset set J to the image of C under the projection Proj J.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              noncomputable def Profinite.NobelingProof.spanCone {I : Type u} {C : Set (IBool)} (hC : IsCompact C) [(s : Finset I) → (i : I) → Decidable (i s)] :

              The limit cone on spanFunctor with point C.

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                noncomputable def Profinite.NobelingProof.spanCone_isLimit {I : Type u} {C : Set (IBool)} (hC : IsCompact C) [(s : Finset I) → (i : I) → Decidable (i s)] :

                spanCone is a limit cone.

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

                  Defining the basis #

                  Our proposed basis consists of products e C iᵣ * ⋯ * e C i₁ with iᵣ > ⋯ > i₁ which cannot be written as linear combinations of lexicographically smaller products. See below for the definition of e.

                  Main definitions #

                  Main results #

                  def Profinite.NobelingProof.e {I : Type u} (C : Set (IBool)) (i : I) :

                  e C i is the locally constant map from C : Set (I → Bool) to sending f to 1 if f.val i = true, and 0 otherwise.

                  Equations
                  Instances For

                    Products I is the type of lists of decreasing elements of I, so a typical element is [i₁, i₂, ...] with i₁ > i₂ > .... We order Products I lexicographically, so [] < [i₁, ...], and [i₁, i₂, ...] < [j₁, j₂, ...] if either i₁ < j₁, or i₁ = j₁ and [i₂, ...] < [j₂, ...].

                    Terms m = [i₁, i₂, ..., iᵣ] of this type will be used to represent products of the form e C i₁ ··· e C iᵣ : LocallyConstant C ℤ . The function associated to m is m.eval.

                    Equations
                    Instances For
                      Equations

                      The evaluation e C i₁ ··· e C iᵣ : C → ℤ of a formal product [i₁, i₂, ..., iᵣ].

                      Equations
                      Instances For

                        The predicate on products which we prove picks out a basis of LocallyConstant C ℤ. We call such a product "good".

                        Equations
                        • One or more equations did not get rendered due to their size.
                        Instances For
                          theorem Profinite.NobelingProof.Products.eval_eq {I : Type u} [LinearOrder I] (C : Set (IBool)) (l : Profinite.NobelingProof.Products I) (x : C) :
                          (Profinite.NobelingProof.Products.eval C l) x = if il, x i = true then 1 else 0
                          theorem Profinite.NobelingProof.Products.evalFacProps {I : Type u} [LinearOrder I] (C : Set (IBool)) {l : Profinite.NobelingProof.Products I} (J : IProp) (K : IProp) (h : al, J a) [(j : I) → Decidable (J j)] [(j : I) → Decidable (K j)] (hJK : ∀ (i : I), J iK i) :

                          The good products span #

                          Most of the argument is developing an API for π C (· ∈ s) when s : Finset I; then the image of C is finite with the discrete topology. In this case, there is a direct argument that the good products span. The general result is deduced from this.

                          Main theorems #

                          noncomputable def Profinite.NobelingProof.πJ {I : Type u} [LinearOrder I] (C : Set (IBool)) (s : Finset I) :

                          The -linear map induced by precomposition of the projection C → π C (· ∈ s).

                          Equations
                          Instances For

                            π C (· ∈ s) is finite for a finite set s.

                            Equations
                            • One or more equations did not get rendered due to their size.
                            noncomputable def Profinite.NobelingProof.spanFinBasis {I : Type u} [LinearOrder I] (C : Set (IBool)) (s : Finset I) (x : (Profinite.NobelingProof.π C fun (x : I) => x s)) :

                            The Kronecker delta as a locally constant map from π C (· ∈ s) to .

                            Equations
                            Instances For
                              def Profinite.NobelingProof.factors {I : Type u} [LinearOrder I] (C : Set (IBool)) (s : Finset I) (x : (Profinite.NobelingProof.π C fun (x : I) => x s)) :

                              A certain explicit list of locally constant maps. The theorem factors_prod_eq_basis shows that the product of the elements in this list is the delta function spanFinBasis C s x.

                              Equations
                              • One or more equations did not get rendered due to their size.
                              Instances For
                                theorem Profinite.NobelingProof.factors_prod_eq_basis_of_eq {I : Type u} [LinearOrder I] (C : Set (IBool)) (s : Finset I) {x : (Profinite.NobelingProof.π C fun (x : I) => x s)} {y : (Profinite.NobelingProof.π C fun (x : I) => x s)} (h : y = x) :
                                theorem Profinite.NobelingProof.e_mem_of_eq_true {I : Type u} [LinearOrder I] (C : Set (IBool)) (s : Finset I) {x : (Profinite.NobelingProof.π C fun (x : I) => x s)} {a : I} (hx : x a = true) :
                                theorem Profinite.NobelingProof.one_sub_e_mem_of_false {I : Type u} [LinearOrder I] (C : Set (IBool)) (s : Finset I) {x : (Profinite.NobelingProof.π C fun (x : I) => x s)} {y : (Profinite.NobelingProof.π C fun (x : I) => x s)} {a : I} (ha : y a = true) (hx : x a = false) :
                                theorem Profinite.NobelingProof.factors_prod_eq_basis_of_ne {I : Type u} [LinearOrder I] (C : Set (IBool)) (s : Finset I) {x : (Profinite.NobelingProof.π C fun (x : I) => x s)} {y : (Profinite.NobelingProof.π C fun (x : I) => x s)} (h : y x) :

                                If s is finite, the product of the elements of the list factors C s x is the delta function at x.

                                If s is a finite subset of I, then the good products span.

                                theorem Profinite.NobelingProof.fin_comap_jointlySurjective {I : Type u} [LinearOrder I] (C : Set (IBool)) (hC : IsClosed C) (f : LocallyConstant C ) :
                                ∃ (s : Finset I) (g : LocallyConstant (Profinite.NobelingProof.π C fun (x : I) => x s) ), f = LocallyConstant.comap { toFun := Profinite.NobelingProof.ProjRestrict C fun (x : I) => x s, continuous_toFun := } g

                                The good products span all of LocallyConstant C ℤ if C is closed.

                                Relating elements of the well-order I with ordinals #

                                We choose a well-ordering on I. This amounts to regarding I as an ordinal, and as such it can be regarded as the set of all strictly smaller ordinals, allowing to apply ordinal induction.

                                Main definitions #

                                def Profinite.NobelingProof.ord (I : Type u) [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (i : I) :

                                A term of I regarded as an ordinal.

                                Equations
                                Instances For
                                  noncomputable def Profinite.NobelingProof.term (I : Type u) [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] {o : Ordinal.{u}} (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :
                                  I

                                  An ordinal regarded as a term of I.

                                  Equations
                                  Instances For
                                    theorem Profinite.NobelingProof.term_ord_aux {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] {i : I} (ho : Profinite.NobelingProof.ord I i < Ordinal.type fun (x x_1 : I) => x < x_1) :
                                    @[simp]
                                    theorem Profinite.NobelingProof.ord_term_aux {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] {o : Ordinal.{u}} (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :
                                    theorem Profinite.NobelingProof.ord_term {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] {o : Ordinal.{u}} (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) (i : I) :
                                    def Profinite.NobelingProof.contained {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) (o : Ordinal.{u}) :

                                    A predicate saying that C is "small" enough to satisfy the inductive hypothesis.

                                    Equations
                                    Instances For
                                      def Profinite.NobelingProof.P (I : Type u) [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (o : Ordinal.{u}) :

                                      The predicate on ordinals which we prove by induction, see GoodProducts.P0, GoodProducts.Plimit and GoodProducts.linearIndependentAux in the section Induction below

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

                                        The zero case of the induction #

                                        In this case, we have contained C 0 which means that C is either empty or a singleton.

                                        The empty list as a Products 

                                        Equations
                                        • Profinite.NobelingProof.Products.nil = { val := [], property := }
                                        Instances For
                                          theorem Profinite.NobelingProof.Products.lt_nil_empty {I : Type u} [LinearOrder I] :
                                          {m : Profinite.NobelingProof.Products I | m < Profinite.NobelingProof.Products.nil} =
                                          theorem Profinite.NobelingProof.Products.isGood_nil {I : Type u} [LinearOrder I] :
                                          Profinite.NobelingProof.Products.isGood {fun (x : I) => false} Profinite.NobelingProof.Products.nil

                                          There is a unique GoodProducts for the singleton {fun _ ↦ false}.

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

                                          -linear maps induced by projections #

                                          We define injective -linear maps between modules of the form LocallyConstant C ℤ induced by precomposition with the projections defined in the section Projections.

                                          Main definitions #

                                          Main result #

                                          theorem Profinite.NobelingProof.isClosed_proj {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) (o : Ordinal.{u}) (hC : IsClosed C) :
                                          @[simp]
                                          theorem Profinite.NobelingProof.πs_apply_apply {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) (o : Ordinal.{u}) (g : LocallyConstant (Profinite.NobelingProof.π C fun (x : I) => Profinite.NobelingProof.ord I x < o) ) :
                                          ∀ (a : C), ((Profinite.NobelingProof.πs C o) g) a = g (Profinite.NobelingProof.ProjRestrict C (fun (x : I) => Profinite.NobelingProof.ord I x < o) a)
                                          noncomputable def Profinite.NobelingProof.πs {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) (o : Ordinal.{u}) :

                                          The -linear map induced by precomposition of the projection C → π C (ord I · < o).

                                          Equations
                                          • One or more equations did not get rendered due to their size.
                                          Instances For
                                            @[simp]
                                            theorem Profinite.NobelingProof.πs'_apply_apply {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o₁ : Ordinal.{u}} {o₂ : Ordinal.{u}} (h : o₁ o₂) (g : LocallyConstant (Profinite.NobelingProof.π C fun (x : I) => Profinite.NobelingProof.ord I x < o₁) ) :
                                            noncomputable def Profinite.NobelingProof.πs' {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o₁ : Ordinal.{u}} {o₂ : Ordinal.{u}} (h : o₁ o₂) :

                                            The -linear map induced by precomposition of the projection π C (ord I · < o₂) → π C (ord I · < o₁) for o₁ ≤ o₂.

                                            Equations
                                            Instances For
                                              theorem Profinite.NobelingProof.coe_πs' {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o₁ : Ordinal.{u}} {o₂ : Ordinal.{u}} (h : o₁ o₂) (f : LocallyConstant (Profinite.NobelingProof.π C fun (x : I) => Profinite.NobelingProof.ord I x < o₁) ) :
                                              theorem Profinite.NobelingProof.injective_πs' {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o₁ : Ordinal.{u}} {o₂ : Ordinal.{u}} (h : o₁ o₂) :
                                              theorem Profinite.NobelingProof.Products.lt_ord_of_lt {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] {l : Profinite.NobelingProof.Products I} {m : Profinite.NobelingProof.Products I} {o : Ordinal.{u}} (h₁ : m < l) (h₂ : il, Profinite.NobelingProof.ord I i < o) (i : I) :

                                              If l is good w.r.t. π C (ord I · < o₁) and o₁ ≤ o₂, then it is good w.r.t. π C (ord I · < o₂)

                                              The limit case of the induction #

                                              We relate linear independence in LocallyConstant (π C (ord I · < o')) ℤ with linear independence in LocallyConstant C ℤ, where contained C o and o' < o.

                                              When o is a limit ordinal, we prove that the good products in LocallyConstant C ℤ are linearly independent if and only if a certain directed union is linearly independent. Each term in this directed union is in bijection with the good products w.r.t. π C (ord I · < o') for an ordinal o' < o, and these are linearly independent by the inductive hypothesis.

                                              Main definitions #

                                              Main results #

                                              def Profinite.NobelingProof.GoodProducts.smaller {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) (o : Ordinal.{u}) :

                                              The image of the GoodProducts for π C (ord I · < o) in LocallyConstant C ℤ. The name smaller refers to the setting in which we will use this, when we are mapping in GoodProducts from a smaller set, i.e. when o is a smaller ordinal than the one C is "contained" in.

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

                                                The map from the image of the GoodProducts in LocallyConstant (π C (ord I · < o)) ℤ to smaller C o

                                                Equations
                                                Instances For

                                                  The image of the GoodProducts in C is equivalent to the union of smaller C o' over all ordinals o' < o.

                                                  Equations
                                                  Instances For
                                                    theorem Profinite.NobelingProof.GoodProducts.range_equiv_factorization {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (ho : Ordinal.IsLimit o) (hsC : Profinite.NobelingProof.contained C o) :
                                                    (fun (p : (⋃ (e : { o' : Ordinal.{u} // o' < o }), Profinite.NobelingProof.GoodProducts.smaller C e)) => p) (Profinite.NobelingProof.GoodProducts.range_equiv C ho hsC).toFun = fun (p : (Profinite.NobelingProof.GoodProducts.range C)) => p

                                                    The successor case in the induction #

                                                    Here we assume that o is an ordinal such that contained C (o+1) and o < I. The element in I corresponding to o is called term I ho, but in this informal docstring we refer to it simply as o.

                                                    This section follows the proof in [scholze2019condensed] quite closely. A translation of the notation there is as follows:

                                                    [scholze2019condensed]                  | This file
                                                    `S₀`                                    |`C0`
                                                    `S₁`                                    |`C1`
                                                    `\overline{S}`                          |`π C (ord I · < o)
                                                    `\overline{S}'`                         |`C'`
                                                    The left map in the exact sequence      |`πs`
                                                    The right map in the exact sequence     |`Linear_CC'`
                                                    

                                                    When comparing the proof of the successor case in Theorem 5.4 in [scholze2019condensed] with this proof, one should read the phrase "is a basis" as "is linearly independent". Also, the short exact sequence in [scholze2019condensed] is only proved to be left exact here (indeed, that is enough since we are only proving linear independence).

                                                    This section is split into two sections. The first one, ExactSequence defines the left exact sequence mentioned in the previous paragraph (see succ_mono and succ_exact). It corresponds to the penultimate paragraph of the proof in [scholze2019condensed]. The second one, GoodProducts corresponds to the last paragraph in the proof in [scholze2019condensed].

                                                    Main definitions #

                                                    The main definitions in the section ExactSequence are all just notation explained in the table above.

                                                    The main definitions in the section GoodProducts are as follows:

                                                    Main results #

                                                    The main results in the section GoodProducts are as follows:

                                                    def Profinite.NobelingProof.C0 {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :
                                                    Set (IBool)

                                                    The subset of C consisting of those elements whose o-th entry is false.

                                                    Equations
                                                    Instances For
                                                      def Profinite.NobelingProof.C1 {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :
                                                      Set (IBool)

                                                      The subset of C consisting of those elements whose o-th entry is true.

                                                      Equations
                                                      Instances For
                                                        theorem Profinite.NobelingProof.isClosed_C0 {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (hC : IsClosed C) (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :
                                                        theorem Profinite.NobelingProof.isClosed_C1 {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (hC : IsClosed C) (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :
                                                        theorem Profinite.NobelingProof.contained_C1 {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :
                                                        theorem Profinite.NobelingProof.union_C0C1_eq {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :
                                                        def Profinite.NobelingProof.C' {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :
                                                        Set (IBool)

                                                        The intersection of C0 and the projection of C1. We will apply the inductive hypothesis to this set.

                                                        Equations
                                                        Instances For
                                                          theorem Profinite.NobelingProof.isClosed_C' {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (hC : IsClosed C) (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :
                                                          theorem Profinite.NobelingProof.contained_C' {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :
                                                          noncomputable def Profinite.NobelingProof.SwapTrue {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (o : Ordinal.{u}) :
                                                          (IBool)IBool

                                                          Swapping the o-th coordinate to true.

                                                          Equations
                                                          Instances For
                                                            def Profinite.NobelingProof.CC'₀ {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :
                                                            (Profinite.NobelingProof.C' C ho)C

                                                            The first way to map C' into C.

                                                            Equations
                                                            Instances For
                                                              noncomputable def Profinite.NobelingProof.CC'₁ {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (hsC : Profinite.NobelingProof.contained C (Order.succ o)) (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :
                                                              (Profinite.NobelingProof.C' C ho)C

                                                              The second way to map C' into C.

                                                              Equations
                                                              Instances For
                                                                theorem Profinite.NobelingProof.continuous_CC'₀ {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :
                                                                theorem Profinite.NobelingProof.continuous_CC'₁ {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (hsC : Profinite.NobelingProof.contained C (Order.succ o)) (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :
                                                                noncomputable def Profinite.NobelingProof.Linear_CC'₀ {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :

                                                                The -linear map induced by precomposing with CC'₀

                                                                Equations
                                                                Instances For
                                                                  noncomputable def Profinite.NobelingProof.Linear_CC'₁ {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (hsC : Profinite.NobelingProof.contained C (Order.succ o)) (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :

                                                                  The -linear map induced by precomposing with CC'₁

                                                                  Equations
                                                                  Instances For
                                                                    noncomputable def Profinite.NobelingProof.Linear_CC' {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (hsC : Profinite.NobelingProof.contained C (Order.succ o)) (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :

                                                                    The difference between Linear_CC'₁ and Linear_CC'₀.

                                                                    Equations
                                                                    Instances For
                                                                      theorem Profinite.NobelingProof.CC_comp_zero {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (hsC : Profinite.NobelingProof.contained C (Order.succ o)) (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) (y : LocallyConstant (Profinite.NobelingProof.π C fun (x : I) => Profinite.NobelingProof.ord I x < o) ) :
                                                                      theorem Profinite.NobelingProof.C0_projOrd {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (hsC : Profinite.NobelingProof.contained C (Order.succ o)) (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) {x : IBool} (hx : x Profinite.NobelingProof.C0 C ho) :
                                                                      theorem Profinite.NobelingProof.C1_projOrd {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (hsC : Profinite.NobelingProof.contained C (Order.succ o)) (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) {x : IBool} (hx : x Profinite.NobelingProof.C1 C ho) :
                                                                      theorem Profinite.NobelingProof.CC_exact {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (hC : IsClosed C) (hsC : Profinite.NobelingProof.contained C (Order.succ o)) (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) {f : LocallyConstant C } (hf : (Profinite.NobelingProof.Linear_CC' C hsC ho) f = 0) :
                                                                      def Profinite.NobelingProof.GoodProducts.MaxProducts {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :

                                                                      The GoodProducts in C that contain o (they necessarily start with o, see GoodProducts.head!_eq_o_of_maxProducts)

                                                                      Equations
                                                                      Instances For

                                                                        The inclusion map from the sum of GoodProducts (π C (ord I · < o)) and (MaxProducts C ho) to Products I.

                                                                        Equations
                                                                        Instances For
                                                                          theorem Profinite.NobelingProof.GoodProducts.injective_sum_to {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) :

                                                                          The equivalence from the sum of GoodProducts (π C (ord I · < o)) and (MaxProducts C ho) to GoodProducts C.

                                                                          Equations
                                                                          Instances For

                                                                            Let

                                                                            N := LocallyConstant (π C (ord I · < o)) ℤ

                                                                            M := LocallyConstant C ℤ

                                                                            P := LocallyConstant (C' C ho) ℤ

                                                                            ι := GoodProducts (π C (ord I · < o))

                                                                            ι' := GoodProducts (C' C ho')

                                                                            v : ι → N := GoodProducts.eval (π C (ord I · < o))

                                                                            Then SumEval C ho is the map u in the diagram below. It is linearly independent if and only if GoodProducts.eval C is, see linearIndependent_iff_sum. The top row is the exact sequence given by succ_exact and succ_mono. The left square commutes by GoodProducts.square_commutes.

                                                                            0 --→ N --→ M --→  P
                                                                                  ↑     ↑      ↑
                                                                                 v|    u|      |
                                                                                  ιι ⊕ ι' ← ι'
                                                                            
                                                                            Equations
                                                                            • One or more equations did not get rendered due to their size.
                                                                            Instances For
                                                                              theorem Profinite.NobelingProof.swapTrue_eq_true {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] {o : Ordinal.{u}} (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) (x : IBool) :
                                                                              theorem Profinite.NobelingProof.mem_C'_eq_false {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) (x : IBool) :
                                                                              theorem Profinite.NobelingProof.Products.max_eq_o_cons_tail' {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] {o : Ordinal.{u}} (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) [Inhabited I] (l : Profinite.NobelingProof.Products I) (hl : l []) (hlh : List.head! l = Profinite.NobelingProof.term I ho) (hlc : List.Chain' (fun (x x_1 : I) => x > x_1) (Profinite.NobelingProof.term I ho :: (Profinite.NobelingProof.Products.Tail l))) :
                                                                              theorem Profinite.NobelingProof.Products.evalCons {I : Type u} [LinearOrder I] (C : Set (IBool)) {l : List I} {a : I} (hla : List.Chain' (fun (x x_1 : I) => x > x_1) (a :: l)) :
                                                                              Profinite.NobelingProof.Products.eval C { val := a :: l, property := hla } = Profinite.NobelingProof.e C a * Profinite.NobelingProof.Products.eval C { val := l, property := }
                                                                              theorem Profinite.NobelingProof.GoodProducts.chain'_cons_of_lt {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (hsC : Profinite.NobelingProof.contained C (Order.succ o)) (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) (l : (Profinite.NobelingProof.GoodProducts.MaxProducts C ho)) (q : Profinite.NobelingProof.Products I) (hq : q < Profinite.NobelingProof.Products.Tail l) :
                                                                              List.Chain' (fun (x x_1 : I) => x > x_1) (Profinite.NobelingProof.term I ho :: q)
                                                                              theorem Profinite.NobelingProof.GoodProducts.good_lt_maxProducts {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) {o : Ordinal.{u}} (hsC : Profinite.NobelingProof.contained C (Order.succ o)) (ho : o < Ordinal.type fun (x x_1 : I) => x < x_1) (q : (Profinite.NobelingProof.GoodProducts (Profinite.NobelingProof.π C fun (x : I) => Profinite.NobelingProof.ord I x < o))) (l : (Profinite.NobelingProof.GoodProducts.MaxProducts C ho)) :
                                                                              List.Lex (fun (x x_1 : I) => x < x_1) q l

                                                                              Given l : MaxProducts C ho, its Tail is a GoodProducts (C' C ho).

                                                                              Equations
                                                                              Instances For

                                                                                The induction #

                                                                                Here we put together the results of the sections Zero, Limit and Successor to prove the predicate P I o holds for all ordinals o, and conclude with the main result:

                                                                                We also define

                                                                                noncomputable def Profinite.NobelingProof.GoodProducts.Basis {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] (C : Set (IBool)) (hC : IsClosed C) :

                                                                                GoodProducts C as a -basis for LocallyConstant C ℤ.

                                                                                Equations
                                                                                Instances For
                                                                                  theorem Profinite.NobelingProof.Nobeling_aux {I : Type u} [LinearOrder I] [IsWellOrder I fun (x x_1 : I) => x < x_1] {S : Profinite} {ι : S.toCompHaus.toTopIBool} (hι : ClosedEmbedding ι) :
                                                                                  Module.Free (LocallyConstant S.toCompHaus.toTop )

                                                                                  Given a profinite set S and a closed embedding S → (I → Bool), the -module LocallyConstant C ℤ is free.

                                                                                  noncomputable def Profinite.Nobeling.ι (S : Profinite) :
                                                                                  S.toCompHaus.toTop{ C : Set S.toCompHaus.toTop // IsClopen C }Bool

                                                                                  The embedding S → (I → Bool) where I is the set of clopens of S.

                                                                                  Equations
                                                                                  Instances For

                                                                                    Nöbeling's theorem: the -module LocallyConstant S ℤ is free for every S : Profinite

                                                                                    Equations
                                                                                    • =