Commit 2025-03-17 13:17 4eedae49

View on Github →

chore(Algebra/Algebra): reorganize Algebra.adjoin and complete lattice (#22557) This PR creates a new file that holds the definition and basic results on Algebra.adjoin and the resulting CompleteLattice (Subalgebra R A) instance, moving definitions downstream from Subalgebra/Basic.lean and some lemmas upstream from RingTheory/Adjoin/Basic.lean. A nice consequence is that we can avoid importing linear algebra (in the form of Basis) in quite a few measure theory files. (In fact we should be able to do a bit better and avoid Algebra altogether, but that's for later PRs.)

Estimated changes

deleted theorem AlgHom.eqOn_sup
deleted theorem AlgHom.equalizer_eq_top
deleted theorem AlgHom.equalizer_same
deleted theorem AlgHom.ext_on_codisjoint
deleted theorem AlgHom.range_eq_top
deleted def Algebra.adjoin
deleted theorem Algebra.coe_bot
deleted theorem Algebra.coe_iInf
deleted theorem Algebra.coe_inf
deleted theorem Algebra.coe_sInf
deleted theorem Algebra.coe_top
deleted theorem Algebra.comap_top
deleted theorem Algebra.eq_top_iff
deleted theorem Algebra.iInf_toSubmodule
deleted theorem Algebra.iSup_induction'
deleted theorem Algebra.iSup_induction
deleted theorem Algebra.inf_toSubmodule
deleted theorem Algebra.inf_toSubsemiring
deleted theorem Algebra.map_bot
deleted theorem Algebra.map_iInf
deleted theorem Algebra.map_inf
deleted theorem Algebra.map_sup
deleted theorem Algebra.map_top
deleted theorem Algebra.mem_bot
deleted theorem Algebra.mem_iInf
deleted theorem Algebra.mem_iSup_of_mem
deleted theorem Algebra.mem_inf
deleted theorem Algebra.mem_sInf
deleted theorem Algebra.mem_sup_left
deleted theorem Algebra.mem_sup_right
deleted theorem Algebra.mem_top
deleted theorem Algebra.mul_mem_sup
deleted theorem Algebra.range_id
deleted theorem Algebra.range_ofId
deleted theorem Algebra.sInf_toSubmodule
deleted theorem Algebra.sSup_def
deleted theorem Algebra.sup_def
deleted theorem Algebra.sup_toSubsemiring
deleted theorem Algebra.toSubmodule_bot
deleted theorem Algebra.toSubring_eq_top
deleted def Algebra.toTop
deleted theorem Algebra.top_toSubmodule
deleted theorem Algebra.top_toSubring
deleted theorem Algebra.top_toSubsemiring
deleted theorem Subalgebra.center_eq_top
deleted theorem Subalgebra.map_comap_eq
deleted def Subalgebra.topEquiv
added theorem AlgHom.adjoin_ext
added theorem AlgHom.eqOn_adjoin_iff
added theorem AlgHom.eqOn_sup
added theorem AlgHom.equalizer_same
added theorem AlgHom.map_adjoin
added theorem AlgHom.range_eq_top
added def Algebra.adjoin
added theorem Algebra.adjoin_empty
added theorem Algebra.adjoin_eq
added theorem Algebra.adjoin_eq_sInf
added theorem Algebra.adjoin_eq_span
added theorem Algebra.adjoin_iUnion
added theorem Algebra.adjoin_image
added theorem Algebra.adjoin_int
added theorem Algebra.adjoin_le
added theorem Algebra.adjoin_le_iff
added theorem Algebra.adjoin_mono
added theorem Algebra.adjoin_nat
added theorem Algebra.adjoin_span
added theorem Algebra.adjoin_union
added theorem Algebra.adjoin_univ
added theorem Algebra.coe_bot
added theorem Algebra.coe_iInf
added theorem Algebra.coe_inf
added theorem Algebra.coe_sInf
added theorem Algebra.coe_top
added theorem Algebra.comap_top
added theorem Algebra.eq_top_iff
added theorem Algebra.iSup_induction
added theorem Algebra.map_bot
added theorem Algebra.map_iInf
added theorem Algebra.map_inf
added theorem Algebra.map_sup
added theorem Algebra.map_top
added theorem Algebra.mem_adjoin_iff
added theorem Algebra.mem_bot
added theorem Algebra.mem_iInf
added theorem Algebra.mem_inf
added theorem Algebra.mem_sInf
added theorem Algebra.mem_sup_left
added theorem Algebra.mem_sup_right
added theorem Algebra.mem_top
added theorem Algebra.mul_mem_sup
added theorem Algebra.range_id
added theorem Algebra.range_ofId
added theorem Algebra.sSup_def
added theorem Algebra.span_le_adjoin
added theorem Algebra.subset_adjoin
added theorem Algebra.sup_def
added def Algebra.toTop
added theorem Algebra.top_toSubring
deleted theorem AlgHom.adjoin_ext
deleted theorem AlgHom.eqOn_adjoin_iff
deleted theorem AlgHom.ext_of_eq_adjoin
deleted theorem AlgHom.map_adjoin
deleted theorem Algebra.adjoin_empty
deleted theorem Algebra.adjoin_eq
deleted theorem Algebra.adjoin_eq_of_le
deleted theorem Algebra.adjoin_eq_sInf
deleted theorem Algebra.adjoin_eq_span
deleted theorem Algebra.adjoin_iUnion
deleted theorem Algebra.adjoin_image
deleted theorem Algebra.adjoin_induction'
deleted theorem Algebra.adjoin_induction
deleted theorem Algebra.adjoin_int
deleted theorem Algebra.adjoin_le
deleted theorem Algebra.adjoin_le_iff
deleted theorem Algebra.adjoin_mono
deleted theorem Algebra.adjoin_nat
deleted theorem Algebra.adjoin_span
deleted theorem Algebra.adjoin_union
deleted theorem Algebra.adjoin_univ
deleted theorem Algebra.mem_adjoin_iff
deleted theorem Algebra.span_le_adjoin
deleted theorem Algebra.subset_adjoin
deleted theorem Subalgebra.comap_map_eq