Commit 2021-02-22 14:12 120feb11
View on Github →refactor(order/filter,topology): review API (#6347)
Filters
- move old filter.map_comaptofilter.map_comap_of_mem;
- add a new filter.map_comapthat doesn't assumerange m ∈ fbut givesmap m (comap m f) = f ⊓ 𝓟 (range m)instead ofmap m (comap m f) = f;
- add filter.comap_le_comap_iff, use it to golf a couple of proofs;
- move some lemmas using filter.map_comap/filter.map_comap_of_memclosure to these lemmas;
- use function.injective minstead of∀ x y, m x = m y → x = yin some lemmas;
- drop filter.le_map_comap_of_surjective',filter.map_comap_of_surjective', andfilter.le_map_comap_of_surjective: the inequalities easily follow from equalities, andfilter.map_comap_of_surjective'is justfilter.map_comap_of_mem+filter.mem_sets_of_superset;
Topology
- add closed_embedding_subtype_coe,ennreal.open_embedding_coe;
- drop inducing_open,inducing_is_closed,embedding_open, andembedding_is_closedreplace them withinducing.is_open_mapandinducing.is_closed_map;
- move old inducing.map_nhds_eqtoinducing.map_nhds_of_mem, the newinducing.map_nhds_eqsaysmap f (𝓝 a) = 𝓝[range f] (f a);
- add inducing.is_closed_iff;
- move old embedding.map_nhds_eqtoembedding.map_nhds_of_mem, the newembedding.map_nhds_eqsaysmap f (𝓝 a) = 𝓝[range f] (f a);
- add open_embedding.map_nhds_eq;
- change signature of is_closed_induced_iffto match other similar lemmas;
- move old map_nhds_induced_eqtomap_nhds_induced_of_mem, the newmap_nhds_induced_eqgive𝓝[range f] (f a)instead of𝓝 (f a).