Commit 2025-02-10 19:23 e790abc2

View on Github →

chore(Order/Filter): split AtTopBot.lean (#21672) This PR splits Order/Filter/AtTopBot.lean into the following files:

  • Order/Filter/AtTopBot/Defs.lean: definition and elementary properties
  • Order/Filter/AtTopBot/Disjoint.lean: showing AtTop and AtBot are disjoint
  • Order/Filter/AtTopBot/Tendsto.lean: basic limits of AtTop and AtBot
  • Order/Filter/AtTopBot/CompleteLattice.lean: results in a (conditionally) complete lattice
  • Order/Filter/AtTopBot/Finset.lean: results involving finite sets
  • Order/Filter/AtTopBot/Map.lean: results involving map/comap
  • Order/Filter/AtTopBot/Prod.lean: results involving product of filters
  • Order/Filter/AtTopBot/Basic.lean: remaining results (those depending on Order.Filter.Bases) The goal is to reduce the dependencies for Topology.Basic. The results are not too exciting for the file itself, but we do get some nice cleanups down the line.

Estimated changes

deleted theorem Filter.Ici_mem_atTop
deleted theorem Filter.Iic_mem_atBot
deleted theorem Filter.Iio_mem_atBot
deleted theorem Filter.Ioi_mem_atTop
deleted theorem Filter.OrderBot.atBot_eq
deleted theorem Filter.OrderTop.atTop_eq
deleted theorem Filter.Tendsto.prod_atBot
deleted theorem Filter.Tendsto.prod_atTop
deleted theorem Filter.Tendsto.subseq_mem
deleted def Filter.atBot
deleted theorem Filter.atBot_Iic_eq
deleted theorem Filter.atBot_Iio_eq
deleted theorem Filter.atBot_basis'
deleted theorem Filter.atBot_basis
deleted theorem Filter.atBot_basis_Iio'
deleted theorem Filter.atBot_basis_Iio
deleted theorem Filter.atBot_neBot
deleted theorem Filter.atBot_neBot_iff
deleted def Filter.atTop
deleted theorem Filter.atTop_Ici_eq
deleted theorem Filter.atTop_Ioi_eq
deleted theorem Filter.atTop_basis'
deleted theorem Filter.atTop_basis
deleted theorem Filter.atTop_basis_Ioi'
deleted theorem Filter.atTop_basis_Ioi
deleted theorem Filter.atTop_neBot
deleted theorem Filter.atTop_neBot_iff
deleted theorem Filter.eventually_atBot
deleted theorem Filter.eventually_atTop
deleted theorem Filter.frequently_atBot'
deleted theorem Filter.frequently_atBot
deleted theorem Filter.frequently_atTop'
deleted theorem Filter.frequently_atTop
deleted theorem Filter.high_scores
deleted theorem Filter.low_scores
deleted theorem Filter.map_atBot_eq
deleted theorem Filter.map_atBot_eq_of_gc
deleted theorem Filter.map_atTop_eq
deleted theorem Filter.map_atTop_eq_of_gc
deleted theorem Filter.map_val_Ici_atTop
deleted theorem Filter.map_val_Iic_atBot
deleted theorem Filter.map_val_Iio_atBot
deleted theorem Filter.map_val_Ioi_atTop
deleted theorem Filter.mem_atBot
deleted theorem Filter.mem_atBot_sets
deleted theorem Filter.mem_atTop
deleted theorem Filter.mem_atTop_sets
deleted theorem Filter.prod_map_atBot_eq
deleted theorem Filter.prod_map_atTop_eq
deleted theorem Filter.tendsto_Ici_atTop
deleted theorem Filter.tendsto_Iic_atBot
deleted theorem Filter.tendsto_Iio_atBot
deleted theorem Filter.tendsto_Ioi_atTop
deleted theorem Filter.tendsto_atBot'
deleted theorem Filter.tendsto_atBot
deleted theorem Filter.tendsto_atBot_mono
deleted theorem Filter.tendsto_atBot_pure
deleted theorem Filter.tendsto_atTop'
deleted theorem Filter.tendsto_atTop
deleted theorem Filter.tendsto_atTop_mono
deleted theorem Filter.tendsto_atTop_pure
deleted theorem IsBot.atBot_eq
deleted theorem IsTop.atTop_eq
deleted theorem Nat.map_cast_int_atTop
deleted theorem OrderIso.comap_atBot
deleted theorem OrderIso.comap_atTop
deleted theorem OrderIso.map_atBot
deleted theorem OrderIso.map_atTop
deleted theorem OrderIso.tendsto_atBot
deleted theorem OrderIso.tendsto_atTop
deleted theorem StrictMono.tendsto_atTop
added theorem Filter.atBot_Iic_eq
added theorem Filter.atBot_Iio_eq
added theorem Filter.atBot_basis'
added theorem Filter.atBot_basis
added theorem Filter.atBot_basis_Iio
added theorem Filter.atBot_neBot
added theorem Filter.atBot_neBot_iff
added theorem Filter.atTop_Ici_eq
added theorem Filter.atTop_Ioi_eq
added theorem Filter.atTop_basis'
added theorem Filter.atTop_basis
added theorem Filter.atTop_basis_Ioi
added theorem Filter.atTop_neBot
added theorem Filter.atTop_neBot_iff
added theorem Filter.high_scores
added theorem Filter.low_scores
added theorem Filter.map_atBot_eq
added theorem Filter.map_atTop_eq
added theorem Filter.mem_atBot_sets
added theorem Filter.mem_atTop_sets
added theorem Filter.tendsto_atBot'
added theorem Filter.tendsto_atTop'
added theorem Nat.map_cast_int_atTop