Commit 2025-08-13 00:55 59e4fba0

View on Github →

refactor: rename Rel to SetRel, restore the old Rel (#27447) Many users are confused that Rel no longer means what it used to. Since the design is not obvious (and the implementation is explicitly part of the interface thanks to abbrev), let's give it a name that makes the choice obvious. This then restores the old definition of Rel, as an abbrev; it's conceivable that many users were just using this as a shorthand, and this stops them being broken by #25587. Such users will of course be broken if they used the old API. This way, users bumping from 4.21.0 to 4.22.0 and using Rel only as a shorthand will not be broken. [#mathlib4 > Changing `Rel` to `Set (α × β)`, to help uniform spaces @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Changing.20.60Rel.60.20to.20.60Set.20.28.CE.B1.20.C3.97.20.CE.B2.29.60.2C.20to.20help.20uniform.20spaces/near/528531852)

Estimated changes

modified theorem Equiv.graph_inv
modified def Function.graph
modified theorem Function.graph_injective
deleted def Rel.cod
deleted theorem Rel.cod_empty
deleted theorem Rel.cod_inv
deleted theorem Rel.cod_mono
deleted theorem Rel.cod_univ
deleted def Rel.comp
deleted theorem Rel.comp_assoc
deleted theorem Rel.comp_empty
deleted theorem Rel.comp_id
deleted theorem Rel.comp_univ
deleted def Rel.core
deleted theorem Rel.core_comp
deleted theorem Rel.core_id
deleted theorem Rel.core_inter
deleted theorem Rel.core_mono
deleted theorem Rel.core_subset_core
deleted theorem Rel.core_union_subset
deleted theorem Rel.core_univ
deleted def Rel.dom
deleted theorem Rel.dom_empty
deleted theorem Rel.dom_inv
deleted theorem Rel.dom_mono
deleted theorem Rel.dom_univ
deleted theorem Rel.empty_comp
deleted theorem Rel.exists_graph_eq_iff
deleted theorem Rel.id_comp
deleted def Rel.image
deleted theorem Rel.image_comp
deleted theorem Rel.image_core_gc
deleted theorem Rel.image_empty_left
deleted theorem Rel.image_empty_right
deleted theorem Rel.image_id
deleted theorem Rel.image_inter_dom
deleted theorem Rel.image_inter_subset
deleted theorem Rel.image_inv
deleted theorem Rel.image_mono
deleted theorem Rel.image_subset_iff
deleted theorem Rel.image_subset_image
deleted theorem Rel.image_union
deleted theorem Rel.image_univ_left
deleted theorem Rel.image_univ_right
deleted def Rel.inv
deleted theorem Rel.inv_comp
deleted theorem Rel.inv_empty
deleted theorem Rel.inv_id
deleted theorem Rel.inv_inv
deleted theorem Rel.inv_mono
deleted theorem Rel.inv_univ
deleted theorem Rel.mem_cod
deleted theorem Rel.mem_comp
deleted theorem Rel.mem_core
deleted theorem Rel.mem_dom
deleted theorem Rel.mem_id
deleted theorem Rel.mem_image
deleted theorem Rel.mem_inv
deleted theorem Rel.mem_preimage
deleted def Rel.preimage
deleted theorem Rel.preimage_comp
deleted theorem Rel.preimage_empty_left
deleted theorem Rel.preimage_empty_right
deleted theorem Rel.preimage_id
deleted theorem Rel.preimage_inter_cod
deleted theorem Rel.preimage_inter_subset
deleted theorem Rel.preimage_inv
deleted theorem Rel.preimage_mono
deleted theorem Rel.preimage_union
deleted theorem Rel.preimage_univ_left
deleted theorem Rel.preimage_univ_right
deleted def Rel.restrictDomain
deleted theorem Rel.univ_comp
added def SetRel.cod
added theorem SetRel.cod_empty
added theorem SetRel.cod_inv
added theorem SetRel.cod_mono
added theorem SetRel.cod_univ
added def SetRel.comp
added theorem SetRel.comp_assoc
added theorem SetRel.comp_empty
added theorem SetRel.comp_id
added theorem SetRel.comp_univ
added def SetRel.core
added theorem SetRel.core_comp
added theorem SetRel.core_id
added theorem SetRel.core_inter
added theorem SetRel.core_mono
added theorem SetRel.core_univ
added def SetRel.dom
added theorem SetRel.dom_empty
added theorem SetRel.dom_inv
added theorem SetRel.dom_mono
added theorem SetRel.dom_univ
added theorem SetRel.empty_comp
added theorem SetRel.id_comp
added def SetRel.image
added theorem SetRel.image_comp
added theorem SetRel.image_core_gc
added theorem SetRel.image_id
added theorem SetRel.image_inter_dom
added theorem SetRel.image_inv
added theorem SetRel.image_mono
added theorem SetRel.image_union
added theorem SetRel.image_univ_left
added def SetRel.inv
added theorem SetRel.inv_comp
added theorem SetRel.inv_empty
added theorem SetRel.inv_id
added theorem SetRel.inv_inv
added theorem SetRel.inv_mono
added theorem SetRel.inv_univ
added theorem SetRel.mem_cod
added theorem SetRel.mem_comp
added theorem SetRel.mem_core
added theorem SetRel.mem_dom
added theorem SetRel.mem_id
added theorem SetRel.mem_image
added theorem SetRel.mem_inv
added theorem SetRel.mem_preimage
added def SetRel.preimage
added theorem SetRel.preimage_comp
added theorem SetRel.preimage_id
added theorem SetRel.preimage_inv
added theorem SetRel.preimage_mono
added theorem SetRel.preimage_union
added theorem SetRel.univ_comp
modified def Filter.RTendsto'
modified def Filter.RTendsto
modified theorem Filter.mem_rcomap'
modified theorem Filter.mem_rmap
modified def Filter.rcomap'
modified theorem Filter.rcomap'_compose
modified theorem Filter.rcomap'_rcomap'
modified theorem Filter.rcomap'_sets
modified def Filter.rcomap
modified theorem Filter.rcomap_compose
modified theorem Filter.rcomap_rcomap
modified theorem Filter.rcomap_sets
modified def Filter.rmap
modified theorem Filter.rmap_compose
modified theorem Filter.rmap_rmap
modified theorem Filter.rmap_sets
modified theorem Filter.rtendsto'_def
modified theorem Filter.rtendsto_def