Commit 2023-12-13 09:43 f7006a73

View on Github →

chore: rename LocalEquiv to PartialEquiv (#8984) The current name is misleading: there's no open set involved; it's just an equivalence between subsets of domain and target. zulip discussion PEquiv is similarly named: this is fine, as they're different designs for the same concept.

Estimated changes

deleted theorem Equiv.refl_toLocalEquiv
deleted theorem Equiv.symm_toLocalEquiv
deleted def Equiv.toLocalEquiv
deleted theorem Equiv.trans_toLocalEquiv
deleted def LocalEquiv.IsImage
deleted theorem LocalEquiv.coe_symm_mk
deleted theorem LocalEquiv.coe_trans
deleted theorem LocalEquiv.coe_trans_symm
deleted def LocalEquiv.copy
deleted theorem LocalEquiv.copy_eq
deleted theorem LocalEquiv.eq_symm_apply
deleted theorem LocalEquiv.invFun_as_coe
deleted theorem LocalEquiv.left_inv
deleted theorem LocalEquiv.map_source''
deleted theorem LocalEquiv.map_source
deleted theorem LocalEquiv.map_target
deleted def LocalEquiv.ofSet
deleted theorem LocalEquiv.ofSet_coe
deleted theorem LocalEquiv.ofSet_source
deleted theorem LocalEquiv.ofSet_symm
deleted theorem LocalEquiv.ofSet_target
deleted theorem LocalEquiv.pi_refl
deleted theorem LocalEquiv.pi_symm
deleted theorem LocalEquiv.pi_symm_apply
deleted theorem LocalEquiv.pi_trans
deleted def LocalEquiv.prod
deleted theorem LocalEquiv.prod_coe
deleted theorem LocalEquiv.prod_coe_symm
deleted theorem LocalEquiv.prod_source
deleted theorem LocalEquiv.prod_symm
deleted theorem LocalEquiv.prod_target
deleted theorem LocalEquiv.prod_trans
deleted theorem LocalEquiv.refl_coe
deleted theorem LocalEquiv.refl_prod_refl
deleted theorem LocalEquiv.refl_source
deleted theorem LocalEquiv.refl_symm
deleted theorem LocalEquiv.refl_target
deleted theorem LocalEquiv.refl_trans
deleted theorem LocalEquiv.restr_coe
deleted theorem LocalEquiv.restr_coe_symm
deleted theorem LocalEquiv.restr_source
deleted theorem LocalEquiv.restr_target
deleted theorem LocalEquiv.restr_trans
deleted theorem LocalEquiv.restr_univ
deleted theorem LocalEquiv.right_inv
deleted theorem LocalEquiv.symm_bijective
deleted theorem LocalEquiv.symm_mapsTo
deleted theorem LocalEquiv.symm_piecewise
deleted theorem LocalEquiv.symm_source
deleted theorem LocalEquiv.symm_symm
deleted theorem LocalEquiv.symm_target
deleted theorem LocalEquiv.trans_apply
deleted theorem LocalEquiv.trans_assoc
deleted theorem LocalEquiv.trans_ofSet
deleted theorem LocalEquiv.trans_refl
deleted theorem LocalEquiv.trans_source''
deleted theorem LocalEquiv.trans_source'
deleted theorem LocalEquiv.trans_source
deleted theorem LocalEquiv.trans_target''
deleted theorem LocalEquiv.trans_target'
deleted theorem LocalEquiv.trans_target
deleted structure LocalEquiv
added theorem PartialEquiv.coe_trans
added theorem PartialEquiv.copy_eq
added theorem PartialEquiv.left_inv
added theorem PartialEquiv.ofSet_coe
added theorem PartialEquiv.pi_refl
added theorem PartialEquiv.pi_symm
added theorem PartialEquiv.pi_trans
added theorem PartialEquiv.prod_coe
added theorem PartialEquiv.prod_symm
added theorem PartialEquiv.refl_coe
added theorem PartialEquiv.refl_symm
added theorem PartialEquiv.restr_coe
added theorem PartialEquiv.right_inv
added theorem PartialEquiv.symm_symm
added structure PartialEquiv