Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

feat(ring_theory/integral_domain): generalize card_fiber_eq_of_mem_range #17653

Open
wants to merge 23 commits into
base: master
Choose a base branch
from

Conversation

urkud
Copy link
Member

@urkud urkud commented Nov 20, 2022

  • Generalize card_fiber_eq_of_mem_range to homomorphisms from a group to a monoid.
  • Rename it to monoid_hom.card_fiber_eq_of_mem_range, use to_additive.

Open in Gitpod

…ange`

* Generalize `card_fiber_eq_of_mem_range` to homomorphisms from a
  group to a monoid.
* Rename it to `monoid_hom.card_fiber_eq_of_mem_range`, use
  `to_additive`.
@urkud urkud added awaiting-review The author would like community review of the PR t-algebra Algebra (groups, rings, fields etc) labels Nov 20, 2022
Comment on lines 136 to 138
@[to_additive] lemma monoid_hom.card_fiber_eq_of_mem_range {M} [monoid M] [decidable_eq M]
(f : G →* M) {x y : M} (hx : x ∈ set.range f) (hy : y ∈ set.range f) :
(univ.filter $ λ g, f g = x).card = (univ.filter $ λ g, f g = y).card :=
Copy link
Collaborator

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

We should probably make an equivalence f⁻¹ {x} ≃f.ker given x ∈ set.range f.

@urkud urkud added awaiting-author A reviewer has asked the author a question or requested changes and removed awaiting-review The author would like community review of the PR labels Nov 23, 2022
@kim-em kim-em added the too-late This PR was ready too late for inclusion in mathlib3 label Jul 16, 2023
@github-actions github-actions bot added the modifies-synchronized-file This PR touches a files that has already been ported to mathlib4, and may need a synchronization PR. label Feb 11, 2024
Sign up for free to subscribe to this conversation on GitHub. Already have an account? Sign in.
Labels
awaiting-author A reviewer has asked the author a question or requested changes modifies-synchronized-file This PR touches a files that has already been ported to mathlib4, and may need a synchronization PR. t-algebra Algebra (groups, rings, fields etc) too-late This PR was ready too late for inclusion in mathlib3
Projects
None yet
Development

Successfully merging this pull request may close these issues.

3 participants