Commit 2025-03-20 16:39 07d2b9ef

View on Github →

chore(Data/Set): split long file Function.lean (#23149) This PR splits the long file Data.Set.Function into a few chunks:

  • Data.Set.Function now focusses on lemmas for predicates such as EqOn, InjOn, MapsTo, ...
  • Data.Set.Piecewise is a new file for results on the definiton Set.piecewise.
  • Data.Set.Prod received some upstreamed results on graphOn and the vertical line test.
  • Data.Set.Restrict is a new file for the definition of Set.restrict and some basic results.

Estimated changes

deleted theorem Set.EqOn.piecewise_ite'
deleted theorem Set.EqOn.piecewise_ite
deleted theorem Set.MapsTo.coe_restrict
deleted theorem Set.MapsTo.piecewise_ite
deleted theorem Set.MapsTo.range_restrict
deleted theorem Set.MapsTo.restrict_inj
deleted theorem Set.apply_piecewise
deleted theorem Set.apply_piecewise₂
deleted def Set.codRestrict
deleted theorem Set.codRestrict_restrict
deleted theorem Set.eqOn_piecewise
deleted theorem Set.eq_restrict_iff
deleted theorem Set.fst_injOn_graph
deleted theorem Set.graphOn_comp
deleted theorem Set.graphOn_empty
deleted theorem Set.graphOn_eq_empty
deleted theorem Set.graphOn_inj
deleted theorem Set.graphOn_insert
deleted theorem Set.graphOn_nonempty
deleted theorem Set.graphOn_prod_graphOn
deleted theorem Set.graphOn_prod_prodMap
deleted theorem Set.graphOn_singleton
deleted theorem Set.graphOn_union
deleted theorem Set.graphOn_univ_eq_range
deleted theorem Set.image_fst_graphOn
deleted theorem Set.image_restrict
deleted theorem Set.image_snd_graphOn
deleted theorem Set.injOn_iff_injective
deleted theorem Set.injective_codRestrict
deleted theorem Set.le_piecewise
deleted theorem Set.mem_graphOn
deleted theorem Set.pi_piecewise
deleted theorem Set.piecewise_compl
deleted theorem Set.piecewise_empty
deleted theorem Set.piecewise_eqOn
deleted theorem Set.piecewise_eqOn_compl
deleted theorem Set.piecewise_eq_of_mem
deleted theorem Set.piecewise_insert
deleted theorem Set.piecewise_insert_self
deleted theorem Set.piecewise_le
deleted theorem Set.piecewise_mem_pi
deleted theorem Set.piecewise_mono
deleted theorem Set.piecewise_op
deleted theorem Set.piecewise_op₂
deleted theorem Set.piecewise_preimage
deleted theorem Set.piecewise_range_comp
deleted theorem Set.piecewise_same
deleted theorem Set.piecewise_singleton
deleted theorem Set.piecewise_univ
deleted theorem Set.range_extend
deleted theorem Set.range_extend_subset
deleted theorem Set.range_piecewise
deleted theorem Set.range_restrict
deleted def Set.restrict
deleted theorem Set.restrictPreimage_mk
deleted theorem Set.restrict_apply
deleted theorem Set.restrict_def
deleted theorem Set.restrict_dite
deleted theorem Set.restrict_dite_compl
deleted theorem Set.restrict_eq
deleted theorem Set.restrict_eq_iff
deleted theorem Set.restrict_extend_range
deleted theorem Set.restrict_ite
deleted theorem Set.restrict_ite_compl
deleted theorem Set.restrict_piecewise
deleted def Set.restrict₂
deleted theorem Set.restrict₂_def
deleted theorem Set.surjOn_iff_surjective
deleted theorem Set.univ_pi_piecewise
deleted theorem Set.val_codRestrict_apply
added theorem Set.EqOn.piecewise_ite
added theorem Set.apply_piecewise
added theorem Set.apply_piecewise₂
added theorem Set.eqOn_piecewise
added theorem Set.le_piecewise
added theorem Set.pi_piecewise
added theorem Set.piecewise_compl
added theorem Set.piecewise_empty
added theorem Set.piecewise_eqOn
added theorem Set.piecewise_insert
added theorem Set.piecewise_le
added theorem Set.piecewise_mem_pi
added theorem Set.piecewise_mono
added theorem Set.piecewise_op
added theorem Set.piecewise_op₂
added theorem Set.piecewise_preimage
added theorem Set.piecewise_same
added theorem Set.piecewise_univ
added theorem Set.range_piecewise
added theorem Set.univ_pi_piecewise
added def Set.codRestrict
added theorem Set.eq_restrict_iff
added theorem Set.image_restrict
added theorem Set.range_extend
added theorem Set.range_restrict
added def Set.restrict
added theorem Set.restrict_apply
added theorem Set.restrict_def
added theorem Set.restrict_dite
added theorem Set.restrict_eq
added theorem Set.restrict_eq_iff
added theorem Set.restrict_ite
added theorem Set.restrict_ite_compl
added theorem Set.restrict_piecewise
added def Set.restrict₂
added theorem Set.restrict₂_def