path
stringlengths
11
71
content
stringlengths
75
124k
Algebra\DirectSum\Algebra.lean
/- Copyright (c) 2021 Eric Wieser. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Eric Wieser -/ import Mathlib.Algebra.Algebra.Defs import Mathlib.Algebra.DirectSum.Module import Mathlib.Algebra.DirectSum.Ring /-! # Additively-graded algebra structures on `⨁ i, A i` This file provides `R`-algebra structures on external direct sums of `R`-modules. Recall that if `A i` are a family of `AddCommMonoid`s indexed by an `AddMonoid`, then an instance of `DirectSum.GMonoid A` is a multiplication `A i → A j → A (i + j)` giving `⨁ i, A i` the structure of a semiring. In this file, we introduce the `DirectSum.GAlgebra R A` class for the case where all `A i` are `R`-modules. This is the extra structure needed to promote `⨁ i, A i` to an `R`-algebra. ## Main definitions * `DirectSum.GAlgebra R A`, the typeclass. * `DirectSum.toAlgebra` extends `DirectSum.toSemiring` to produce an `AlgHom`. -/ universe uι uR uA uB variable {ι : Type uι} namespace DirectSum open DirectSum variable (R : Type uR) (A : ι → Type uA) {B : Type uB} variable [CommSemiring R] [∀ i, AddCommMonoid (A i)] [∀ i, Module R (A i)] variable [AddMonoid ι] [GSemiring A] section /-- A graded version of `Algebra`. An instance of `DirectSum.GAlgebra R A` endows `(⨁ i, A i)` with an `R`-algebra structure. -/ class GAlgebra where toFun : R →+ A 0 map_one : toFun 1 = GradedMonoid.GOne.one map_mul : ∀ r s, GradedMonoid.mk _ (toFun (r * s)) = .mk _ (GradedMonoid.GMul.mul (toFun r) (toFun s)) commutes : ∀ (r) (x : GradedMonoid A), .mk _ (toFun r) * x = x * .mk _ (toFun r) smul_def : ∀ (r) (x : GradedMonoid A), r • x = .mk _ (toFun r) * x end variable [Semiring B] [GAlgebra R A] [Algebra R B] instance _root_.GradedMonoid.smulCommClass_right : SMulCommClass R (GradedMonoid A) (GradedMonoid A) where smul_comm s x y := by dsimp rw [GAlgebra.smul_def, GAlgebra.smul_def, ← mul_assoc, GAlgebra.commutes, mul_assoc] instance _root_.GradedMonoid.isScalarTower_right : IsScalarTower R (GradedMonoid A) (GradedMonoid A) where smul_assoc s x y := by dsimp rw [GAlgebra.smul_def, GAlgebra.smul_def, ← mul_assoc] variable [DecidableEq ι] instance : Algebra R (⨁ i, A i) where toFun := (DirectSum.of A 0).comp GAlgebra.toFun map_zero' := AddMonoidHom.map_zero _ map_add' := AddMonoidHom.map_add _ map_one' := DFunLike.congr_arg (DirectSum.of A 0) GAlgebra.map_one map_mul' a b := by simp only [AddMonoidHom.comp_apply] rw [of_mul_of] apply DFinsupp.single_eq_of_sigma_eq (GAlgebra.map_mul a b) commutes' r x := by change AddMonoidHom.mul (DirectSum.of _ _ _) x = AddMonoidHom.mul.flip (DirectSum.of _ _ _) x apply DFunLike.congr_fun _ x ext i xi : 2 dsimp only [AddMonoidHom.comp_apply, AddMonoidHom.mul_apply, AddMonoidHom.flip_apply] rw [of_mul_of, of_mul_of] apply DFinsupp.single_eq_of_sigma_eq (GAlgebra.commutes r ⟨i, xi⟩) smul_def' r x := by change DistribMulAction.toAddMonoidHom _ r x = AddMonoidHom.mul (DirectSum.of _ _ _) x apply DFunLike.congr_fun _ x ext i xi : 2 dsimp only [AddMonoidHom.comp_apply, DistribMulAction.toAddMonoidHom_apply, AddMonoidHom.mul_apply] rw [DirectSum.of_mul_of, ← of_smul] apply DFinsupp.single_eq_of_sigma_eq (GAlgebra.smul_def r ⟨i, xi⟩) theorem algebraMap_apply (r : R) : algebraMap R (⨁ i, A i) r = DirectSum.of A 0 (GAlgebra.toFun r) := rfl theorem algebraMap_toAddMonoid_hom : ↑(algebraMap R (⨁ i, A i)) = (DirectSum.of A 0).comp (GAlgebra.toFun : R →+ A 0) := rfl /-- A family of `LinearMap`s preserving `DirectSum.GOne.one` and `DirectSum.GMul.mul` describes an `AlgHom` on `⨁ i, A i`. This is a stronger version of `DirectSum.toSemiring`. Of particular interest is the case when `A i` are bundled subojects, `f` is the family of coercions such as `Submodule.subtype (A i)`, and the `[GMonoid A]` structure originates from `DirectSum.GMonoid.ofAddSubmodules`, in which case the proofs about `GOne` and `GMul` can be discharged by `rfl`. -/ @[simps] def toAlgebra (f : ∀ i, A i →ₗ[R] B) (hone : f _ GradedMonoid.GOne.one = 1) (hmul : ∀ {i j} (ai : A i) (aj : A j), f _ (GradedMonoid.GMul.mul ai aj) = f _ ai * f _ aj) : (⨁ i, A i) →ₐ[R] B := { toSemiring (fun i => (f i).toAddMonoidHom) hone @hmul with toFun := toSemiring (fun i => (f i).toAddMonoidHom) hone @hmul commutes' := fun r => by show toModule R _ _ f (algebraMap R _ r) = _ rw [Algebra.algebraMap_eq_smul_one, Algebra.algebraMap_eq_smul_one, map_smul, one_def, ← lof_eq_of R, toModule_lof, hone] } /-- Two `AlgHom`s out of a direct sum are equal if they agree on the generators. See note [partially-applied ext lemmas]. -/ @[ext] theorem algHom_ext' ⦃f g : (⨁ i, A i) →ₐ[R] B⦄ (h : ∀ i, f.toLinearMap.comp (lof _ _ A i) = g.toLinearMap.comp (lof _ _ A i)) : f = g := AlgHom.toLinearMap_injective <| DirectSum.linearMap_ext _ h theorem algHom_ext ⦃f g : (⨁ i, A i) →ₐ[R] B⦄ (h : ∀ i x, f (of A i x) = g (of A i x)) : f = g := algHom_ext' R A fun i => LinearMap.ext <| h i /-- The piecewise multiplication from the `Mul` instance, as a bundled linear homomorphism. This is the graded version of `LinearMap.mul`, and the linear version of `DirectSum.gMulHom` -/ @[simps] def gMulLHom {i j} : A i →ₗ[R] A j →ₗ[R] A (i + j) where toFun a := { toFun := fun b => GradedMonoid.GMul.mul a b map_smul' := fun r x => by injection (smul_comm r (GradedMonoid.mk _ a) (GradedMonoid.mk _ x)).symm map_add' := GNonUnitalNonAssocSemiring.mul_add _ } map_smul' r x := LinearMap.ext fun y => by injection smul_assoc r (GradedMonoid.mk _ x) (GradedMonoid.mk _ y) map_add' _ _ := LinearMap.ext fun _ => GNonUnitalNonAssocSemiring.add_mul _ _ _ end DirectSum /-! ### Concrete instances -/ /-- A direct sum of copies of an `Algebra` inherits the algebra structure. -/ @[simps] instance Algebra.directSumGAlgebra {R A : Type*} [AddMonoid ι] [CommSemiring R] [Semiring A] [Algebra R A] : DirectSum.GAlgebra R fun _ : ι => A where toFun := (algebraMap R A).toAddMonoidHom map_one := (algebraMap R A).map_one map_mul a b := Sigma.ext (zero_add _).symm (heq_of_eq <| (algebraMap R A).map_mul a b) commutes := fun _ ⟨_, _⟩ => Sigma.ext ((zero_add _).trans (add_zero _).symm) (heq_of_eq <| Algebra.commutes _ _) smul_def := fun _ ⟨_, _⟩ => Sigma.ext (zero_add _).symm (heq_of_eq <| Algebra.smul_def _ _)
Algebra\DirectSum\Basic.lean
/- Copyright (c) 2019 Kenny Lau. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Kenny Lau -/ import Mathlib.Algebra.Group.Submonoid.Operations import Mathlib.Data.DFinsupp.Basic /-! # Direct sum This file defines the direct sum of abelian groups, indexed by a discrete type. ## Notation `⨁ i, β i` is the n-ary direct sum `DirectSum`. This notation is in the `DirectSum` locale, accessible after `open DirectSum`. ## References * https://en.wikipedia.org/wiki/Direct_sum -/ open Function universe u v w u₁ variable (ι : Type v) (β : ι → Type w) /-- `DirectSum ι β` is the direct sum of a family of additive commutative monoids `β i`. Note: `open DirectSum` will enable the notation `⨁ i, β i` for `DirectSum ι β`. -/ def DirectSum [∀ i, AddCommMonoid (β i)] : Type _ := -- Porting note: Failed to synthesize -- Π₀ i, β i deriving AddCommMonoid, Inhabited -- See https://github.com/leanprover-community/mathlib4/issues/5020 Π₀ i, β i -- Porting note (#10754): Added inhabited instance manually instance [∀ i, AddCommMonoid (β i)] : Inhabited (DirectSum ι β) := inferInstanceAs (Inhabited (Π₀ i, β i)) -- Porting note (#10754): Added addCommMonoid instance manually instance [∀ i, AddCommMonoid (β i)] : AddCommMonoid (DirectSum ι β) := inferInstanceAs (AddCommMonoid (Π₀ i, β i)) instance [∀ i, AddCommMonoid (β i)] : DFunLike (DirectSum ι β) _ fun i : ι => β i := inferInstanceAs (DFunLike (Π₀ i, β i) _ _) instance [∀ i, AddCommMonoid (β i)] : CoeFun (DirectSum ι β) fun _ => ∀ i : ι, β i := inferInstanceAs (CoeFun (Π₀ i, β i) fun _ => ∀ i : ι, β i) /-- `⨁ i, f i` is notation for `DirectSum _ f` and equals the direct sum of `fun i ↦ f i`. Taking the direct sum over multiple arguments is possible, e.g. `⨁ (i) (j), f i j`. -/ scoped[DirectSum] notation3 "⨁ "(...)", "r:(scoped f => DirectSum _ f) => r -- Porting note: The below recreates some of the lean3 notation, not fully yet -- section -- open Batteries.ExtendedBinder -- syntax (name := bigdirectsum) "⨁ " extBinders ", " term : term -- macro_rules (kind := bigdirectsum) -- | `(⨁ $_:ident, $y:ident → $z:ident) => `(DirectSum _ (fun $y ↦ $z)) -- | `(⨁ $x:ident, $p) => `(DirectSum _ (fun $x ↦ $p)) -- | `(⨁ $_:ident : $t:ident, $p) => `(DirectSum _ (fun $t ↦ $p)) -- | `(⨁ ($x:ident) ($y:ident), $p) => `(DirectSum _ (fun $x ↦ fun $y ↦ $p)) -- end instance [DecidableEq ι] [∀ i, AddCommMonoid (β i)] [∀ i, DecidableEq (β i)] : DecidableEq (DirectSum ι β) := inferInstanceAs <| DecidableEq (Π₀ i, β i) namespace DirectSum variable {ι} section AddCommGroup variable [∀ i, AddCommGroup (β i)] instance : AddCommGroup (DirectSum ι β) := inferInstanceAs (AddCommGroup (Π₀ i, β i)) variable {β} @[simp] theorem sub_apply (g₁ g₂ : ⨁ i, β i) (i : ι) : (g₁ - g₂) i = g₁ i - g₂ i := rfl end AddCommGroup variable [∀ i, AddCommMonoid (β i)] @[simp] theorem zero_apply (i : ι) : (0 : ⨁ i, β i) i = 0 := rfl variable {β} @[simp] theorem add_apply (g₁ g₂ : ⨁ i, β i) (i : ι) : (g₁ + g₂) i = g₁ i + g₂ i := rfl section DecidableEq variable [DecidableEq ι] variable (β) /-- `mk β s x` is the element of `⨁ i, β i` that is zero outside `s` and has coefficient `x i` for `i` in `s`. -/ def mk (s : Finset ι) : (∀ i : (↑s : Set ι), β i.1) →+ ⨁ i, β i where toFun := DFinsupp.mk s map_add' _ _ := DFinsupp.mk_add map_zero' := DFinsupp.mk_zero /-- `of i` is the natural inclusion map from `β i` to `⨁ i, β i`. -/ def of (i : ι) : β i →+ ⨁ i, β i := DFinsupp.singleAddHom β i variable {β} @[simp] theorem of_eq_same (i : ι) (x : β i) : (of _ i x) i = x := DFinsupp.single_eq_same theorem of_eq_of_ne (i j : ι) (x : β i) (h : i ≠ j) : (of _ i x) j = 0 := DFinsupp.single_eq_of_ne h lemma of_apply {i : ι} (j : ι) (x : β i) : of β i x j = if h : i = j then Eq.recOn h x else 0 := DFinsupp.single_apply theorem mk_apply_of_mem {s : Finset ι} {f : ∀ i : (↑s : Set ι), β i.val} {n : ι} (hn : n ∈ s) : mk β s f n = f ⟨n, hn⟩ := by dsimp only [Finset.coe_sort_coe, mk, AddMonoidHom.coe_mk, ZeroHom.coe_mk, DFinsupp.mk_apply] rw [dif_pos hn] theorem mk_apply_of_not_mem {s : Finset ι} {f : ∀ i : (↑s : Set ι), β i.val} {n : ι} (hn : n ∉ s) : mk β s f n = 0 := by dsimp only [Finset.coe_sort_coe, mk, AddMonoidHom.coe_mk, ZeroHom.coe_mk, DFinsupp.mk_apply] rw [dif_neg hn] @[simp] theorem support_zero [∀ (i : ι) (x : β i), Decidable (x ≠ 0)] : (0 : ⨁ i, β i).support = ∅ := DFinsupp.support_zero @[simp] theorem support_of [∀ (i : ι) (x : β i), Decidable (x ≠ 0)] (i : ι) (x : β i) (h : x ≠ 0) : (of _ i x).support = {i} := DFinsupp.support_single_ne_zero h theorem support_of_subset [∀ (i : ι) (x : β i), Decidable (x ≠ 0)] {i : ι} {b : β i} : (of _ i b).support ⊆ {i} := DFinsupp.support_single_subset theorem sum_support_of [∀ (i : ι) (x : β i), Decidable (x ≠ 0)] (x : ⨁ i, β i) : (∑ i ∈ x.support, of β i (x i)) = x := DFinsupp.sum_single theorem sum_univ_of [Fintype ι] (x : ⨁ i, β i) : ∑ i ∈ Finset.univ, of β i (x i) = x := by apply DFinsupp.ext (fun i ↦ ?_) rw [DFinsupp.finset_sum_apply] simp [of_apply] theorem mk_injective (s : Finset ι) : Function.Injective (mk β s) := DFinsupp.mk_injective s theorem of_injective (i : ι) : Function.Injective (of β i) := DFinsupp.single_injective @[elab_as_elim] protected theorem induction_on {C : (⨁ i, β i) → Prop} (x : ⨁ i, β i) (H_zero : C 0) (H_basic : ∀ (i : ι) (x : β i), C (of β i x)) (H_plus : ∀ x y, C x → C y → C (x + y)) : C x := by apply DFinsupp.induction x H_zero intro i b f h1 h2 ih solve_by_elim /-- If two additive homomorphisms from `⨁ i, β i` are equal on each `of β i y`, then they are equal. -/ theorem addHom_ext {γ : Type*} [AddMonoid γ] ⦃f g : (⨁ i, β i) →+ γ⦄ (H : ∀ (i : ι) (y : β i), f (of _ i y) = g (of _ i y)) : f = g := DFinsupp.addHom_ext H /-- If two additive homomorphisms from `⨁ i, β i` are equal on each `of β i y`, then they are equal. See note [partially-applied ext lemmas]. -/ @[ext high] theorem addHom_ext' {γ : Type*} [AddMonoid γ] ⦃f g : (⨁ i, β i) →+ γ⦄ (H : ∀ i : ι, f.comp (of _ i) = g.comp (of _ i)) : f = g := addHom_ext fun i => DFunLike.congr_fun <| H i variable {γ : Type u₁} [AddCommMonoid γ] section ToAddMonoid variable (φ : ∀ i, β i →+ γ) (ψ : (⨁ i, β i) →+ γ) -- Porting note: The elaborator is struggling with `liftAddHom`. Passing it `β` explicitly helps. -- This applies to roughly the remainder of the file. /-- `toAddMonoid φ` is the natural homomorphism from `⨁ i, β i` to `γ` induced by a family `φ` of homomorphisms `β i → γ`. -/ def toAddMonoid : (⨁ i, β i) →+ γ := DFinsupp.liftAddHom (β := β) φ @[simp] theorem toAddMonoid_of (i) (x : β i) : toAddMonoid φ (of β i x) = φ i x := DFinsupp.liftAddHom_apply_single φ i x theorem toAddMonoid.unique (f : ⨁ i, β i) : ψ f = toAddMonoid (fun i => ψ.comp (of β i)) f := by congr -- Porting note (#11041): `ext` applies addHom_ext' here, which isn't what we want. apply DFinsupp.addHom_ext' simp [toAddMonoid, of] lemma toAddMonoid_injective : Injective (toAddMonoid : (∀ i, β i →+ γ) → (⨁ i, β i) →+ γ) := DFinsupp.liftAddHom.injective @[simp] lemma toAddMonoid_inj {f g : ∀ i, β i →+ γ} : toAddMonoid f = toAddMonoid g ↔ f = g := toAddMonoid_injective.eq_iff end ToAddMonoid section FromAddMonoid /-- `fromAddMonoid φ` is the natural homomorphism from `γ` to `⨁ i, β i` induced by a family `φ` of homomorphisms `γ → β i`. Note that this is not an isomorphism. Not every homomorphism `γ →+ ⨁ i, β i` arises in this way. -/ def fromAddMonoid : (⨁ i, γ →+ β i) →+ γ →+ ⨁ i, β i := toAddMonoid fun i => AddMonoidHom.compHom (of β i) @[simp] theorem fromAddMonoid_of (i : ι) (f : γ →+ β i) : fromAddMonoid (of _ i f) = (of _ i).comp f := by rw [fromAddMonoid, toAddMonoid_of] rfl theorem fromAddMonoid_of_apply (i : ι) (f : γ →+ β i) (x : γ) : fromAddMonoid (of _ i f) x = of _ i (f x) := by rw [fromAddMonoid_of, AddMonoidHom.coe_comp, Function.comp] end FromAddMonoid variable (β) -- TODO: generalize this to remove the assumption `S ⊆ T`. /-- `setToSet β S T h` is the natural homomorphism `⨁ (i : S), β i → ⨁ (i : T), β i`, where `h : S ⊆ T`. -/ def setToSet (S T : Set ι) (H : S ⊆ T) : (⨁ i : S, β i) →+ ⨁ i : T, β i := toAddMonoid fun i => of (fun i : Subtype T => β i) ⟨↑i, H i.2⟩ end DecidableEq instance unique [∀ i, Subsingleton (β i)] : Unique (⨁ i, β i) := DFinsupp.unique /-- A direct sum over an empty type is trivial. -/ instance uniqueOfIsEmpty [IsEmpty ι] : Unique (⨁ i, β i) := DFinsupp.uniqueOfIsEmpty /-- The natural equivalence between `⨁ _ : ι, M` and `M` when `Unique ι`. -/ protected def id (M : Type v) (ι : Type* := PUnit) [AddCommMonoid M] [Unique ι] : (⨁ _ : ι, M) ≃+ M := { DirectSum.toAddMonoid fun _ => AddMonoidHom.id M with toFun := DirectSum.toAddMonoid fun _ => AddMonoidHom.id M invFun := of (fun _ => M) default left_inv := fun x => DirectSum.induction_on x (by rw [AddMonoidHom.map_zero, AddMonoidHom.map_zero]) (fun p x => by rw [Unique.default_eq p, toAddMonoid_of]; rfl) fun x y ihx ihy => by rw [AddMonoidHom.map_add, AddMonoidHom.map_add, ihx, ihy] right_inv := fun x => toAddMonoid_of _ _ _ } section CongrLeft variable {κ : Type*} /-- Reindexing terms of a direct sum. -/ def equivCongrLeft (h : ι ≃ κ) : (⨁ i, β i) ≃+ ⨁ k, β (h.symm k) := { DFinsupp.equivCongrLeft h with map_add' := DFinsupp.comapDomain'_add _ h.right_inv} @[simp] theorem equivCongrLeft_apply (h : ι ≃ κ) (f : ⨁ i, β i) (k : κ) : equivCongrLeft h f k = f (h.symm k) := by exact DFinsupp.comapDomain'_apply _ h.right_inv _ _ end CongrLeft section Option variable {α : Option ι → Type w} [∀ i, AddCommMonoid (α i)] /-- Isomorphism obtained by separating the term of index `none` of a direct sum over `Option ι`. -/ @[simps!] noncomputable def addEquivProdDirectSum : (⨁ i, α i) ≃+ α none × ⨁ i, α (some i) := { DFinsupp.equivProdDFinsupp with map_add' := DFinsupp.equivProdDFinsupp_add } end Option section Sigma variable [DecidableEq ι] {α : ι → Type u} {δ : ∀ i, α i → Type w} [∀ i j, AddCommMonoid (δ i j)] /-- The natural map between `⨁ (i : Σ i, α i), δ i.1 i.2` and `⨁ i (j : α i), δ i j`. -/ def sigmaCurry : (⨁ i : Σ _i, _, δ i.1 i.2) →+ ⨁ (i) (j), δ i j where toFun := DFinsupp.sigmaCurry (δ := δ) map_zero' := DFinsupp.sigmaCurry_zero map_add' f g := DFinsupp.sigmaCurry_add f g @[simp] theorem sigmaCurry_apply (f : ⨁ i : Σ _i, _, δ i.1 i.2) (i : ι) (j : α i) : sigmaCurry f i j = f ⟨i, j⟩ := DFinsupp.sigmaCurry_apply (δ := δ) _ i j /-- The natural map between `⨁ i (j : α i), δ i j` and `Π₀ (i : Σ i, α i), δ i.1 i.2`, inverse of `curry`. -/ def sigmaUncurry : (⨁ (i) (j), δ i j) →+ ⨁ i : Σ _i, _, δ i.1 i.2 where toFun := DFinsupp.sigmaUncurry map_zero' := DFinsupp.sigmaUncurry_zero map_add' := DFinsupp.sigmaUncurry_add @[simp] theorem sigmaUncurry_apply (f : ⨁ (i) (j), δ i j) (i : ι) (j : α i) : sigmaUncurry f ⟨i, j⟩ = f i j := DFinsupp.sigmaUncurry_apply f i j /-- The natural map between `⨁ (i : Σ i, α i), δ i.1 i.2` and `⨁ i (j : α i), δ i j`. -/ def sigmaCurryEquiv : (⨁ i : Σ _i, _, δ i.1 i.2) ≃+ ⨁ (i) (j), δ i j := { sigmaCurry, DFinsupp.sigmaCurryEquiv with } end Sigma /-- The canonical embedding from `⨁ i, A i` to `M` where `A` is a collection of `AddSubmonoid M` indexed by `ι`. When `S = Submodule _ M`, this is available as a `LinearMap`, `DirectSum.coe_linearMap`. -/ protected def coeAddMonoidHom {M S : Type*} [DecidableEq ι] [AddCommMonoid M] [SetLike S M] [AddSubmonoidClass S M] (A : ι → S) : (⨁ i, A i) →+ M := toAddMonoid fun i => AddSubmonoidClass.subtype (A i) theorem coeAddMonoidHom_eq_dfinsupp_sum [DecidableEq ι] {M S : Type*} [DecidableEq M] [AddCommMonoid M] [SetLike S M] [AddSubmonoidClass S M] (A : ι → S) (x : DirectSum ι fun i => A i) : DirectSum.coeAddMonoidHom A x = DFinsupp.sum x fun i => (fun x : A i => ↑x) := by simp only [DirectSum.coeAddMonoidHom, toAddMonoid, DFinsupp.liftAddHom, AddEquiv.coe_mk, Equiv.coe_fn_mk] exact DFinsupp.sumAddHom_apply _ x @[simp] theorem coeAddMonoidHom_of {M S : Type*} [DecidableEq ι] [AddCommMonoid M] [SetLike S M] [AddSubmonoidClass S M] (A : ι → S) (i : ι) (x : A i) : DirectSum.coeAddMonoidHom A (of (fun i => A i) i x) = x := toAddMonoid_of _ _ _ theorem coe_of_apply {M S : Type*} [DecidableEq ι] [AddCommMonoid M] [SetLike S M] [AddSubmonoidClass S M] {A : ι → S} (i j : ι) (x : A i) : (of (fun i ↦ {x // x ∈ A i}) i x j : M) = if i = j then x else 0 := by obtain rfl | h := Decidable.eq_or_ne i j · rw [DirectSum.of_eq_same, if_pos rfl] · rw [DirectSum.of_eq_of_ne _ _ _ h, if_neg h, ZeroMemClass.coe_zero, ZeroMemClass.coe_zero] /-- The `DirectSum` formed by a collection of additive submonoids (or subgroups, or submodules) of `M` is said to be internal if the canonical map `(⨁ i, A i) →+ M` is bijective. For the alternate statement in terms of independence and spanning, see `DirectSum.subgroup_isInternal_iff_independent_and_supr_eq_top` and `DirectSum.isInternal_submodule_iff_independent_and_iSup_eq_top`. -/ def IsInternal {M S : Type*} [DecidableEq ι] [AddCommMonoid M] [SetLike S M] [AddSubmonoidClass S M] (A : ι → S) : Prop := Function.Bijective (DirectSum.coeAddMonoidHom A) theorem IsInternal.addSubmonoid_iSup_eq_top {M : Type*} [DecidableEq ι] [AddCommMonoid M] (A : ι → AddSubmonoid M) (h : IsInternal A) : iSup A = ⊤ := by rw [AddSubmonoid.iSup_eq_mrange_dfinsupp_sumAddHom, AddMonoidHom.mrange_top_iff_surjective] exact Function.Bijective.surjective h variable {M S : Type*} [AddCommMonoid M] [SetLike S M] [AddSubmonoidClass S M] theorem support_subset [DecidableEq ι] [DecidableEq M] (A : ι → S) (x : DirectSum ι fun i => A i) : (Function.support fun i => (x i : M)) ⊆ ↑(DFinsupp.support x) := by intro m simp only [Function.mem_support, Finset.mem_coe, DFinsupp.mem_support_toFun, not_imp_not, ZeroMemClass.coe_eq_zero, imp_self] theorem finite_support (A : ι → S) (x : DirectSum ι fun i => A i) : (Function.support fun i => (x i : M)).Finite := by classical exact (DFinsupp.support x).finite_toSet.subset (DirectSum.support_subset _ x) end DirectSum
Algebra\DirectSum\Decomposition.lean
/- Copyright (c) 2022 Eric Wieser. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Eric Wieser, Jujian Zhang -/ import Mathlib.Algebra.DirectSum.Module import Mathlib.Algebra.Module.Submodule.Basic /-! # Decompositions of additive monoids, groups, and modules into direct sums ## Main definitions * `DirectSum.Decomposition ℳ`: A typeclass to provide a constructive decomposition from an additive monoid `M` into a family of additive submonoids `ℳ` * `DirectSum.decompose ℳ`: The canonical equivalence provided by the above typeclass ## Main statements * `DirectSum.Decomposition.isInternal`: The link to `DirectSum.IsInternal`. ## Implementation details As we want to talk about different types of decomposition (additive monoids, modules, rings, ...), we choose to avoid heavily bundling `DirectSum.decompose`, instead making copies for the `AddEquiv`, `LinearEquiv`, etc. This means we have to repeat statements that follow from these bundled homs, but means we don't have to repeat statements for different types of decomposition. -/ variable {ι R M σ : Type*} open DirectSum namespace DirectSum section AddCommMonoid variable [DecidableEq ι] [AddCommMonoid M] variable [SetLike σ M] [AddSubmonoidClass σ M] (ℳ : ι → σ) /-- A decomposition is an equivalence between an additive monoid `M` and a direct sum of additive submonoids `ℳ i` of that `M`, such that the "recomposition" is canonical. This definition also works for additive groups and modules. This is a version of `DirectSum.IsInternal` which comes with a constructive inverse to the canonical "recomposition" rather than just a proof that the "recomposition" is bijective. Often it is easier to construct a term of this type via `Decomposition.ofAddHom` or `Decomposition.ofLinearMap`. -/ class Decomposition where decompose' : M → ⨁ i, ℳ i left_inv : Function.LeftInverse (DirectSum.coeAddMonoidHom ℳ) decompose' right_inv : Function.RightInverse (DirectSum.coeAddMonoidHom ℳ) decompose' /-- `DirectSum.Decomposition` instances, while carrying data, are always equal. -/ instance : Subsingleton (Decomposition ℳ) := ⟨fun x y ↦ by cases' x with x xl xr cases' y with y yl yr congr exact Function.LeftInverse.eq_rightInverse xr yl⟩ /-- A convenience method to construct a decomposition from an `AddMonoidHom`, such that the proofs of left and right inverse can be constructed via `ext`. -/ abbrev Decomposition.ofAddHom (decompose : M →+ ⨁ i, ℳ i) (h_left_inv : (DirectSum.coeAddMonoidHom ℳ).comp decompose = .id _) (h_right_inv : decompose.comp (DirectSum.coeAddMonoidHom ℳ) = .id _) : Decomposition ℳ where decompose' := decompose left_inv := DFunLike.congr_fun h_left_inv right_inv := DFunLike.congr_fun h_right_inv /-- Noncomputably conjure a decomposition instance from a `DirectSum.IsInternal` proof. -/ noncomputable def IsInternal.chooseDecomposition (h : IsInternal ℳ) : DirectSum.Decomposition ℳ where decompose' := (Equiv.ofBijective _ h).symm left_inv := (Equiv.ofBijective _ h).right_inv right_inv := (Equiv.ofBijective _ h).left_inv variable [Decomposition ℳ] protected theorem Decomposition.isInternal : DirectSum.IsInternal ℳ := ⟨Decomposition.right_inv.injective, Decomposition.left_inv.surjective⟩ /-- If `M` is graded by `ι` with degree `i` component `ℳ i`, then it is isomorphic as to a direct sum of components. This is the canonical spelling of the `decompose'` field. -/ def decompose : M ≃ ⨁ i, ℳ i where toFun := Decomposition.decompose' invFun := DirectSum.coeAddMonoidHom ℳ left_inv := Decomposition.left_inv right_inv := Decomposition.right_inv protected theorem Decomposition.inductionOn {p : M → Prop} (h_zero : p 0) (h_homogeneous : ∀ {i} (m : ℳ i), p (m : M)) (h_add : ∀ m m' : M, p m → p m' → p (m + m')) : ∀ m, p m := by let ℳ' : ι → AddSubmonoid M := fun i ↦ (⟨⟨ℳ i, fun x y ↦ AddMemClass.add_mem x y⟩, (ZeroMemClass.zero_mem _)⟩ : AddSubmonoid M) haveI t : DirectSum.Decomposition ℳ' := { decompose' := DirectSum.decompose ℳ left_inv := fun _ ↦ (decompose ℳ).left_inv _ right_inv := fun _ ↦ (decompose ℳ).right_inv _ } have mem : ∀ m, m ∈ iSup ℳ' := fun _m ↦ (DirectSum.IsInternal.addSubmonoid_iSup_eq_top ℳ' (Decomposition.isInternal ℳ')).symm ▸ trivial -- Porting note: needs to use @ even though no implicit argument is provided exact fun m ↦ @AddSubmonoid.iSup_induction _ _ _ ℳ' _ _ (mem m) (fun i m h ↦ h_homogeneous ⟨m, h⟩) h_zero h_add -- exact fun m ↦ -- AddSubmonoid.iSup_induction ℳ' (mem m) (fun i m h ↦ h_homogeneous ⟨m, h⟩) h_zero h_add @[simp] theorem Decomposition.decompose'_eq : Decomposition.decompose' = decompose ℳ := rfl @[simp] theorem decompose_symm_of {i : ι} (x : ℳ i) : (decompose ℳ).symm (DirectSum.of _ i x) = x := DirectSum.coeAddMonoidHom_of ℳ _ _ @[simp] theorem decompose_coe {i : ι} (x : ℳ i) : decompose ℳ (x : M) = DirectSum.of _ i x := by rw [← decompose_symm_of _, Equiv.apply_symm_apply] theorem decompose_of_mem {x : M} {i : ι} (hx : x ∈ ℳ i) : decompose ℳ x = DirectSum.of (fun i ↦ ℳ i) i ⟨x, hx⟩ := decompose_coe _ ⟨x, hx⟩ theorem decompose_of_mem_same {x : M} {i : ι} (hx : x ∈ ℳ i) : (decompose ℳ x i : M) = x := by rw [decompose_of_mem _ hx, DirectSum.of_eq_same, Subtype.coe_mk] theorem decompose_of_mem_ne {x : M} {i j : ι} (hx : x ∈ ℳ i) (hij : i ≠ j) : (decompose ℳ x j : M) = 0 := by rw [decompose_of_mem _ hx, DirectSum.of_eq_of_ne _ _ _ hij, ZeroMemClass.coe_zero] theorem degree_eq_of_mem_mem {x : M} {i j : ι} (hxi : x ∈ ℳ i) (hxj : x ∈ ℳ j) (hx : x ≠ 0) : i = j := by contrapose! hx; rw [← decompose_of_mem_same ℳ hxj, decompose_of_mem_ne ℳ hxi hx] /-- If `M` is graded by `ι` with degree `i` component `ℳ i`, then it is isomorphic as an additive monoid to a direct sum of components. -/ -- Porting note: deleted [simps] and added the corresponding lemmas by hand def decomposeAddEquiv : M ≃+ ⨁ i, ℳ i := AddEquiv.symm { (decompose ℳ).symm with map_add' := map_add (DirectSum.coeAddMonoidHom ℳ) } @[simp] lemma decomposeAddEquiv_apply (a : M) : decomposeAddEquiv ℳ a = decompose ℳ a := rfl @[simp] lemma decomposeAddEquiv_symm_apply (a : ⨁ i, ℳ i) : (decomposeAddEquiv ℳ).symm a = (decompose ℳ).symm a := rfl @[simp] theorem decompose_zero : decompose ℳ (0 : M) = 0 := map_zero (decomposeAddEquiv ℳ) @[simp] theorem decompose_symm_zero : (decompose ℳ).symm 0 = (0 : M) := map_zero (decomposeAddEquiv ℳ).symm @[simp] theorem decompose_add (x y : M) : decompose ℳ (x + y) = decompose ℳ x + decompose ℳ y := map_add (decomposeAddEquiv ℳ) x y @[simp] theorem decompose_symm_add (x y : ⨁ i, ℳ i) : (decompose ℳ).symm (x + y) = (decompose ℳ).symm x + (decompose ℳ).symm y := map_add (decomposeAddEquiv ℳ).symm x y @[simp] theorem decompose_sum {ι'} (s : Finset ι') (f : ι' → M) : decompose ℳ (∑ i ∈ s, f i) = ∑ i ∈ s, decompose ℳ (f i) := map_sum (decomposeAddEquiv ℳ) f s @[simp] theorem decompose_symm_sum {ι'} (s : Finset ι') (f : ι' → ⨁ i, ℳ i) : (decompose ℳ).symm (∑ i ∈ s, f i) = ∑ i ∈ s, (decompose ℳ).symm (f i) := map_sum (decomposeAddEquiv ℳ).symm f s theorem sum_support_decompose [∀ (i) (x : ℳ i), Decidable (x ≠ 0)] (r : M) : (∑ i ∈ (decompose ℳ r).support, (decompose ℳ r i : M)) = r := by conv_rhs => rw [← (decompose ℳ).symm_apply_apply r, ← sum_support_of (decompose ℳ r)] rw [decompose_symm_sum] simp_rw [decompose_symm_of] end AddCommMonoid /-- The `-` in the statements below doesn't resolve without this line. This seems to be a problem of synthesized vs inferred typeclasses disagreeing. If we replace the statement of `decompose_neg` with `@Eq (⨁ i, ℳ i) (decompose ℳ (-x)) (-decompose ℳ x)` instead of `decompose ℳ (-x) = -decompose ℳ x`, which forces the typeclasses needed by `⨁ i, ℳ i` to be found by unification rather than synthesis, then everything works fine without this instance. -/ instance addCommGroupSetLike [AddCommGroup M] [SetLike σ M] [AddSubgroupClass σ M] (ℳ : ι → σ) : AddCommGroup (⨁ i, ℳ i) := by infer_instance section AddCommGroup variable [DecidableEq ι] [AddCommGroup M] variable [SetLike σ M] [AddSubgroupClass σ M] (ℳ : ι → σ) variable [Decomposition ℳ] @[simp] theorem decompose_neg (x : M) : decompose ℳ (-x) = -decompose ℳ x := map_neg (decomposeAddEquiv ℳ) x @[simp] theorem decompose_symm_neg (x : ⨁ i, ℳ i) : (decompose ℳ).symm (-x) = -(decompose ℳ).symm x := map_neg (decomposeAddEquiv ℳ).symm x @[simp] theorem decompose_sub (x y : M) : decompose ℳ (x - y) = decompose ℳ x - decompose ℳ y := map_sub (decomposeAddEquiv ℳ) x y @[simp] theorem decompose_symm_sub (x y : ⨁ i, ℳ i) : (decompose ℳ).symm (x - y) = (decompose ℳ).symm x - (decompose ℳ).symm y := map_sub (decomposeAddEquiv ℳ).symm x y end AddCommGroup section Module variable [DecidableEq ι] [Semiring R] [AddCommMonoid M] [Module R M] variable (ℳ : ι → Submodule R M) /-- A convenience method to construct a decomposition from an `LinearMap`, such that the proofs of left and right inverse can be constructed via `ext`. -/ abbrev Decomposition.ofLinearMap (decompose : M →ₗ[R] ⨁ i, ℳ i) (h_left_inv : DirectSum.coeLinearMap ℳ ∘ₗ decompose = .id) (h_right_inv : decompose ∘ₗ DirectSum.coeLinearMap ℳ = .id) : Decomposition ℳ where decompose' := decompose left_inv := DFunLike.congr_fun h_left_inv right_inv := DFunLike.congr_fun h_right_inv variable [Decomposition ℳ] /-- If `M` is graded by `ι` with degree `i` component `ℳ i`, then it is isomorphic as a module to a direct sum of components. -/ def decomposeLinearEquiv : M ≃ₗ[R] ⨁ i, ℳ i := LinearEquiv.symm { (decomposeAddEquiv ℳ).symm with map_smul' := map_smul (DirectSum.coeLinearMap ℳ) } @[simp] theorem decomposeLinearEquiv_apply (m : M) : decomposeLinearEquiv ℳ m = decompose ℳ m := rfl @[simp] theorem decomposeLinearEquiv_symm_apply (m : ⨁ i, ℳ i) : (decomposeLinearEquiv ℳ).symm m = (decompose ℳ).symm m := rfl @[simp] theorem decompose_smul (r : R) (x : M) : decompose ℳ (r • x) = r • decompose ℳ x := map_smul (decomposeLinearEquiv ℳ) r x @[simp] theorem decomposeLinearEquiv_symm_comp_lof (i : ι) : (decomposeLinearEquiv ℳ).symm ∘ₗ lof R ι (ℳ ·) i = (ℳ i).subtype := LinearMap.ext <| decompose_symm_of _ /-- Two linear maps from a module with a decomposition agree if they agree on every piece. Note this cannot be `@[ext]` as `ℳ` cannot be inferred. -/ theorem decompose_lhom_ext {N} [AddCommMonoid N] [Module R N] ⦃f g : M →ₗ[R] N⦄ (h : ∀ i, f ∘ₗ (ℳ i).subtype = g ∘ₗ (ℳ i).subtype) : f = g := LinearMap.ext <| (decomposeLinearEquiv ℳ).symm.surjective.forall.mpr <| suffices f ∘ₗ (decomposeLinearEquiv ℳ).symm = (g ∘ₗ (decomposeLinearEquiv ℳ).symm : (⨁ i, ℳ i) →ₗ[R] N) from DFunLike.congr_fun this linearMap_ext _ fun i => by simp_rw [LinearMap.comp_assoc, decomposeLinearEquiv_symm_comp_lof ℳ i, h] end Module end DirectSum
Algebra\DirectSum\Finsupp.lean
/- Copyright (c) 2019 Johannes Hölzl. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Johannes Hölzl -/ import Mathlib.Algebra.DirectSum.Module import Mathlib.Data.Finsupp.ToDFinsupp /-! # Results on direct sums and finitely supported functions. 1. The linear equivalence between finitely supported functions `ι →₀ M` and the direct sum of copies of `M` indexed by `ι`. -/ universe u v w noncomputable section open DirectSum open LinearMap Submodule variable {R : Type u} {M : Type v} [Semiring R] [AddCommMonoid M] [Module R M] section finsuppLequivDirectSum variable (R M) (ι : Type*) [DecidableEq ι] /-- The finitely supported functions `ι →₀ M` are in linear equivalence with the direct sum of copies of M indexed by ι. -/ def finsuppLEquivDirectSum : (ι →₀ M) ≃ₗ[R] ⨁ _ : ι, M := haveI : ∀ m : M, Decidable (m ≠ 0) := Classical.decPred _ finsuppLequivDFinsupp R @[simp] theorem finsuppLEquivDirectSum_single (i : ι) (m : M) : finsuppLEquivDirectSum R M ι (Finsupp.single i m) = DirectSum.lof R ι _ i m := Finsupp.toDFinsupp_single i m @[simp] theorem finsuppLEquivDirectSum_symm_lof (i : ι) (m : M) : (finsuppLEquivDirectSum R M ι).symm (DirectSum.lof R ι _ i m) = Finsupp.single i m := letI : ∀ m : M, Decidable (m ≠ 0) := Classical.decPred _ DFinsupp.toFinsupp_single i m end finsuppLequivDirectSum
Algebra\DirectSum\Internal.lean
/- Copyright (c) 2021 Eric Wieser. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Eric Wieser, Kevin Buzzard, Jujian Zhang, Fangming Li -/ import Mathlib.Algebra.Algebra.Operations import Mathlib.Algebra.Algebra.Subalgebra.Basic import Mathlib.Algebra.DirectSum.Algebra /-! # Internally graded rings and algebras This module provides `DirectSum.GSemiring` and `DirectSum.GCommSemiring` instances for a collection of subobjects `A` when a `SetLike.GradedMonoid` instance is available: * `SetLike.gnonUnitalNonAssocSemiring` * `SetLike.gsemiring` * `SetLike.gcommSemiring` With these instances in place, it provides the bundled canonical maps out of a direct sum of subobjects into their carrier type: * `DirectSum.coeRingHom` (a `RingHom` version of `DirectSum.coeAddMonoidHom`) * `DirectSum.coeAlgHom` (an `AlgHom` version of `DirectSum.coeLinearMap`) Strictly the definitions in this file are not sufficient to fully define an "internal" direct sum; to represent this case, `(h : DirectSum.IsInternal A) [SetLike.GradedMonoid A]` is needed. In the future there will likely be a data-carrying, constructive, typeclass version of `DirectSum.IsInternal` for providing an explicit decomposition function. When `CompleteLattice.Independent (Set.range A)` (a weaker condition than `DirectSum.IsInternal A`), these provide a grading of `⨆ i, A i`, and the mapping `⨁ i, A i →+ ⨆ i, A i` can be obtained as `DirectSum.toAddMonoid (fun i ↦ AddSubmonoid.inclusion <| le_iSup A i)`. This file also provides some extra structure on `A 0`, namely: * `SetLike.GradeZero.subsemiring`, which leads to * `SetLike.GradeZero.instSemiring` * `SetLike.GradeZero.instCommSemiring` * `SetLike.GradeZero.subring`, which leads to * `SetLike.GradeZero.instRing` * `SetLike.GradeZero.instCommRing` * `SetLike.GradeZero.subalgebra`, which leads to * `SetLike.GradeZero.instAlgebra` ## Tags internally graded ring -/ open DirectSum variable {ι : Type*} {σ S R : Type*} instance AddCommMonoid.ofSubmonoidOnSemiring [Semiring R] [SetLike σ R] [AddSubmonoidClass σ R] (A : ι → σ) : ∀ i, AddCommMonoid (A i) := fun i => by infer_instance instance AddCommGroup.ofSubgroupOnRing [Ring R] [SetLike σ R] [AddSubgroupClass σ R] (A : ι → σ) : ∀ i, AddCommGroup (A i) := fun i => by infer_instance theorem SetLike.algebraMap_mem_graded [Zero ι] [CommSemiring S] [Semiring R] [Algebra S R] (A : ι → Submodule S R) [SetLike.GradedOne A] (s : S) : algebraMap S R s ∈ A 0 := by rw [Algebra.algebraMap_eq_smul_one] exact (A 0).smul_mem s <| SetLike.one_mem_graded _ theorem SetLike.natCast_mem_graded [Zero ι] [AddMonoidWithOne R] [SetLike σ R] [AddSubmonoidClass σ R] (A : ι → σ) [SetLike.GradedOne A] (n : ℕ) : (n : R) ∈ A 0 := by induction' n with _ n_ih · rw [Nat.cast_zero] exact zero_mem (A 0) · rw [Nat.cast_succ] exact add_mem n_ih (SetLike.one_mem_graded _) @[deprecated (since := "2024-04-17")] alias SetLike.nat_cast_mem_graded := SetLike.natCast_mem_graded theorem SetLike.intCast_mem_graded [Zero ι] [AddGroupWithOne R] [SetLike σ R] [AddSubgroupClass σ R] (A : ι → σ) [SetLike.GradedOne A] (z : ℤ) : (z : R) ∈ A 0 := by induction z · rw [Int.ofNat_eq_coe, Int.cast_natCast] exact SetLike.natCast_mem_graded _ _ · rw [Int.cast_negSucc] exact neg_mem (SetLike.natCast_mem_graded _ _) @[deprecated (since := "2024-04-17")] alias SetLike.int_cast_mem_graded := SetLike.intCast_mem_graded section DirectSum variable [DecidableEq ι] /-! #### From `AddSubmonoid`s and `AddSubgroup`s -/ namespace SetLike /-- Build a `DirectSum.GNonUnitalNonAssocSemiring` instance for a collection of additive submonoids. -/ instance gnonUnitalNonAssocSemiring [Add ι] [NonUnitalNonAssocSemiring R] [SetLike σ R] [AddSubmonoidClass σ R] (A : ι → σ) [SetLike.GradedMul A] : DirectSum.GNonUnitalNonAssocSemiring fun i => A i := { SetLike.gMul A with mul_zero := fun _ => Subtype.ext (mul_zero _) zero_mul := fun _ => Subtype.ext (zero_mul _) mul_add := fun _ _ _ => Subtype.ext (mul_add _ _ _) add_mul := fun _ _ _ => Subtype.ext (add_mul _ _ _) } /-- Build a `DirectSum.GSemiring` instance for a collection of additive submonoids. -/ instance gsemiring [AddMonoid ι] [Semiring R] [SetLike σ R] [AddSubmonoidClass σ R] (A : ι → σ) [SetLike.GradedMonoid A] : DirectSum.GSemiring fun i => A i := { SetLike.gMonoid A with mul_zero := fun _ => Subtype.ext (mul_zero _) zero_mul := fun _ => Subtype.ext (zero_mul _) mul_add := fun _ _ _ => Subtype.ext (mul_add _ _ _) add_mul := fun _ _ _ => Subtype.ext (add_mul _ _ _) natCast := fun n => ⟨n, SetLike.natCast_mem_graded _ _⟩ natCast_zero := Subtype.ext Nat.cast_zero natCast_succ := fun n => Subtype.ext (Nat.cast_succ n) } /-- Build a `DirectSum.GCommSemiring` instance for a collection of additive submonoids. -/ instance gcommSemiring [AddCommMonoid ι] [CommSemiring R] [SetLike σ R] [AddSubmonoidClass σ R] (A : ι → σ) [SetLike.GradedMonoid A] : DirectSum.GCommSemiring fun i => A i := { SetLike.gCommMonoid A, SetLike.gsemiring A with } /-- Build a `DirectSum.GRing` instance for a collection of additive subgroups. -/ instance gring [AddMonoid ι] [Ring R] [SetLike σ R] [AddSubgroupClass σ R] (A : ι → σ) [SetLike.GradedMonoid A] : DirectSum.GRing fun i => A i := { SetLike.gsemiring A with intCast := fun z => ⟨z, SetLike.intCast_mem_graded _ _⟩ intCast_ofNat := fun _n => Subtype.ext <| Int.cast_natCast _ intCast_negSucc_ofNat := fun n => Subtype.ext <| Int.cast_negSucc n } /-- Build a `DirectSum.GCommRing` instance for a collection of additive submonoids. -/ instance gcommRing [AddCommMonoid ι] [CommRing R] [SetLike σ R] [AddSubgroupClass σ R] (A : ι → σ) [SetLike.GradedMonoid A] : DirectSum.GCommRing fun i => A i := { SetLike.gCommMonoid A, SetLike.gring A with } end SetLike namespace DirectSum section coe variable [Semiring R] [SetLike σ R] [AddSubmonoidClass σ R] (A : ι → σ) /-- The canonical ring isomorphism between `⨁ i, A i` and `R`-/ def coeRingHom [AddMonoid ι] [SetLike.GradedMonoid A] : (⨁ i, A i) →+* R := DirectSum.toSemiring (fun i => AddSubmonoidClass.subtype (A i)) rfl fun _ _ => rfl /-- The canonical ring isomorphism between `⨁ i, A i` and `R`-/ @[simp] theorem coeRingHom_of [AddMonoid ι] [SetLike.GradedMonoid A] (i : ι) (x : A i) : (coeRingHom A : _ →+* R) (of (fun i => A i) i x) = x := DirectSum.toSemiring_of _ _ _ _ _ theorem coe_mul_apply [AddMonoid ι] [SetLike.GradedMonoid A] [∀ (i : ι) (x : A i), Decidable (x ≠ 0)] (r r' : ⨁ i, A i) (n : ι) : ((r * r') n : R) = ∑ ij ∈ (r.support ×ˢ r'.support).filter (fun ij : ι × ι => ij.1 + ij.2 = n), (r ij.1 * r' ij.2 : R) := by rw [mul_eq_sum_support_ghas_mul, DFinsupp.finset_sum_apply, AddSubmonoidClass.coe_finset_sum] simp_rw [coe_of_apply, apply_ite, ZeroMemClass.coe_zero, ← Finset.sum_filter, SetLike.coe_gMul] theorem coe_mul_apply_eq_dfinsupp_sum [AddMonoid ι] [SetLike.GradedMonoid A] [∀ (i : ι) (x : A i), Decidable (x ≠ 0)] (r r' : ⨁ i, A i) (n : ι) : ((r * r') n : R) = r.sum fun i ri => r'.sum fun j rj => if i + j = n then (ri * rj : R) else 0 := by rw [mul_eq_dfinsupp_sum] iterate 2 rw [DFinsupp.sum_apply, DFinsupp.sum, AddSubmonoidClass.coe_finset_sum]; congr; ext dsimp only split_ifs with h · subst h rw [of_eq_same] rfl · rw [of_eq_of_ne _ _ _ h] rfl theorem coe_of_mul_apply_aux [AddMonoid ι] [SetLike.GradedMonoid A] {i : ι} (r : A i) (r' : ⨁ i, A i) {j n : ι} (H : ∀ x : ι, i + x = n ↔ x = j) : ((of (fun i => A i) i r * r') n : R) = r * r' j := by classical rw [coe_mul_apply_eq_dfinsupp_sum] apply (DFinsupp.sum_single_index _).trans swap · simp_rw [ZeroMemClass.coe_zero, zero_mul, ite_self] exact DFinsupp.sum_zero simp_rw [DFinsupp.sum, H, Finset.sum_ite_eq'] split_ifs with h · rfl rw [DFinsupp.not_mem_support_iff.mp h, ZeroMemClass.coe_zero, mul_zero] theorem coe_mul_of_apply_aux [AddMonoid ι] [SetLike.GradedMonoid A] (r : ⨁ i, A i) {i : ι} (r' : A i) {j n : ι} (H : ∀ x : ι, x + i = n ↔ x = j) : ((r * of (fun i => A i) i r') n : R) = r j * r' := by classical rw [coe_mul_apply_eq_dfinsupp_sum, DFinsupp.sum_comm] apply (DFinsupp.sum_single_index _).trans swap · simp_rw [ZeroMemClass.coe_zero, mul_zero, ite_self] exact DFinsupp.sum_zero simp_rw [DFinsupp.sum, H, Finset.sum_ite_eq'] split_ifs with h · rfl rw [DFinsupp.not_mem_support_iff.mp h, ZeroMemClass.coe_zero, zero_mul] theorem coe_of_mul_apply_add [AddLeftCancelMonoid ι] [SetLike.GradedMonoid A] {i : ι} (r : A i) (r' : ⨁ i, A i) (j : ι) : ((of (fun i => A i) i r * r') (i + j) : R) = r * r' j := coe_of_mul_apply_aux _ _ _ fun _x => ⟨fun h => add_left_cancel h, fun h => h ▸ rfl⟩ theorem coe_mul_of_apply_add [AddRightCancelMonoid ι] [SetLike.GradedMonoid A] (r : ⨁ i, A i) {i : ι} (r' : A i) (j : ι) : ((r * of (fun i => A i) i r') (j + i) : R) = r j * r' := coe_mul_of_apply_aux _ _ _ fun _x => ⟨fun h => add_right_cancel h, fun h => h ▸ rfl⟩ end coe section CanonicallyOrderedAddCommMonoid variable [Semiring R] [SetLike σ R] [AddSubmonoidClass σ R] (A : ι → σ) variable [CanonicallyOrderedAddCommMonoid ι] [SetLike.GradedMonoid A] theorem coe_of_mul_apply_of_not_le {i : ι} (r : A i) (r' : ⨁ i, A i) (n : ι) (h : ¬i ≤ n) : ((of (fun i => A i) i r * r') n : R) = 0 := by classical rw [coe_mul_apply_eq_dfinsupp_sum] apply (DFinsupp.sum_single_index _).trans swap · simp_rw [ZeroMemClass.coe_zero, zero_mul, ite_self] exact DFinsupp.sum_zero · rw [DFinsupp.sum, Finset.sum_ite_of_false, Finset.sum_const_zero] exact fun x _ H => h ((self_le_add_right i x).trans_eq H) theorem coe_mul_of_apply_of_not_le (r : ⨁ i, A i) {i : ι} (r' : A i) (n : ι) (h : ¬i ≤ n) : ((r * of (fun i => A i) i r') n : R) = 0 := by classical rw [coe_mul_apply_eq_dfinsupp_sum, DFinsupp.sum_comm] apply (DFinsupp.sum_single_index _).trans swap · simp_rw [ZeroMemClass.coe_zero, mul_zero, ite_self] exact DFinsupp.sum_zero · rw [DFinsupp.sum, Finset.sum_ite_of_false, Finset.sum_const_zero] exact fun x _ H => h ((self_le_add_left i x).trans_eq H) variable [Sub ι] [OrderedSub ι] [ContravariantClass ι ι (· + ·) (· ≤ ·)] /- The following two lemmas only require the same hypotheses as `eq_tsub_iff_add_eq_of_le`, but we state them for `CanonicallyOrderedAddCommMonoid` + the above three typeclasses for convenience. -/ theorem coe_mul_of_apply_of_le (r : ⨁ i, A i) {i : ι} (r' : A i) (n : ι) (h : i ≤ n) : ((r * of (fun i => A i) i r') n : R) = r (n - i) * r' := coe_mul_of_apply_aux _ _ _ fun _x => (eq_tsub_iff_add_eq_of_le h).symm theorem coe_of_mul_apply_of_le {i : ι} (r : A i) (r' : ⨁ i, A i) (n : ι) (h : i ≤ n) : ((of (fun i => A i) i r * r') n : R) = r * r' (n - i) := coe_of_mul_apply_aux _ _ _ fun x => by rw [eq_tsub_iff_add_eq_of_le h, add_comm] theorem coe_mul_of_apply (r : ⨁ i, A i) {i : ι} (r' : A i) (n : ι) [Decidable (i ≤ n)] : ((r * of (fun i => A i) i r') n : R) = if i ≤ n then (r (n - i) : R) * r' else 0 := by split_ifs with h exacts [coe_mul_of_apply_of_le _ _ _ n h, coe_mul_of_apply_of_not_le _ _ _ n h] theorem coe_of_mul_apply {i : ι} (r : A i) (r' : ⨁ i, A i) (n : ι) [Decidable (i ≤ n)] : ((of (fun i => A i) i r * r') n : R) = if i ≤ n then (r * r' (n - i) : R) else 0 := by split_ifs with h exacts [coe_of_mul_apply_of_le _ _ _ n h, coe_of_mul_apply_of_not_le _ _ _ n h] end CanonicallyOrderedAddCommMonoid end DirectSum /-! #### From `Submodule`s -/ namespace Submodule /-- Build a `DirectSum.GAlgebra` instance for a collection of `Submodule`s. -/ instance galgebra [AddMonoid ι] [CommSemiring S] [Semiring R] [Algebra S R] (A : ι → Submodule S R) [SetLike.GradedMonoid A] : DirectSum.GAlgebra S fun i => A i where toFun := ((Algebra.linearMap S R).codRestrict (A 0) <| SetLike.algebraMap_mem_graded A).toAddMonoidHom map_one := Subtype.ext <| (algebraMap S R).map_one map_mul _x _y := Sigma.subtype_ext (add_zero 0).symm <| (algebraMap S R).map_mul _ _ commutes := fun _r ⟨i, _xi⟩ => Sigma.subtype_ext ((zero_add i).trans (add_zero i).symm) <| Algebra.commutes _ _ smul_def := fun _r ⟨i, _xi⟩ => Sigma.subtype_ext (zero_add i).symm <| Algebra.smul_def _ _ @[simp] theorem setLike.coe_galgebra_toFun {ι} [AddMonoid ι] [CommSemiring S] [Semiring R] [Algebra S R] (A : ι → Submodule S R) [SetLike.GradedMonoid A] (s : S) : (DirectSum.GAlgebra.toFun (A := fun i => A i) s) = (algebraMap S R s : R) := rfl /-- A direct sum of powers of a submodule of an algebra has a multiplicative structure. -/ instance nat_power_gradedMonoid [CommSemiring S] [Semiring R] [Algebra S R] (p : Submodule S R) : SetLike.GradedMonoid fun i : ℕ => p ^ i where one_mem := by rw [← one_le, pow_zero] mul_mem i j p q hp hq := by rw [pow_add] exact Submodule.mul_mem_mul hp hq end Submodule /-- The canonical algebra isomorphism between `⨁ i, A i` and `R`. -/ def DirectSum.coeAlgHom [AddMonoid ι] [CommSemiring S] [Semiring R] [Algebra S R] (A : ι → Submodule S R) [SetLike.GradedMonoid A] : (⨁ i, A i) →ₐ[S] R := DirectSum.toAlgebra S _ (fun i => (A i).subtype) rfl (fun _ _ => rfl) /-- The supremum of submodules that form a graded monoid is a subalgebra, and equal to the range of `DirectSum.coeAlgHom`. -/ theorem Submodule.iSup_eq_toSubmodule_range [AddMonoid ι] [CommSemiring S] [Semiring R] [Algebra S R] (A : ι → Submodule S R) [SetLike.GradedMonoid A] : ⨆ i, A i = Subalgebra.toSubmodule (DirectSum.coeAlgHom A).range := (Submodule.iSup_eq_range_dfinsupp_lsum A).trans <| SetLike.coe_injective rfl @[simp] theorem DirectSum.coeAlgHom_of [AddMonoid ι] [CommSemiring S] [Semiring R] [Algebra S R] (A : ι → Submodule S R) [SetLike.GradedMonoid A] (i : ι) (x : A i) : DirectSum.coeAlgHom A (DirectSum.of (fun i => A i) i x) = x := DirectSum.toSemiring_of _ (by rfl) (fun _ _ => (by rfl)) _ _ end DirectSum /-! ### Facts about grade zero -/ namespace SetLike.GradeZero section Semiring variable [Semiring R] [AddMonoid ι] [SetLike σ R] [AddSubmonoidClass σ R] variable (A : ι → σ) [SetLike.GradedMonoid A] /-- The subsemiring `A 0` of `R`. -/ def subsemiring : Subsemiring R where carrier := A 0 __ := submonoid A add_mem' := add_mem zero_mem' := zero_mem (A 0) -- TODO: it might be expensive to unify `A` in this instance in practice /-- The semiring `A 0` inherited from `R` in the presence of `SetLike.GradedMonoid A`. -/ instance instSemiring : Semiring (A 0) := (subsemiring A).toSemiring /- The linter message "error: SetLike.GradeZero.coe_natCast.{u_4, u_2, u_1} Left-hand side does not simplify, when using the simp lemma on itself." is wrong. The LHS does simplify. -/ @[nolint simpNF, simp, norm_cast] theorem coe_natCast (n : ℕ) : (n : A 0) = (n : R) := rfl /- The linter message "error: SetLike.GradeZero.coe_ofNat.{u_4, u_2, u_1} Left-hand side does not simplify, when using the simp lemma on itself." is wrong. The LHS does simplify. -/ @[nolint simpNF, simp, norm_cast] theorem coe_ofNat (n : ℕ) [n.AtLeastTwo] : (no_index (OfNat.ofNat n) : A 0) = (OfNat.ofNat n : R) := rfl end Semiring section CommSemiring variable [CommSemiring R] [AddCommMonoid ι] [SetLike σ R] [AddSubmonoidClass σ R] variable (A : ι → σ) [SetLike.GradedMonoid A] -- TODO: it might be expensive to unify `A` in this instance in practice /--The commutative semiring `A 0` inherited from `R` in the presence of `SetLike.GradedMonoid A`.-/ instance instCommSemiring : CommSemiring (A 0) := (subsemiring A).toCommSemiring end CommSemiring section Ring variable [Ring R] [AddMonoid ι] [SetLike σ R] [AddSubgroupClass σ R] variable (A : ι → σ) [SetLike.GradedMonoid A] /-- The subring `A 0` of `R`. -/ def subring : Subring R where carrier := A 0 __ := subsemiring A neg_mem' := neg_mem -- TODO: it might be expensive to unify `A` in this instances in practice /-- The ring `A 0` inherited from `R` in the presence of `SetLike.GradedMonoid A`. -/ instance instRing : Ring (A 0) := (subring A).toRing theorem coe_intCast (z : ℤ) : (z : A 0) = (z : R) := rfl end Ring section CommRing variable [CommRing R] [AddCommMonoid ι] [SetLike σ R] [AddSubgroupClass σ R] variable (A : ι → σ) [SetLike.GradedMonoid A] -- TODO: it might be expensive to unify `A` in this instances in practice /-- The commutative ring `A 0` inherited from `R` in the presence of `SetLike.GradedMonoid A`. -/ instance instCommRing : CommRing (A 0) := (subring A).toCommRing end CommRing section Algebra variable [CommSemiring S] [Semiring R] [Algebra S R] [AddMonoid ι] variable (A : ι → Submodule S R) [SetLike.GradedMonoid A] /-- The subalgebra `A 0` of `R`. -/ def subalgebra : Subalgebra S R where carrier := A 0 __ := subsemiring A algebraMap_mem' := algebraMap_mem_graded A -- TODO: it might be expensive to unify `A` in this instances in practice /-- The `S`-algebra `A 0` inherited from `R` in the presence of `SetLike.GradedMonoid A`. -/ instance instAlgebra : Algebra S (A 0) := inferInstanceAs <| Algebra S (subalgebra A) /- The linter message "error: SetLike.GradeZero.coe_algebraMap.{u_4, u_3, u_1} Left-hand side does not simplify, when using the simp lemma on itself." is wrong. The LHS does simplify. -/ @[nolint simpNF, simp, norm_cast] theorem coe_algebraMap (s : S) : ↑(algebraMap _ (A 0) s) = algebraMap _ R s := rfl end Algebra end SetLike.GradeZero section HomogeneousElement theorem SetLike.homogeneous_zero_submodule [Zero ι] [Semiring S] [AddCommMonoid R] [Module S R] (A : ι → Submodule S R) : SetLike.Homogeneous A (0 : R) := ⟨0, Submodule.zero_mem _⟩ theorem SetLike.Homogeneous.smul [CommSemiring S] [Semiring R] [Algebra S R] {A : ι → Submodule S R} {s : S} {r : R} (hr : SetLike.Homogeneous A r) : SetLike.Homogeneous A (s • r) := let ⟨i, hi⟩ := hr ⟨i, Submodule.smul_mem _ _ hi⟩ end HomogeneousElement
Algebra\DirectSum\LinearMap.lean
/- Copyright (c) 2023 Oliver Nash. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Oliver Nash -/ import Mathlib.LinearAlgebra.FreeModule.Finite.Basic import Mathlib.LinearAlgebra.FreeModule.PID import Mathlib.LinearAlgebra.Eigenspace.Basic import Mathlib.LinearAlgebra.Trace /-! # Linear maps between direct sums This file contains results about linear maps which respect direct sum decompositions of their domain and codomain. -/ open Set DirectSum namespace LinearMap variable {ι R M : Type*} [CommRing R] [AddCommGroup M] [Module R M] {N : ι → Submodule R M} section IsInternal variable [DecidableEq ι] /-- If a linear map `f : M₁ → M₂` respects direct sum decompositions of `M₁` and `M₂`, then it has a block diagonal matrix with respect to bases compatible with the direct sum decompositions. -/ lemma toMatrix_directSum_collectedBasis_eq_blockDiagonal' {R M₁ M₂ : Type*} [CommSemiring R] [AddCommMonoid M₁] [Module R M₁] {N₁ : ι → Submodule R M₁} (h₁ : IsInternal N₁) [AddCommMonoid M₂] [Module R M₂] {N₂ : ι → Submodule R M₂} (h₂ : IsInternal N₂) {κ₁ κ₂ : ι → Type*} [∀ i, Fintype (κ₁ i)] [∀ i, Finite (κ₂ i)] [∀ i, DecidableEq (κ₁ i)] [Fintype ι] (b₁ : (i : ι) → Basis (κ₁ i) R (N₁ i)) (b₂ : (i : ι) → Basis (κ₂ i) R (N₂ i)) {f : M₁ →ₗ[R] M₂} (hf : ∀ i, MapsTo f (N₁ i) (N₂ i)) : toMatrix (h₁.collectedBasis b₁) (h₂.collectedBasis b₂) f = Matrix.blockDiagonal' fun i ↦ toMatrix (b₁ i) (b₂ i) (f.restrict (hf i)) := by ext ⟨i, _⟩ ⟨j, _⟩ simp only [toMatrix_apply, Matrix.blockDiagonal'_apply] rcases eq_or_ne i j with rfl | hij · simp [h₂.collectedBasis_repr_of_mem _ (hf _ (Subtype.mem _)), restrict_apply] · simp [hij, h₂.collectedBasis_repr_of_mem_ne _ hij.symm (hf _ (Subtype.mem _))] lemma diag_toMatrix_directSum_collectedBasis_eq_zero_of_mapsTo_ne {κ : ι → Type*} [∀ i, Fintype (κ i)] [∀ i, DecidableEq (κ i)] {s : Finset ι} (h : IsInternal fun i : s ↦ N i) (b : (i : s) → Basis (κ i) R (N i)) (σ : ι → ι) (hσ : ∀ i, σ i ≠ i) {f : Module.End R M} (hf : ∀ i, MapsTo f (N i) (N <| σ i)) (hN : ∀ i, i ∉ s → N i = ⊥) : Matrix.diag (toMatrix (h.collectedBasis b) (h.collectedBasis b) f) = 0 := by ext ⟨i, k⟩ simp only [Matrix.diag_apply, Pi.zero_apply, toMatrix_apply, IsInternal.collectedBasis_coe] by_cases hi : σ i ∈ s · let j : s := ⟨σ i, hi⟩ replace hσ : j ≠ i := fun hij ↦ hσ i <| Subtype.ext_iff.mp hij exact h.collectedBasis_repr_of_mem_ne b hσ <| hf _ <| Subtype.mem (b i k) · suffices f (b i k) = 0 by simp [this] simpa [hN _ hi] using hf i <| Subtype.mem (b i k) variable [∀ i, Module.Finite R (N i)] [∀ i, Module.Free R (N i)] /-- The trace of an endomorphism of a direct sum is the sum of the traces on each component. See also `LinearMap.trace_restrict_eq_sum_trace_restrict`. -/ lemma trace_eq_sum_trace_restrict (h : IsInternal N) [Fintype ι] {f : M →ₗ[R] M} (hf : ∀ i, MapsTo f (N i) (N i)) : trace R M f = ∑ i, trace R (N i) (f.restrict (hf i)) := by let b : (i : ι) → Basis _ R (N i) := fun i ↦ Module.Free.chooseBasis R (N i) simp_rw [trace_eq_matrix_trace R (h.collectedBasis b), toMatrix_directSum_collectedBasis_eq_blockDiagonal' h h b b hf, Matrix.trace_blockDiagonal', ← trace_eq_matrix_trace] lemma trace_eq_sum_trace_restrict' (h : IsInternal N) (hN : {i | N i ≠ ⊥}.Finite) {f : M →ₗ[R] M} (hf : ∀ i, MapsTo f (N i) (N i)) : trace R M f = ∑ i ∈ hN.toFinset, trace R (N i) (f.restrict (hf i)) := by let _ : Fintype {i // N i ≠ ⊥} := hN.fintype let _ : Fintype {i | N i ≠ ⊥} := hN.fintype rw [← Finset.sum_coe_sort, trace_eq_sum_trace_restrict (isInternal_ne_bot_iff.mpr h) _] exact Fintype.sum_equiv hN.subtypeEquivToFinset _ _ (fun i ↦ rfl) lemma trace_eq_zero_of_mapsTo_ne (h : IsInternal N) [IsNoetherian R M] (σ : ι → ι) (hσ : ∀ i, σ i ≠ i) {f : Module.End R M} (hf : ∀ i, MapsTo f (N i) (N <| σ i)) : trace R M f = 0 := by have hN : {i | N i ≠ ⊥}.Finite := CompleteLattice.WellFounded.finite_ne_bot_of_independent (wellFounded_submodule_gt R M) h.submodule_independent let s := hN.toFinset let κ := fun i ↦ Module.Free.ChooseBasisIndex R (N i) let b : (i : s) → Basis (κ i) R (N i) := fun i ↦ Module.Free.chooseBasis R (N i) replace h : IsInternal fun i : s ↦ N i := by convert DirectSum.isInternal_ne_bot_iff.mpr h <;> simp [s] simp_rw [trace_eq_matrix_trace R (h.collectedBasis b), Matrix.trace, diag_toMatrix_directSum_collectedBasis_eq_zero_of_mapsTo_ne h b σ hσ hf (by simp [s]), Pi.zero_apply, Finset.sum_const_zero] /-- If `f` and `g` are commuting endomorphisms of a finite, free `R`-module `M`, such that `f` is triangularizable, then to prove that the trace of `g ∘ f` vanishes, it is sufficient to prove that the trace of `g` vanishes on each generalized eigenspace of `f`. -/ lemma trace_comp_eq_zero_of_commute_of_trace_restrict_eq_zero [IsDomain R] [IsPrincipalIdealRing R] [Module.Free R M] [Module.Finite R M] {f g : Module.End R M} (h_comm : Commute f g) (hf : ⨆ μ, ⨆ k, f.genEigenspace μ k = ⊤) (hg : ∀ μ, trace R _ (g.restrict (f.mapsTo_iSup_genEigenspace_of_comm h_comm μ)) = 0) : trace R _ (g ∘ₗ f) = 0 := by have hfg : ∀ μ, MapsTo (g ∘ₗ f) ↑(⨆ k, f.genEigenspace μ k) ↑(⨆ k, f.genEigenspace μ k) := fun μ ↦ (f.mapsTo_iSup_genEigenspace_of_comm h_comm μ).comp (f.mapsTo_iSup_genEigenspace_of_comm rfl μ) suffices ∀ μ, trace R _ ((g ∘ₗ f).restrict (hfg μ)) = 0 by classical have hds := DirectSum.isInternal_submodule_of_independent_of_iSup_eq_top f.independent_genEigenspace hf have h_fin : {μ | ⨆ k, f.genEigenspace μ k ≠ ⊥}.Finite := CompleteLattice.WellFounded.finite_ne_bot_of_independent (isNoetherian_iff_wellFounded.mp inferInstance) f.independent_genEigenspace simp [trace_eq_sum_trace_restrict' hds h_fin hfg, this] intro μ replace h_comm : Commute (g.restrict (f.mapsTo_iSup_genEigenspace_of_comm h_comm μ)) (f.restrict (f.mapsTo_iSup_genEigenspace_of_comm rfl μ)) := restrict_commute h_comm.symm _ _ rw [restrict_comp, trace_comp_eq_mul_of_commute_of_isNilpotent μ h_comm (f.isNilpotent_restrict_iSup_sub_algebraMap μ), hg, mul_zero] lemma mapsTo_biSup_of_mapsTo {ι : Type*} {N : ι → Submodule R M} (s : Set ι) {f : Module.End R M} (hf : ∀ i, MapsTo f (N i) (N i)) : MapsTo f ↑(⨆ i ∈ s, N i) ↑(⨆ i ∈ s, N i) := by replace hf : ∀ i, (N i).map f ≤ N i := fun i ↦ Submodule.map_le_iff_le_comap.mpr (hf i) suffices (⨆ i ∈ s, N i).map f ≤ ⨆ i ∈ s, N i from Submodule.map_le_iff_le_comap.mp this simpa only [Submodule.map_iSup] using iSup₂_mono <| fun i _ ↦ hf i end IsInternal /-- The trace of an endomorphism of a direct sum is the sum of the traces on each component. Note that it is important the statement gives the user definitional control over `p` since the _type_ of the term `trace R p (f.restrict hp')` depends on `p`. -/ lemma trace_eq_sum_trace_restrict_of_eq_biSup [∀ i, Module.Finite R (N i)] [∀ i, Module.Free R (N i)] (s : Finset ι) (h : CompleteLattice.Independent <| fun i : s ↦ N i) {f : Module.End R M} (hf : ∀ i, MapsTo f (N i) (N i)) (p : Submodule R M) (hp : p = ⨆ i ∈ s, N i) (hp' : MapsTo f p p := hp ▸ mapsTo_biSup_of_mapsTo (s : Set ι) hf) : trace R p (f.restrict hp') = ∑ i ∈ s, trace R (N i) (f.restrict (hf i)) := by classical let N' : s → Submodule R p := fun i ↦ (N i).comap p.subtype replace h : IsInternal N' := hp ▸ isInternal_biSup_submodule_of_independent (s : Set ι) h have hf' : ∀ i, MapsTo (restrict f hp') (N' i) (N' i) := fun i x hx' ↦ by simpa using hf i hx' let e : (i : s) → N' i ≃ₗ[R] N i := fun ⟨i, hi⟩ ↦ (N i).comapSubtypeEquivOfLe (hp ▸ le_biSup N hi) have _i1 : ∀ i, Module.Finite R (N' i) := fun i ↦ Module.Finite.equiv (e i).symm have _i2 : ∀ i, Module.Free R (N' i) := fun i ↦ Module.Free.of_equiv (e i).symm rw [trace_eq_sum_trace_restrict h hf', ← s.sum_coe_sort] have : ∀ i : s, f.restrict (hf i) = (e i).conj ((f.restrict hp').restrict (hf' i)) := fun _ ↦ rfl simp [this] end LinearMap
Algebra\DirectSum\Module.lean
/- Copyright (c) 2018 Kenny Lau. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Kenny Lau -/ import Mathlib.Algebra.DirectSum.Basic import Mathlib.LinearAlgebra.DFinsupp import Mathlib.LinearAlgebra.Basis /-! # Direct sum of modules The first part of the file provides constructors for direct sums of modules. It provides a construction of the direct sum using the universal property and proves its uniqueness (`DirectSum.toModule.unique`). The second part of the file covers the special case of direct sums of submodules of a fixed module `M`. There is a canonical linear map from this direct sum to `M` (`DirectSum.coeLinearMap`), and the construction is of particular importance when this linear map is an equivalence; that is, when the submodules provide an internal decomposition of `M`. The property is defined more generally elsewhere as `DirectSum.IsInternal`, but its basic consequences on `Submodule`s are established in this file. -/ universe u v w u₁ namespace DirectSum open DirectSum section General variable {R : Type u} [Semiring R] variable {ι : Type v} variable {M : ι → Type w} [∀ i, AddCommMonoid (M i)] [∀ i, Module R (M i)] instance : Module R (⨁ i, M i) := DFinsupp.module instance {S : Type*} [Semiring S] [∀ i, Module S (M i)] [∀ i, SMulCommClass R S (M i)] : SMulCommClass R S (⨁ i, M i) := DFinsupp.smulCommClass instance {S : Type*} [Semiring S] [SMul R S] [∀ i, Module S (M i)] [∀ i, IsScalarTower R S (M i)] : IsScalarTower R S (⨁ i, M i) := DFinsupp.isScalarTower instance [∀ i, Module Rᵐᵒᵖ (M i)] [∀ i, IsCentralScalar R (M i)] : IsCentralScalar R (⨁ i, M i) := DFinsupp.isCentralScalar theorem smul_apply (b : R) (v : ⨁ i, M i) (i : ι) : (b • v) i = b • v i := DFinsupp.smul_apply _ _ _ variable (R ι M) section DecidableEq variable [DecidableEq ι] /-- Create the direct sum given a family `M` of `R` modules indexed over `ι`. -/ def lmk : ∀ s : Finset ι, (∀ i : (↑s : Set ι), M i.val) →ₗ[R] ⨁ i, M i := DFinsupp.lmk /-- Inclusion of each component into the direct sum. -/ def lof : ∀ i : ι, M i →ₗ[R] ⨁ i, M i := DFinsupp.lsingle theorem lof_eq_of (i : ι) (b : M i) : lof R ι M i b = of M i b := rfl variable {ι M} theorem single_eq_lof (i : ι) (b : M i) : DFinsupp.single i b = lof R ι M i b := rfl /-- Scalar multiplication commutes with direct sums. -/ theorem mk_smul (s : Finset ι) (c : R) (x) : mk M s (c • x) = c • mk M s x := (lmk R ι M s).map_smul c x /-- Scalar multiplication commutes with the inclusion of each component into the direct sum. -/ theorem of_smul (i : ι) (c : R) (x) : of M i (c • x) = c • of M i x := (lof R ι M i).map_smul c x variable {R} theorem support_smul [∀ (i : ι) (x : M i), Decidable (x ≠ 0)] (c : R) (v : ⨁ i, M i) : (c • v).support ⊆ v.support := DFinsupp.support_smul _ _ variable {N : Type u₁} [AddCommMonoid N] [Module R N] variable (φ : ∀ i, M i →ₗ[R] N) variable (R ι N) /-- The linear map constructed using the universal property of the coproduct. -/ def toModule : (⨁ i, M i) →ₗ[R] N := DFunLike.coe (DFinsupp.lsum ℕ) φ /-- Coproducts in the categories of modules and additive monoids commute with the forgetful functor from modules to additive monoids. -/ theorem coe_toModule_eq_coe_toAddMonoid : (toModule R ι N φ : (⨁ i, M i) → N) = toAddMonoid fun i ↦ (φ i).toAddMonoidHom := rfl variable {ι N φ} /-- The map constructed using the universal property gives back the original maps when restricted to each component. -/ @[simp] theorem toModule_lof (i) (x : M i) : toModule R ι N φ (lof R ι M i x) = φ i x := toAddMonoid_of (fun i ↦ (φ i).toAddMonoidHom) i x variable (ψ : (⨁ i, M i) →ₗ[R] N) /-- Every linear map from a direct sum agrees with the one obtained by applying the universal property to each of its components. -/ theorem toModule.unique (f : ⨁ i, M i) : ψ f = toModule R ι N (fun i ↦ ψ.comp <| lof R ι M i) f := toAddMonoid.unique ψ.toAddMonoidHom f variable {ψ} {ψ' : (⨁ i, M i) →ₗ[R] N} /-- Two `LinearMap`s out of a direct sum are equal if they agree on the generators. See note [partially-applied ext lemmas]. -/ @[ext] theorem linearMap_ext ⦃ψ ψ' : (⨁ i, M i) →ₗ[R] N⦄ (H : ∀ i, ψ.comp (lof R ι M i) = ψ'.comp (lof R ι M i)) : ψ = ψ' := DFinsupp.lhom_ext' H /-- The inclusion of a subset of the direct summands into a larger subset of the direct summands, as a linear map. -/ def lsetToSet (S T : Set ι) (H : S ⊆ T) : (⨁ i : S, M i) →ₗ[R] ⨁ i : T, M i := toModule R _ _ fun i ↦ lof R T (fun i : Subtype T ↦ M i) ⟨i, H i.prop⟩ variable (ι M) /-- Given `Fintype α`, `linearEquivFunOnFintype R` is the natural `R`-linear equivalence between `⨁ i, M i` and `∀ i, M i`. -/ @[simps apply] def linearEquivFunOnFintype [Fintype ι] : (⨁ i, M i) ≃ₗ[R] ∀ i, M i := { DFinsupp.equivFunOnFintype with toFun := (↑) map_add' := fun f g ↦ by ext rw [add_apply, Pi.add_apply] map_smul' := fun c f ↦ by simp_rw [RingHom.id_apply] rw [DFinsupp.coe_smul] } variable {ι M} @[simp] theorem linearEquivFunOnFintype_lof [Fintype ι] (i : ι) (m : M i) : (linearEquivFunOnFintype R ι M) (lof R ι M i m) = Pi.single i m := by ext a change (DFinsupp.equivFunOnFintype (lof R ι M i m)) a = _ convert _root_.congr_fun (DFinsupp.equivFunOnFintype_single i m) a @[simp] theorem linearEquivFunOnFintype_symm_single [Fintype ι] (i : ι) (m : M i) : (linearEquivFunOnFintype R ι M).symm (Pi.single i m) = lof R ι M i m := by change (DFinsupp.equivFunOnFintype.symm (Pi.single i m)) = _ rw [DFinsupp.equivFunOnFintype_symm_single i m] rfl end DecidableEq @[simp] theorem linearEquivFunOnFintype_symm_coe [Fintype ι] (f : ⨁ i, M i) : (linearEquivFunOnFintype R ι M).symm f = f := by simp [linearEquivFunOnFintype] /-- The natural linear equivalence between `⨁ _ : ι, M` and `M` when `Unique ι`. -/ protected def lid (M : Type v) (ι : Type* := PUnit) [AddCommMonoid M] [Module R M] [Unique ι] : (⨁ _ : ι, M) ≃ₗ[R] M := { DirectSum.id M ι, toModule R ι M fun _ ↦ LinearMap.id with } /-- The projection map onto one component, as a linear map. -/ def component (i : ι) : (⨁ i, M i) →ₗ[R] M i := DFinsupp.lapply i variable {ι M} theorem apply_eq_component (f : ⨁ i, M i) (i : ι) : f i = component R ι M i f := rfl -- Note(kmill): `@[ext]` cannot prove `ext_iff` because `R` is not determined by `f` or `g`. @[ext (iff := false)] theorem ext {f g : ⨁ i, M i} (h : ∀ i, component R ι M i f = component R ι M i g) : f = g := DFinsupp.ext h theorem ext_iff {f g : ⨁ i, M i} : f = g ↔ ∀ i, component R ι M i f = component R ι M i g := ⟨fun h _ ↦ by rw [h], ext R⟩ @[simp] theorem lof_apply [DecidableEq ι] (i : ι) (b : M i) : ((lof R ι M i) b) i = b := DFinsupp.single_eq_same @[simp] theorem component.lof_self [DecidableEq ι] (i : ι) (b : M i) : component R ι M i ((lof R ι M i) b) = b := lof_apply R i b theorem component.of [DecidableEq ι] (i j : ι) (b : M j) : component R ι M i ((lof R ι M j) b) = if h : j = i then Eq.recOn h b else 0 := DFinsupp.single_apply section CongrLeft variable {κ : Type*} /-- Reindexing terms of a direct sum is linear. -/ def lequivCongrLeft (h : ι ≃ κ) : (⨁ i, M i) ≃ₗ[R] ⨁ k, M (h.symm k) := { equivCongrLeft h with map_smul' := DFinsupp.comapDomain'_smul h.invFun h.right_inv } @[simp] theorem lequivCongrLeft_apply (h : ι ≃ κ) (f : ⨁ i, M i) (k : κ) : lequivCongrLeft R h f k = f (h.symm k) := equivCongrLeft_apply _ _ _ end CongrLeft section Sigma variable {α : ι → Type*} {δ : ∀ i, α i → Type w} variable [DecidableEq ι] [∀ i j, AddCommMonoid (δ i j)] [∀ i j, Module R (δ i j)] /-- `curry` as a linear map. -/ def sigmaLcurry : (⨁ i : Σi, _, δ i.1 i.2) →ₗ[R] ⨁ (i) (j), δ i j := { sigmaCurry with map_smul' := fun r ↦ by convert DFinsupp.sigmaCurry_smul (δ := δ) r } @[simp] theorem sigmaLcurry_apply (f : ⨁ i : Σ_, _, δ i.1 i.2) (i : ι) (j : α i) : sigmaLcurry R f i j = f ⟨i, j⟩ := sigmaCurry_apply f i j /-- `uncurry` as a linear map. -/ def sigmaLuncurry : (⨁ (i) (j), δ i j) →ₗ[R] ⨁ i : Σ_, _, δ i.1 i.2 := { sigmaUncurry with map_smul' := DFinsupp.sigmaUncurry_smul } @[simp] theorem sigmaLuncurry_apply (f : ⨁ (i) (j), δ i j) (i : ι) (j : α i) : sigmaLuncurry R f ⟨i, j⟩ = f i j := sigmaUncurry_apply f i j /-- `curryEquiv` as a linear equiv. -/ def sigmaLcurryEquiv : (⨁ i : Σ_, _, δ i.1 i.2) ≃ₗ[R] ⨁ (i) (j), δ i j := { sigmaCurryEquiv, sigmaLcurry R with } end Sigma section Option variable {α : Option ι → Type w} [∀ i, AddCommMonoid (α i)] [∀ i, Module R (α i)] /-- Linear isomorphism obtained by separating the term of index `none` of a direct sum over `Option ι`. -/ @[simps] noncomputable def lequivProdDirectSum : (⨁ i, α i) ≃ₗ[R] α none × ⨁ i, α (some i) := { addEquivProdDirectSum with map_smul' := DFinsupp.equivProdDFinsupp_smul } end Option end General section Submodule section Semiring variable {R : Type u} [Semiring R] variable {ι : Type v} [dec_ι : DecidableEq ι] variable {M : Type*} [AddCommMonoid M] [Module R M] variable (A : ι → Submodule R M) /-- The canonical embedding from `⨁ i, A i` to `M` where `A` is a collection of `Submodule R M` indexed by `ι`. This is `DirectSum.coeAddMonoidHom` as a `LinearMap`. -/ def coeLinearMap : (⨁ i, A i) →ₗ[R] M := toModule R ι M fun i ↦ (A i).subtype theorem coeLinearMap_eq_dfinsupp_sum [DecidableEq M] (x : DirectSum ι fun i => A i) : coeLinearMap A x = DFinsupp.sum x fun i => (fun x : A i => ↑x) := by simp only [coeLinearMap, toModule, DFinsupp.lsum, LinearEquiv.coe_mk, LinearMap.coe_mk, AddHom.coe_mk] rw [DFinsupp.sumAddHom_apply] simp only [LinearMap.toAddMonoidHom_coe, Submodule.coeSubtype] @[simp] theorem coeLinearMap_of (i : ι) (x : A i) : DirectSum.coeLinearMap A (of (fun i ↦ A i) i x) = x := -- Porting note: spelled out arguments. (I don't know how this works.) toAddMonoid_of (β := fun i => A i) (fun i ↦ ((A i).subtype : A i →+ M)) i x variable {A} @[simp] theorem IsInternal.ofBijective_coeLinearMap_same (h : IsInternal A) {i : ι} (x : A i) : (LinearEquiv.ofBijective (coeLinearMap A) h).symm x i = x := by rw [← coeLinearMap_of, LinearEquiv.ofBijective_symm_apply_apply, of_eq_same] @[simp] theorem IsInternal.ofBijective_coeLinearMap_of_ne (h : IsInternal A) {i j : ι} (hij : i ≠ j) (x : A i) : (LinearEquiv.ofBijective (coeLinearMap A) h).symm x j = 0 := by rw [← coeLinearMap_of, LinearEquiv.ofBijective_symm_apply_apply, of_eq_of_ne i j _ hij] theorem IsInternal.ofBijective_coeLinearMap_of_mem (h : IsInternal A) {i : ι} {x : M} (hx : x ∈ A i) : (LinearEquiv.ofBijective (coeLinearMap A) h).symm x i = ⟨x, hx⟩ := h.ofBijective_coeLinearMap_same ⟨x, hx⟩ theorem IsInternal.ofBijective_coeLinearMap_of_mem_ne (h : IsInternal A) {i j : ι} (hij : i ≠ j) {x : M} (hx : x ∈ A i) : (LinearEquiv.ofBijective (coeLinearMap A) h).symm x j = 0 := h.ofBijective_coeLinearMap_of_ne hij ⟨x, hx⟩ /-- If a direct sum of submodules is internal then the submodules span the module. -/ theorem IsInternal.submodule_iSup_eq_top (h : IsInternal A) : iSup A = ⊤ := by rw [Submodule.iSup_eq_range_dfinsupp_lsum, LinearMap.range_eq_top] exact Function.Bijective.surjective h /-- If a direct sum of submodules is internal then the submodules are independent. -/ theorem IsInternal.submodule_independent (h : IsInternal A) : CompleteLattice.Independent A := CompleteLattice.independent_of_dfinsupp_lsum_injective _ h.injective /-- Given an internal direct sum decomposition of a module `M`, and a basis for each of the components of the direct sum, the disjoint union of these bases is a basis for `M`. -/ noncomputable def IsInternal.collectedBasis (h : IsInternal A) {α : ι → Type*} (v : ∀ i, Basis (α i) R (A i)) : Basis (Σi, α i) R M where repr := ((LinearEquiv.ofBijective (DirectSum.coeLinearMap A) h).symm ≪≫ₗ DFinsupp.mapRange.linearEquiv fun i ↦ (v i).repr) ≪≫ₗ (sigmaFinsuppLequivDFinsupp R).symm @[simp] theorem IsInternal.collectedBasis_coe (h : IsInternal A) {α : ι → Type*} (v : ∀ i, Basis (α i) R (A i)) : ⇑(h.collectedBasis v) = fun a : Σi, α i ↦ ↑(v a.1 a.2) := by funext a -- Porting note: was -- simp only [IsInternal.collectedBasis, toModule, coeLinearMap, Basis.coe_ofRepr, -- Basis.repr_symm_apply, DFinsupp.lsum_apply_apply, DFinsupp.mapRange.linearEquiv_apply, -- DFinsupp.mapRange.linearEquiv_symm, DFinsupp.mapRange_single, Finsupp.total_single, -- LinearEquiv.ofBijective_apply, LinearEquiv.symm_symm, LinearEquiv.symm_trans_apply, one_smul, -- sigmaFinsuppAddEquivDFinsupp_apply, sigmaFinsuppEquivDFinsupp_single, -- sigmaFinsuppLequivDFinsupp_apply] -- convert DFinsupp.sumAddHom_single (fun i ↦ (A i).subtype.toAddMonoidHom) a.1 (v a.1 a.2) simp only [IsInternal.collectedBasis, coeLinearMap, Basis.coe_ofRepr, LinearEquiv.trans_symm, LinearEquiv.symm_symm, LinearEquiv.trans_apply, sigmaFinsuppLequivDFinsupp_apply, sigmaFinsuppEquivDFinsupp_single, LinearEquiv.ofBijective_apply, sigmaFinsuppAddEquivDFinsupp_apply] rw [DFinsupp.mapRange.linearEquiv_symm] erw [DFinsupp.mapRange.linearEquiv_apply] simp only [DFinsupp.mapRange_single, Basis.repr_symm_apply, Finsupp.total_single, one_smul, toModule] erw [DFinsupp.lsum_single] simp only [Submodule.coeSubtype] theorem IsInternal.collectedBasis_mem (h : IsInternal A) {α : ι → Type*} (v : ∀ i, Basis (α i) R (A i)) (a : Σi, α i) : h.collectedBasis v a ∈ A a.1 := by simp theorem IsInternal.collectedBasis_repr_of_mem (h : IsInternal A) {α : ι → Type*} (v : ∀ i, Basis (α i) R (A i)) {x : M} {i : ι} {a : α i} (hx : x ∈ A i) : (h.collectedBasis v).repr x ⟨i, a⟩ = (v i).repr ⟨x, hx⟩ a := by change (sigmaFinsuppLequivDFinsupp R).symm (DFinsupp.mapRange _ (fun i ↦ map_zero _) _) _ = _ simp [h.ofBijective_coeLinearMap_of_mem hx] theorem IsInternal.collectedBasis_repr_of_mem_ne (h : IsInternal A) {α : ι → Type*} (v : ∀ i, Basis (α i) R (A i)) {x : M} {i j : ι} (hij : i ≠ j) {a : α j} (hx : x ∈ A i) : (h.collectedBasis v).repr x ⟨j, a⟩ = 0 := by change (sigmaFinsuppLequivDFinsupp R).symm (DFinsupp.mapRange _ (fun i ↦ map_zero _) _) _ = _ simp [h.ofBijective_coeLinearMap_of_mem_ne hij hx] /-- When indexed by only two distinct elements, `DirectSum.IsInternal` implies the two submodules are complementary. Over a `Ring R`, this is true as an iff, as `DirectSum.isInternal_submodule_iff_isCompl`. -/ theorem IsInternal.isCompl {A : ι → Submodule R M} {i j : ι} (hij : i ≠ j) (h : (Set.univ : Set ι) = {i, j}) (hi : IsInternal A) : IsCompl (A i) (A j) := ⟨hi.submodule_independent.pairwiseDisjoint hij, codisjoint_iff.mpr <| Eq.symm <| hi.submodule_iSup_eq_top.symm.trans <| by rw [← sSup_pair, iSup, ← Set.image_univ, h, Set.image_insert_eq, Set.image_singleton]⟩ end Semiring section Ring variable {R : Type u} [Ring R] variable {ι : Type v} [dec_ι : DecidableEq ι] variable {M : Type*} [AddCommGroup M] [Module R M] /-- Note that this is not generally true for `[Semiring R]`; see `CompleteLattice.Independent.dfinsupp_lsum_injective` for details. -/ theorem isInternal_submodule_of_independent_of_iSup_eq_top {A : ι → Submodule R M} (hi : CompleteLattice.Independent A) (hs : iSup A = ⊤) : IsInternal A := ⟨hi.dfinsupp_lsum_injective, -- Note: #8386 had to specify value of `f` (LinearMap.range_eq_top (f := DFinsupp.lsum _ _)).1 <| (Submodule.iSup_eq_range_dfinsupp_lsum _).symm.trans hs⟩ /-- `iff` version of `DirectSum.isInternal_submodule_of_independent_of_iSup_eq_top`, `DirectSum.IsInternal.submodule_independent`, and `DirectSum.IsInternal.submodule_iSup_eq_top`. -/ theorem isInternal_submodule_iff_independent_and_iSup_eq_top (A : ι → Submodule R M) : IsInternal A ↔ CompleteLattice.Independent A ∧ iSup A = ⊤ := ⟨fun i ↦ ⟨i.submodule_independent, i.submodule_iSup_eq_top⟩, And.rec isInternal_submodule_of_independent_of_iSup_eq_top⟩ /-- If a collection of submodules has just two indices, `i` and `j`, then `DirectSum.IsInternal` is equivalent to `isCompl`. -/ theorem isInternal_submodule_iff_isCompl (A : ι → Submodule R M) {i j : ι} (hij : i ≠ j) (h : (Set.univ : Set ι) = {i, j}) : IsInternal A ↔ IsCompl (A i) (A j) := by have : ∀ k, k = i ∨ k = j := fun k ↦ by simpa using Set.ext_iff.mp h k rw [isInternal_submodule_iff_independent_and_iSup_eq_top, iSup, ← Set.image_univ, h, Set.image_insert_eq, Set.image_singleton, sSup_pair, CompleteLattice.independent_pair hij this] exact ⟨fun ⟨hd, ht⟩ ↦ ⟨hd, codisjoint_iff.mpr ht⟩, fun ⟨hd, ht⟩ ↦ ⟨hd, ht.eq_top⟩⟩ @[simp] theorem isInternal_ne_bot_iff {A : ι → Submodule R M} : IsInternal (fun i : {i // A i ≠ ⊥} ↦ A i) ↔ IsInternal A := by simp only [isInternal_submodule_iff_independent_and_iSup_eq_top] exact Iff.and CompleteLattice.independent_ne_bot_iff_independent <| by simp lemma isInternal_biSup_submodule_of_independent {A : ι → Submodule R M} (s : Set ι) (h : CompleteLattice.Independent <| fun i : s ↦ A i) : IsInternal <| fun (i : s) ↦ (A i).comap (⨆ i ∈ s, A i).subtype := by refine (isInternal_submodule_iff_independent_and_iSup_eq_top _).mpr ⟨?_, by simp [iSup_subtype]⟩ let p := ⨆ i ∈ s, A i have hp : ∀ i ∈ s, A i ≤ p := fun i hi ↦ le_biSup A hi let e : Submodule R p ≃o Set.Iic p := p.mapIic suffices (e ∘ fun i : s ↦ (A i).comap p.subtype) = fun i ↦ ⟨A i, hp i i.property⟩ by rw [← CompleteLattice.independent_map_orderIso_iff e, this] exact CompleteLattice.independent_of_independent_coe_Iic_comp h ext i m change m ∈ ((A i).comap p.subtype).map p.subtype ↔ _ rw [Submodule.map_comap_subtype, inf_of_le_right (hp i i.property)] /-! Now copy the lemmas for subgroup and submonoids. -/ theorem IsInternal.addSubmonoid_independent {M : Type*} [AddCommMonoid M] {A : ι → AddSubmonoid M} (h : IsInternal A) : CompleteLattice.Independent A := CompleteLattice.independent_of_dfinsupp_sumAddHom_injective _ h.injective theorem IsInternal.addSubgroup_independent {M : Type*} [AddCommGroup M] {A : ι → AddSubgroup M} (h : IsInternal A) : CompleteLattice.Independent A := CompleteLattice.independent_of_dfinsupp_sumAddHom_injective' _ h.injective end Ring end Submodule end DirectSum
Algebra\DirectSum\Ring.lean
/- Copyright (c) 2021 Eric Wieser. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Eric Wieser -/ import Mathlib.Algebra.GradedMonoid import Mathlib.Algebra.DirectSum.Basic /-! # Additively-graded multiplicative structures on `⨁ i, A i` This module provides a set of heterogeneous typeclasses for defining a multiplicative structure over `⨁ i, A i` such that `(*) : A i → A j → A (i + j)`; that is to say, `A` forms an additively-graded ring. The typeclasses are: * `DirectSum.GNonUnitalNonAssocSemiring A` * `DirectSum.GSemiring A` * `DirectSum.GRing A` * `DirectSum.GCommSemiring A` * `DirectSum.GCommRing A` Respectively, these imbue the external direct sum `⨁ i, A i` with: * `DirectSum.nonUnitalNonAssocSemiring`, `DirectSum.nonUnitalNonAssocRing` * `DirectSum.semiring` * `DirectSum.ring` * `DirectSum.commSemiring` * `DirectSum.commRing` the base ring `A 0` with: * `DirectSum.GradeZero.nonUnitalNonAssocSemiring`, `DirectSum.GradeZero.nonUnitalNonAssocRing` * `DirectSum.GradeZero.semiring` * `DirectSum.GradeZero.ring` * `DirectSum.GradeZero.commSemiring` * `DirectSum.GradeZero.commRing` and the `i`th grade `A i` with `A 0`-actions (`•`) defined as left-multiplication: * `DirectSum.GradeZero.smul (A 0)`, `DirectSum.GradeZero.smulWithZero (A 0)` * `DirectSum.GradeZero.module (A 0)` * (nothing) * (nothing) * (nothing) Note that in the presence of these instances, `⨁ i, A i` itself inherits an `A 0`-action. `DirectSum.ofZeroRingHom : A 0 →+* ⨁ i, A i` provides `DirectSum.of A 0` as a ring homomorphism. `DirectSum.toSemiring` extends `DirectSum.toAddMonoid` to produce a `RingHom`. ## Direct sums of subobjects Additionally, this module provides helper functions to construct `GSemiring` and `GCommSemiring` instances for: * `A : ι → Submonoid S`: `DirectSum.GSemiring.ofAddSubmonoids`, `DirectSum.GCommSemiring.ofAddSubmonoids`. * `A : ι → Subgroup S`: `DirectSum.GSemiring.ofAddSubgroups`, `DirectSum.GCommSemiring.ofAddSubgroups`. * `A : ι → Submodule S`: `DirectSum.GSemiring.ofSubmodules`, `DirectSum.GCommSemiring.ofSubmodules`. If `CompleteLattice.independent (Set.range A)`, these provide a gradation of `⨆ i, A i`, and the mapping `⨁ i, A i →+ ⨆ i, A i` can be obtained as `DirectSum.toMonoid (fun i ↦ AddSubmonoid.inclusion <| le_iSup A i)`. ## Tags graded ring, filtered ring, direct sum, add_submonoid -/ variable {ι : Type*} [DecidableEq ι] namespace DirectSum open DirectSum /-! ### Typeclasses -/ section Defs variable (A : ι → Type*) /-- A graded version of `NonUnitalNonAssocSemiring`. -/ class GNonUnitalNonAssocSemiring [Add ι] [∀ i, AddCommMonoid (A i)] extends GradedMonoid.GMul A where /-- Multiplication from the right with any graded component's zero vanishes. -/ mul_zero : ∀ {i j} (a : A i), mul a (0 : A j) = 0 /-- Multiplication from the left with any graded component's zero vanishes. -/ zero_mul : ∀ {i j} (b : A j), mul (0 : A i) b = 0 /-- Multiplication from the right between graded components distributes with respect to addition. -/ mul_add : ∀ {i j} (a : A i) (b c : A j), mul a (b + c) = mul a b + mul a c /-- Multiplication from the left between graded components distributes with respect to addition. -/ add_mul : ∀ {i j} (a b : A i) (c : A j), mul (a + b) c = mul a c + mul b c end Defs section Defs variable (A : ι → Type*) /-- A graded version of `Semiring`. -/ class GSemiring [AddMonoid ι] [∀ i, AddCommMonoid (A i)] extends GNonUnitalNonAssocSemiring A, GradedMonoid.GMonoid A where /-- The canonical map from ℕ to the zeroth component of a graded semiring. -/ natCast : ℕ → A 0 /-- The canonical map from ℕ to a graded semiring respects zero. -/ natCast_zero : natCast 0 = 0 /-- The canonical map from ℕ to a graded semiring respects successors. -/ natCast_succ : ∀ n : ℕ, natCast (n + 1) = natCast n + GradedMonoid.GOne.one /-- A graded version of `CommSemiring`. -/ class GCommSemiring [AddCommMonoid ι] [∀ i, AddCommMonoid (A i)] extends GSemiring A, GradedMonoid.GCommMonoid A /-- A graded version of `Ring`. -/ class GRing [AddMonoid ι] [∀ i, AddCommGroup (A i)] extends GSemiring A where /-- The canonical map from ℤ to the zeroth component of a graded ring. -/ intCast : ℤ → A 0 /-- The canonical map from ℤ to a graded ring extends the canonical map from ℕ to the underlying graded semiring. -/ intCast_ofNat : ∀ n : ℕ, intCast n = natCast n /-- On negative integers, the canonical map from ℤ to a graded ring is the negative extension of the canonical map from ℕ to the underlying graded semiring. -/ -- Porting note: -(n+1) -> Int.negSucc intCast_negSucc_ofNat : ∀ n : ℕ, intCast (Int.negSucc n) = -natCast (n + 1 : ℕ) /-- A graded version of `CommRing`. -/ class GCommRing [AddCommMonoid ι] [∀ i, AddCommGroup (A i)] extends GRing A, GCommSemiring A end Defs theorem of_eq_of_gradedMonoid_eq {A : ι → Type*} [∀ i : ι, AddCommMonoid (A i)] {i j : ι} {a : A i} {b : A j} (h : GradedMonoid.mk i a = GradedMonoid.mk j b) : DirectSum.of A i a = DirectSum.of A j b := DFinsupp.single_eq_of_sigma_eq h variable (A : ι → Type*) /-! ### Instances for `⨁ i, A i` -/ section One variable [Zero ι] [GradedMonoid.GOne A] [∀ i, AddCommMonoid (A i)] instance : One (⨁ i, A i) where one := DirectSum.of A 0 GradedMonoid.GOne.one theorem one_def : 1 = DirectSum.of A 0 GradedMonoid.GOne.one := rfl end One section Mul variable [Add ι] [∀ i, AddCommMonoid (A i)] [GNonUnitalNonAssocSemiring A] open AddMonoidHom (flip_apply coe_comp compHom) /-- The piecewise multiplication from the `Mul` instance, as a bundled homomorphism. -/ @[simps] def gMulHom {i j} : A i →+ A j →+ A (i + j) where toFun a := { toFun := fun b => GradedMonoid.GMul.mul a b map_zero' := GNonUnitalNonAssocSemiring.mul_zero _ map_add' := GNonUnitalNonAssocSemiring.mul_add _ } map_zero' := AddMonoidHom.ext fun a => GNonUnitalNonAssocSemiring.zero_mul a map_add' _ _ := AddMonoidHom.ext fun _ => GNonUnitalNonAssocSemiring.add_mul _ _ _ /-- The multiplication from the `Mul` instance, as a bundled homomorphism. -/ -- See note [non-reducible instance] @[reducible] def mulHom : (⨁ i, A i) →+ (⨁ i, A i) →+ ⨁ i, A i := DirectSum.toAddMonoid fun _ => AddMonoidHom.flip <| DirectSum.toAddMonoid fun _ => AddMonoidHom.flip <| (DirectSum.of A _).compHom.comp <| gMulHom A instance instMul : Mul (⨁ i, A i) where mul := fun a b => mulHom A a b instance : NonUnitalNonAssocSemiring (⨁ i, A i) := { (inferInstance : AddCommMonoid _) with zero_mul := fun _ => by simp only [Mul.mul, HMul.hMul, map_zero, AddMonoidHom.zero_apply] mul_zero := fun _ => by simp only [Mul.mul, HMul.hMul, AddMonoidHom.map_zero] left_distrib := fun _ _ _ => by simp only [Mul.mul, HMul.hMul, AddMonoidHom.map_add] right_distrib := fun _ _ _ => by simp only [Mul.mul, HMul.hMul, AddMonoidHom.map_add, AddMonoidHom.add_apply] } variable {A} theorem mulHom_apply (a b : ⨁ i, A i) : mulHom A a b = a * b := rfl theorem mulHom_of_of {i j} (a : A i) (b : A j) : mulHom A (of A i a) (of A j b) = of A (i + j) (GradedMonoid.GMul.mul a b) := by unfold mulHom simp only [toAddMonoid_of, flip_apply, coe_comp, Function.comp_apply] rfl theorem of_mul_of {i j} (a : A i) (b : A j) : of A i a * of A j b = of _ (i + j) (GradedMonoid.GMul.mul a b) := mulHom_of_of a b end Mul section Semiring variable [∀ i, AddCommMonoid (A i)] [AddMonoid ι] [GSemiring A] open AddMonoidHom (flipHom coe_comp compHom flip_apply) private nonrec theorem one_mul (x : ⨁ i, A i) : 1 * x = x := by suffices mulHom A One.one = AddMonoidHom.id (⨁ i, A i) from DFunLike.congr_fun this x apply addHom_ext; intro i xi simp only [One.one] rw [mulHom_of_of] exact of_eq_of_gradedMonoid_eq (one_mul <| GradedMonoid.mk i xi) -- Porting note (#11083): `suffices` is very slow here. private nonrec theorem mul_one (x : ⨁ i, A i) : x * 1 = x := by suffices (mulHom A).flip One.one = AddMonoidHom.id (⨁ i, A i) from DFunLike.congr_fun this x apply addHom_ext; intro i xi simp only [One.one] rw [flip_apply, mulHom_of_of] exact of_eq_of_gradedMonoid_eq (mul_one <| GradedMonoid.mk i xi) /- Porting note: Some auxiliary statements were needed in the proof of the `suffices`, otherwise would timeout -/ private theorem mul_assoc (a b c : ⨁ i, A i) : a * b * c = a * (b * c) := by -- (`fun a b c => a * b * c` as a bundled hom) = (`fun a b c => a * (b * c)` as a bundled hom) suffices (mulHom A).compHom.comp (mulHom A) = (AddMonoidHom.compHom flipHom <| (mulHom A).flip.compHom.comp (mulHom A)).flip by have sol := DFunLike.congr_fun (DFunLike.congr_fun (DFunLike.congr_fun this a) b) c have aux : ∀ a b, (mulHom A) a b = a * b := fun _ _ ↦ rfl simp only [coe_comp, Function.comp_apply, AddMonoidHom.compHom_apply_apply, aux, flip_apply, AddMonoidHom.flipHom_apply] at sol exact sol ext ai ax bi bx ci cx dsimp only [coe_comp, Function.comp_apply, AddMonoidHom.compHom_apply_apply, flip_apply, AddMonoidHom.flipHom_apply] simp_rw [mulHom_of_of] exact of_eq_of_gradedMonoid_eq (_root_.mul_assoc (GradedMonoid.mk ai ax) ⟨bi, bx⟩ ⟨ci, cx⟩) instance instNatCast : NatCast (⨁ i, A i) where natCast := fun n => of _ _ (GSemiring.natCast n) /-- The `Semiring` structure derived from `GSemiring A`. -/ instance semiring : Semiring (⨁ i, A i) := { (inferInstance : NonUnitalNonAssocSemiring _) with one_mul := one_mul A mul_one := mul_one A mul_assoc := mul_assoc A toNatCast := instNatCast _ natCast_zero := by simp only [NatCast.natCast, GSemiring.natCast_zero, map_zero] natCast_succ := fun n => by simp_rw [NatCast.natCast, GSemiring.natCast_succ] rw [map_add] rfl } theorem ofPow {i} (a : A i) (n : ℕ) : of _ i a ^ n = of _ (n • i) (GradedMonoid.GMonoid.gnpow _ a) := by induction' n with n n_ih · exact of_eq_of_gradedMonoid_eq (pow_zero <| GradedMonoid.mk _ a).symm · rw [pow_succ, n_ih, of_mul_of] exact of_eq_of_gradedMonoid_eq (pow_succ (GradedMonoid.mk _ a) n).symm theorem ofList_dProd {α} (l : List α) (fι : α → ι) (fA : ∀ a, A (fι a)) : of A _ (l.dProd fι fA) = (l.map fun a => of A (fι a) (fA a)).prod := by induction' l with head tail · simp only [List.map_nil, List.prod_nil, List.dProd_nil] rfl · rename_i ih simp only [List.map_cons, List.prod_cons, List.dProd_cons, ← ih] rw [DirectSum.of_mul_of (fA head)] rfl theorem list_prod_ofFn_of_eq_dProd (n : ℕ) (fι : Fin n → ι) (fA : ∀ a, A (fι a)) : (List.ofFn fun a => of A (fι a) (fA a)).prod = of A _ ((List.finRange n).dProd fι fA) := by rw [List.ofFn_eq_map, ofList_dProd] theorem mul_eq_dfinsupp_sum [∀ (i : ι) (x : A i), Decidable (x ≠ 0)] (a a' : ⨁ i, A i) : a * a' = a.sum fun i ai => a'.sum fun j aj => DirectSum.of _ _ <| GradedMonoid.GMul.mul ai aj := by change mulHom _ a a' = _ -- Porting note: I have no idea how the proof from ml3 worked it used to be -- simpa only [mul_hom, to_add_monoid, dfinsupp.lift_add_hom_apply, dfinsupp.sum_add_hom_apply, -- add_monoid_hom.dfinsupp_sum_apply, flip_apply, add_monoid_hom.dfinsupp_sum_add_hom_apply], rw [mulHom, toAddMonoid, DFinsupp.liftAddHom_apply] -- This used to be `rw`, but we need `erw` after leanprover/lean4#2644 erw [DFinsupp.sumAddHom_apply] rw [AddMonoidHom.dfinsupp_sum_apply] apply congrArg _ funext x simp_rw [flip_apply] erw [DFinsupp.sumAddHom_apply] simp only [gMulHom, AddMonoidHom.dfinsupp_sum_apply, flip_apply, coe_comp, AddMonoidHom.coe_mk, ZeroHom.coe_mk, Function.comp_apply, AddMonoidHom.compHom_apply_apply] /-- A heavily unfolded version of the definition of multiplication -/ theorem mul_eq_sum_support_ghas_mul [∀ (i : ι) (x : A i), Decidable (x ≠ 0)] (a a' : ⨁ i, A i) : a * a' = ∑ ij ∈ DFinsupp.support a ×ˢ DFinsupp.support a', DirectSum.of _ _ (GradedMonoid.GMul.mul (a ij.fst) (a' ij.snd)) := by simp only [mul_eq_dfinsupp_sum, DFinsupp.sum, Finset.sum_product] end Semiring section CommSemiring variable [∀ i, AddCommMonoid (A i)] [AddCommMonoid ι] [GCommSemiring A] private theorem mul_comm (a b : ⨁ i, A i) : a * b = b * a := by suffices mulHom A = (mulHom A).flip by rw [← mulHom_apply, this, AddMonoidHom.flip_apply, mulHom_apply] apply addHom_ext; intro ai ax; apply addHom_ext; intro bi bx rw [AddMonoidHom.flip_apply, mulHom_of_of, mulHom_of_of] exact of_eq_of_gradedMonoid_eq (GCommSemiring.mul_comm ⟨ai, ax⟩ ⟨bi, bx⟩) /-- The `CommSemiring` structure derived from `GCommSemiring A`. -/ instance commSemiring : CommSemiring (⨁ i, A i) := { DirectSum.semiring A with mul_comm := mul_comm A } end CommSemiring section NonUnitalNonAssocRing variable [∀ i, AddCommGroup (A i)] [Add ι] [GNonUnitalNonAssocSemiring A] /-- The `Ring` derived from `GSemiring A`. -/ instance nonAssocRing : NonUnitalNonAssocRing (⨁ i, A i) := { (inferInstance : NonUnitalNonAssocSemiring (⨁ i, A i)), (inferInstance : AddCommGroup (⨁ i, A i)) with } end NonUnitalNonAssocRing section Ring variable [∀ i, AddCommGroup (A i)] [AddMonoid ι] [GRing A] -- Porting note: overspecified fields in ml4 /-- The `Ring` derived from `GSemiring A`. -/ instance ring : Ring (⨁ i, A i) := { DirectSum.semiring A, (inferInstance : AddCommGroup (⨁ i, A i)) with toIntCast.intCast := fun z => of A 0 <| (GRing.intCast z) intCast_ofNat := fun _ => congrArg (of A 0) <| GRing.intCast_ofNat _ intCast_negSucc := fun _ => (congrArg (of A 0) <| GRing.intCast_negSucc_ofNat _).trans <| map_neg _ _} end Ring section CommRing variable [∀ i, AddCommGroup (A i)] [AddCommMonoid ι] [GCommRing A] /-- The `CommRing` derived from `GCommSemiring A`. -/ instance commRing : CommRing (⨁ i, A i) := { DirectSum.ring A, DirectSum.commSemiring A with } end CommRing /-! ### Instances for `A 0` The various `G*` instances are enough to promote the `AddCommMonoid (A 0)` structure to various types of multiplicative structure. -/ section GradeZero section One variable [Zero ι] [GradedMonoid.GOne A] [∀ i, AddCommMonoid (A i)] @[simp] theorem of_zero_one : of _ 0 (1 : A 0) = 1 := rfl end One section Mul variable [AddZeroClass ι] [∀ i, AddCommMonoid (A i)] [GNonUnitalNonAssocSemiring A] @[simp] theorem of_zero_smul {i} (a : A 0) (b : A i) : of _ _ (a • b) = of _ _ a * of _ _ b := (of_eq_of_gradedMonoid_eq (GradedMonoid.mk_zero_smul a b)).trans (of_mul_of _ _).symm @[simp] theorem of_zero_mul (a b : A 0) : of _ 0 (a * b) = of _ 0 a * of _ 0 b := of_zero_smul A a b instance GradeZero.nonUnitalNonAssocSemiring : NonUnitalNonAssocSemiring (A 0) := Function.Injective.nonUnitalNonAssocSemiring (of A 0) DFinsupp.single_injective (of A 0).map_zero (of A 0).map_add (of_zero_mul A) (map_nsmul _) instance GradeZero.smulWithZero (i : ι) : SMulWithZero (A 0) (A i) := by letI := SMulWithZero.compHom (⨁ i, A i) (of A 0).toZeroHom exact Function.Injective.smulWithZero (of A i).toZeroHom DFinsupp.single_injective (of_zero_smul A) end Mul section Semiring variable [∀ i, AddCommMonoid (A i)] [AddMonoid ι] [GSemiring A] @[simp] theorem of_zero_pow (a : A 0) : ∀ n : ℕ, of A 0 (a ^ n) = of A 0 a ^ n | 0 => by rw [pow_zero, pow_zero, DirectSum.of_zero_one] -- Porting note: Lean doesn't think this terminates if we only use `of_zero_pow` alone | n + 1 => by rw [pow_succ, pow_succ, of_zero_mul, of_zero_pow _ n] instance : NatCast (A 0) := ⟨GSemiring.natCast⟩ -- TODO: These could be replaced by the general lemmas for `AddMonoidHomClass` (`map_natCast'` and -- `map_ofNat'`) if those were marked `@[simp low]`. @[simp] theorem of_natCast (n : ℕ) : of A 0 n = n := rfl -- See note [no_index around OfNat.ofNat] @[simp] theorem of_zero_ofNat (n : ℕ) [n.AtLeastTwo] : of A 0 (no_index (OfNat.ofNat n)) = OfNat.ofNat n := of_natCast A n /-- The `Semiring` structure derived from `GSemiring A`. -/ instance GradeZero.semiring : Semiring (A 0) := Function.Injective.semiring (of A 0) DFinsupp.single_injective (of A 0).map_zero (of_zero_one A) (of A 0).map_add (of_zero_mul A) (fun _ _ ↦ (of A 0).map_nsmul _ _) (fun _ _ => of_zero_pow _ _ _) (of_natCast A) /-- `of A 0` is a `RingHom`, using the `DirectSum.GradeZero.semiring` structure. -/ def ofZeroRingHom : A 0 →+* ⨁ i, A i := { of _ 0 with map_one' := of_zero_one A map_mul' := of_zero_mul A } /-- Each grade `A i` derives an `A 0`-module structure from `GSemiring A`. Note that this results in an overall `Module (A 0) (⨁ i, A i)` structure via `DirectSum.module`. -/ instance GradeZero.module {i} : Module (A 0) (A i) := letI := Module.compHom (⨁ i, A i) (ofZeroRingHom A) DFinsupp.single_injective.module (A 0) (of A i) fun a => of_zero_smul A a end Semiring section CommSemiring variable [∀ i, AddCommMonoid (A i)] [AddCommMonoid ι] [GCommSemiring A] /-- The `CommSemiring` structure derived from `GCommSemiring A`. -/ instance GradeZero.commSemiring : CommSemiring (A 0) := Function.Injective.commSemiring (of A 0) DFinsupp.single_injective (of A 0).map_zero (of_zero_one A) (of A 0).map_add (of_zero_mul A) (fun _ _ ↦ map_nsmul _ _ _) (fun _ _ => of_zero_pow _ _ _) (of_natCast A) end CommSemiring section Ring variable [∀ i, AddCommGroup (A i)] [AddZeroClass ι] [GNonUnitalNonAssocSemiring A] /-- The `NonUnitalNonAssocRing` derived from `GNonUnitalNonAssocSemiring A`. -/ instance GradeZero.nonUnitalNonAssocRing : NonUnitalNonAssocRing (A 0) := Function.Injective.nonUnitalNonAssocRing (of A 0) DFinsupp.single_injective (of A 0).map_zero (of A 0).map_add (of_zero_mul A) (of A 0).map_neg (of A 0).map_sub (fun _ _ ↦ map_nsmul _ _ _) (fun _ _ ↦ map_zsmul _ _ _) end Ring section Ring variable [∀ i, AddCommGroup (A i)] [AddMonoid ι] [GRing A] instance : IntCast (A 0) := ⟨GRing.intCast⟩ @[simp] theorem of_intCast (n : ℤ) : of A 0 n = n := by rfl /-- The `Ring` derived from `GSemiring A`. -/ instance GradeZero.ring : Ring (A 0) := Function.Injective.ring (of A 0) DFinsupp.single_injective (of A 0).map_zero (of_zero_one A) (of A 0).map_add (of_zero_mul A) (of A 0).map_neg (of A 0).map_sub (fun _ _ ↦ map_nsmul _ _ _) (fun _ _ ↦ map_zsmul _ _ _) (fun _ _ => of_zero_pow _ _ _) (of_natCast A) (of_intCast A) end Ring section CommRing variable [∀ i, AddCommGroup (A i)] [AddCommMonoid ι] [GCommRing A] /-- The `CommRing` derived from `GCommSemiring A`. -/ instance GradeZero.commRing : CommRing (A 0) := Function.Injective.commRing (of A 0) DFinsupp.single_injective (of A 0).map_zero (of_zero_one A) (of A 0).map_add (of_zero_mul A) (of A 0).map_neg (of A 0).map_sub (fun _ _ ↦ map_nsmul _ _ _) (fun _ _ ↦ map_zsmul _ _ _) (fun _ _ => of_zero_pow _ _ _) (of_natCast A) (of_intCast A) end CommRing end GradeZero section ToSemiring variable {R : Type*} [∀ i, AddCommMonoid (A i)] [AddMonoid ι] [GSemiring A] [Semiring R] variable {A} /-- If two ring homomorphisms from `⨁ i, A i` are equal on each `of A i y`, then they are equal. See note [partially-applied ext lemmas]. -/ @[ext] theorem ringHom_ext' ⦃F G : (⨁ i, A i) →+* R⦄ (h : ∀ i, (↑F : _ →+ R).comp (of A i) = (↑G : _ →+ R).comp (of A i)) : F = G := RingHom.coe_addMonoidHom_injective <| DirectSum.addHom_ext' h /-- Two `RingHom`s out of a direct sum are equal if they agree on the generators. -/ theorem ringHom_ext ⦃f g : (⨁ i, A i) →+* R⦄ (h : ∀ i x, f (of A i x) = g (of A i x)) : f = g := ringHom_ext' fun i => AddMonoidHom.ext <| h i /-- A family of `AddMonoidHom`s preserving `DirectSum.One.one` and `DirectSum.Mul.mul` describes a `RingHom`s on `⨁ i, A i`. This is a stronger version of `DirectSum.toMonoid`. Of particular interest is the case when `A i` are bundled subojects, `f` is the family of coercions such as `AddSubmonoid.subtype (A i)`, and the `[GSemiring A]` structure originates from `DirectSum.gsemiring.ofAddSubmonoids`, in which case the proofs about `GOne` and `GMul` can be discharged by `rfl`. -/ @[simps] def toSemiring (f : ∀ i, A i →+ R) (hone : f _ GradedMonoid.GOne.one = 1) (hmul : ∀ {i j} (ai : A i) (aj : A j), f _ (GradedMonoid.GMul.mul ai aj) = f _ ai * f _ aj) : (⨁ i, A i) →+* R := { toAddMonoid f with toFun := toAddMonoid f map_one' := by change (toAddMonoid f) (of _ 0 _) = 1 rw [toAddMonoid_of] exact hone map_mul' := by rw [(toAddMonoid f).map_mul_iff] refine DirectSum.addHom_ext' (fun xi ↦ AddMonoidHom.ext (fun xv ↦ ?_)) refine DirectSum.addHom_ext' (fun yi ↦ AddMonoidHom.ext (fun yv ↦ ?_)) show toAddMonoid f (of A xi xv * of A yi yv) = toAddMonoid f (of A xi xv) * toAddMonoid f (of A yi yv) simp_rw [of_mul_of, toAddMonoid_of] exact hmul _ _ } -- Porting note (#10618): removed @[simp] as simp can prove this theorem toSemiring_of (f : ∀ i, A i →+ R) (hone hmul) (i : ι) (x : A i) : toSemiring f hone hmul (of _ i x) = f _ x := toAddMonoid_of f i x @[simp] theorem toSemiring_coe_addMonoidHom (f : ∀ i, A i →+ R) (hone hmul) : (toSemiring f hone hmul : (⨁ i, A i) →+ R) = toAddMonoid f := rfl /-- Families of `AddMonoidHom`s preserving `DirectSum.One.one` and `DirectSum.Mul.mul` are isomorphic to `RingHom`s on `⨁ i, A i`. This is a stronger version of `DFinsupp.liftAddHom`. -/ @[simps] def liftRingHom : { f : ∀ {i}, A i →+ R // f GradedMonoid.GOne.one = 1 ∧ ∀ {i j} (ai : A i) (aj : A j), f (GradedMonoid.GMul.mul ai aj) = f ai * f aj } ≃ ((⨁ i, A i) →+* R) where toFun f := toSemiring (fun _ => f.1) f.2.1 f.2.2 invFun F := ⟨by intro i; exact (F : (⨁ i, A i) →+ R).comp (of _ i), by simp only [AddMonoidHom.comp_apply] rw [← F.map_one] rfl, by intros i j ai aj simp only [AddMonoidHom.comp_apply, AddMonoidHom.coe_coe] rw [← F.map_mul (of A i ai), of_mul_of ai]⟩ left_inv f := by ext xi xv exact toAddMonoid_of (fun _ => f.1) xi xv right_inv F := by apply RingHom.coe_addMonoidHom_injective refine DirectSum.addHom_ext' (fun xi ↦ AddMonoidHom.ext (fun xv ↦ ?_)) simp only [RingHom.coe_addMonoidHom_mk, DirectSum.toAddMonoid_of, AddMonoidHom.mk_coe, AddMonoidHom.comp_apply, toSemiring_coe_addMonoidHom] end ToSemiring end DirectSum /-! ### Concrete instances -/ section Uniform variable (ι) /-- A direct sum of copies of a `Semiring` inherits the multiplication structure. -/ instance NonUnitalNonAssocSemiring.directSumGNonUnitalNonAssocSemiring {R : Type*} [AddMonoid ι] [NonUnitalNonAssocSemiring R] : DirectSum.GNonUnitalNonAssocSemiring fun _ : ι => R := { -- Porting note: removed Mul.gMul ι with and we seem ok mul_zero := mul_zero zero_mul := zero_mul mul_add := mul_add add_mul := add_mul } /-- A direct sum of copies of a `Semiring` inherits the multiplication structure. -/ instance Semiring.directSumGSemiring {R : Type*} [AddMonoid ι] [Semiring R] : DirectSum.GSemiring fun _ : ι => R := { NonUnitalNonAssocSemiring.directSumGNonUnitalNonAssocSemiring ι, Monoid.gMonoid ι with natCast := fun n => n natCast_zero := Nat.cast_zero natCast_succ := Nat.cast_succ } open DirectSum -- To check `Mul.gmul_mul` matches example {R : Type*} [AddMonoid ι] [Semiring R] (i j : ι) (a b : R) : (DirectSum.of _ i a * DirectSum.of _ j b : ⨁ _, R) = DirectSum.of _ (i + j) (a * b) := by rw [DirectSum.of_mul_of, Mul.gMul_mul] /-- A direct sum of copies of a `CommSemiring` inherits the commutative multiplication structure. -/ instance CommSemiring.directSumGCommSemiring {R : Type*} [AddCommMonoid ι] [CommSemiring R] : DirectSum.GCommSemiring fun _ : ι => R := { CommMonoid.gCommMonoid ι, Semiring.directSumGSemiring ι with } end Uniform
Algebra\Divisibility\Basic.lean
/- Copyright (c) 2014 Jeremy Avigad. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Jeremy Avigad, Leonardo de Moura, Floris van Doorn, Amelia Livingston, Yury Kudryashov, Neil Strickland, Aaron Anderson -/ import Mathlib.Algebra.Group.Basic import Mathlib.Algebra.Group.Hom.Defs import Mathlib.Tactic.Common /-! # Divisibility This file defines the basics of the divisibility relation in the context of `(Comm)` `Monoid`s. ## Main definitions * `semigroupDvd` ## Implementation notes The divisibility relation is defined for all monoids, and as such, depends on the order of multiplication if the monoid is not commutative. There are two possible conventions for divisibility in the noncommutative context, and this relation follows the convention for ordinals, so `a | b` is defined as `∃ c, b = a * c`. ## Tags divisibility, divides -/ variable {α : Type*} section Semigroup variable [Semigroup α] {a b c : α} /-- There are two possible conventions for divisibility, which coincide in a `CommMonoid`. This matches the convention for ordinals. -/ instance (priority := 100) semigroupDvd : Dvd α := Dvd.mk fun a b => ∃ c, b = a * c -- TODO: this used to not have `c` explicit, but that seems to be important -- for use with tactics, similar to `Exists.intro` theorem Dvd.intro (c : α) (h : a * c = b) : a ∣ b := Exists.intro c h.symm alias dvd_of_mul_right_eq := Dvd.intro theorem exists_eq_mul_right_of_dvd (h : a ∣ b) : ∃ c, b = a * c := h theorem dvd_def : a ∣ b ↔ ∃ c, b = a * c := Iff.rfl alias dvd_iff_exists_eq_mul_right := dvd_def theorem Dvd.elim {P : Prop} {a b : α} (H₁ : a ∣ b) (H₂ : ∀ c, b = a * c → P) : P := Exists.elim H₁ H₂ attribute [local simp] mul_assoc mul_comm mul_left_comm @[trans] theorem dvd_trans : a ∣ b → b ∣ c → a ∣ c | ⟨d, h₁⟩, ⟨e, h₂⟩ => ⟨d * e, h₁ ▸ h₂.trans <| mul_assoc a d e⟩ alias Dvd.dvd.trans := dvd_trans /-- Transitivity of `|` for use in `calc` blocks. -/ instance : IsTrans α Dvd.dvd := ⟨fun _ _ _ => dvd_trans⟩ @[simp] theorem dvd_mul_right (a b : α) : a ∣ a * b := Dvd.intro b rfl theorem dvd_mul_of_dvd_left (h : a ∣ b) (c : α) : a ∣ b * c := h.trans (dvd_mul_right b c) alias Dvd.dvd.mul_right := dvd_mul_of_dvd_left theorem dvd_of_mul_right_dvd (h : a * b ∣ c) : a ∣ c := (dvd_mul_right a b).trans h section map_dvd variable {M N : Type*} theorem map_dvd [Semigroup M] [Semigroup N] {F : Type*} [FunLike F M N] [MulHomClass F M N] (f : F) {a b} : a ∣ b → f a ∣ f b | ⟨c, h⟩ => ⟨f c, h.symm ▸ map_mul f a c⟩ theorem MulHom.map_dvd [Semigroup M] [Semigroup N] (f : M →ₙ* N) {a b} : a ∣ b → f a ∣ f b := _root_.map_dvd f theorem MonoidHom.map_dvd [Monoid M] [Monoid N] (f : M →* N) {a b} : a ∣ b → f a ∣ f b := _root_.map_dvd f end map_dvd /-- An element `a` in a semigroup is primal if whenever `a` is a divisor of `b * c`, it can be factored as the product of a divisor of `b` and a divisor of `c`. -/ def IsPrimal (a : α) : Prop := ∀ ⦃b c⦄, a ∣ b * c → ∃ a₁ a₂, a₁ ∣ b ∧ a₂ ∣ c ∧ a = a₁ * a₂ variable (α) in /-- A monoid is a decomposition monoid if every element is primal. An integral domain whose multiplicative monoid is a decomposition monoid, is called a pre-Schreier domain; it is a Schreier domain if it is moreover integrally closed. -/ @[mk_iff] class DecompositionMonoid : Prop where primal (a : α) : IsPrimal a theorem exists_dvd_and_dvd_of_dvd_mul [DecompositionMonoid α] {b c a : α} (H : a ∣ b * c) : ∃ a₁ a₂, a₁ ∣ b ∧ a₂ ∣ c ∧ a = a₁ * a₂ := DecompositionMonoid.primal a H end Semigroup section Monoid variable [Monoid α] {a b c : α} {m n : ℕ} @[refl, simp] theorem dvd_refl (a : α) : a ∣ a := Dvd.intro 1 (mul_one a) theorem dvd_rfl : ∀ {a : α}, a ∣ a := fun {a} => dvd_refl a instance : IsRefl α (· ∣ ·) := ⟨dvd_refl⟩ theorem one_dvd (a : α) : 1 ∣ a := Dvd.intro a (one_mul a) theorem dvd_of_eq (h : a = b) : a ∣ b := by rw [h] alias Eq.dvd := dvd_of_eq lemma pow_dvd_pow (a : α) (h : m ≤ n) : a ^ m ∣ a ^ n := ⟨a ^ (n - m), by rw [← pow_add, Nat.add_comm, Nat.sub_add_cancel h]⟩ lemma dvd_pow (hab : a ∣ b) : ∀ {n : ℕ} (_ : n ≠ 0), a ∣ b ^ n | 0, hn => (hn rfl).elim | n + 1, _ => by rw [pow_succ']; exact hab.mul_right _ alias Dvd.dvd.pow := dvd_pow lemma dvd_pow_self (a : α) {n : ℕ} (hn : n ≠ 0) : a ∣ a ^ n := dvd_rfl.pow hn theorem mul_dvd_mul_left (a : α) (h : b ∣ c) : a * b ∣ a * c := by obtain ⟨d, rfl⟩ := h use d rw [mul_assoc] end Monoid section CommSemigroup variable [CommSemigroup α] {a b c : α} theorem Dvd.intro_left (c : α) (h : c * a = b) : a ∣ b := Dvd.intro c (by rw [mul_comm] at h; apply h) alias dvd_of_mul_left_eq := Dvd.intro_left theorem exists_eq_mul_left_of_dvd (h : a ∣ b) : ∃ c, b = c * a := Dvd.elim h fun c => fun H1 : b = a * c => Exists.intro c (Eq.trans H1 (mul_comm a c)) theorem dvd_iff_exists_eq_mul_left : a ∣ b ↔ ∃ c, b = c * a := ⟨exists_eq_mul_left_of_dvd, by rintro ⟨c, rfl⟩ exact ⟨c, mul_comm _ _⟩⟩ theorem Dvd.elim_left {P : Prop} (h₁ : a ∣ b) (h₂ : ∀ c, b = c * a → P) : P := Exists.elim (exists_eq_mul_left_of_dvd h₁) fun c => fun h₃ : b = c * a => h₂ c h₃ @[simp] theorem dvd_mul_left (a b : α) : a ∣ b * a := Dvd.intro b (mul_comm a b) theorem dvd_mul_of_dvd_right (h : a ∣ b) (c : α) : a ∣ c * b := by rw [mul_comm]; exact h.mul_right _ alias Dvd.dvd.mul_left := dvd_mul_of_dvd_right attribute [local simp] mul_assoc mul_comm mul_left_comm theorem mul_dvd_mul : ∀ {a b c d : α}, a ∣ b → c ∣ d → a * c ∣ b * d | a, _, c, _, ⟨e, rfl⟩, ⟨f, rfl⟩ => ⟨e * f, by simp⟩ theorem dvd_of_mul_left_dvd (h : a * b ∣ c) : b ∣ c := Dvd.elim h fun d ceq => Dvd.intro (a * d) (by simp [ceq]) theorem dvd_mul [DecompositionMonoid α] {k m n : α} : k ∣ m * n ↔ ∃ d₁ d₂, d₁ ∣ m ∧ d₂ ∣ n ∧ k = d₁ * d₂ := by refine ⟨exists_dvd_and_dvd_of_dvd_mul, ?_⟩ rintro ⟨d₁, d₂, hy, hz, rfl⟩ exact mul_dvd_mul hy hz end CommSemigroup section CommMonoid variable [CommMonoid α] {a b : α} theorem mul_dvd_mul_right (h : a ∣ b) (c : α) : a * c ∣ b * c := mul_dvd_mul h (dvd_refl c) theorem pow_dvd_pow_of_dvd (h : a ∣ b) : ∀ n : ℕ, a ^ n ∣ b ^ n | 0 => by rw [pow_zero, pow_zero] | n + 1 => by rw [pow_succ, pow_succ] exact mul_dvd_mul (pow_dvd_pow_of_dvd h n) h end CommMonoid
Algebra\Divisibility\Prod.lean
/- Copyright (c) 2023 Johan Commelin. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Johan Commelin -/ import Mathlib.Algebra.Divisibility.Basic import Mathlib.Algebra.Group.Prod import Mathlib.Tactic.Common /-! # Lemmas about the divisibility relation in product (semi)groups -/ variable {ι G₁ G₂ : Type*} {G : ι → Type*} [Semigroup G₁] [Semigroup G₂] [∀ i, Semigroup (G i)] theorem prod_dvd_iff {x y : G₁ × G₂} : x ∣ y ↔ x.1 ∣ y.1 ∧ x.2 ∣ y.2 := by cases x; cases y simp only [dvd_def, Prod.exists, Prod.mk_mul_mk, Prod.mk.injEq, exists_and_left, exists_and_right, and_self, true_and] @[simp] theorem Prod.mk_dvd_mk {x₁ y₁ : G₁} {x₂ y₂ : G₂} : (x₁, x₂) ∣ (y₁, y₂) ↔ x₁ ∣ y₁ ∧ x₂ ∣ y₂ := prod_dvd_iff instance [DecompositionMonoid G₁] [DecompositionMonoid G₂] : DecompositionMonoid (G₁ × G₂) where primal a b c h := by simp_rw [prod_dvd_iff] at h ⊢ obtain ⟨a₁, a₁', h₁, h₁', eq₁⟩ := DecompositionMonoid.primal a.1 h.1 obtain ⟨a₂, a₂', h₂, h₂', eq₂⟩ := DecompositionMonoid.primal a.2 h.2 -- aesop works here exact ⟨(a₁, a₂), (a₁', a₂'), ⟨h₁, h₂⟩, ⟨h₁', h₂'⟩, Prod.ext eq₁ eq₂⟩ theorem pi_dvd_iff {x y : ∀ i, G i} : x ∣ y ↔ ∀ i, x i ∣ y i := by simp_rw [dvd_def, Function.funext_iff, Classical.skolem]; rfl instance [∀ i, DecompositionMonoid (G i)] : DecompositionMonoid (∀ i, G i) where primal a b c h := by simp_rw [pi_dvd_iff] at h ⊢ choose a₁ a₂ h₁ h₂ eq using fun i ↦ DecompositionMonoid.primal _ (h i) exact ⟨a₁, a₂, h₁, h₂, funext eq⟩
Algebra\Divisibility\Units.lean
/- Copyright (c) 2014 Jeremy Avigad. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Jeremy Avigad, Leonardo de Moura, Floris van Doorn, Amelia Livingston, Yury Kudryashov, Neil Strickland, Aaron Anderson -/ import Mathlib.Algebra.Divisibility.Basic import Mathlib.Algebra.Group.Units /-! # Divisibility and units ## Main definition * `IsRelPrime x y`: that `x` and `y` are relatively prime, defined to mean that the only common divisors of `x` and `y` are the units. -/ variable {α : Type*} namespace Units section Monoid variable [Monoid α] {a b : α} {u : αˣ} /-- Elements of the unit group of a monoid represented as elements of the monoid divide any element of the monoid. -/ theorem coe_dvd : ↑u ∣ a := ⟨↑u⁻¹ * a, by simp⟩ /-- In a monoid, an element `a` divides an element `b` iff `a` divides all associates of `b`. -/ theorem dvd_mul_right : a ∣ b * u ↔ a ∣ b := Iff.intro (fun ⟨c, Eq⟩ ↦ ⟨c * ↑u⁻¹, by rw [← mul_assoc, ← Eq, Units.mul_inv_cancel_right]⟩) fun ⟨c, Eq⟩ ↦ Eq.symm ▸ (_root_.dvd_mul_right _ _).mul_right _ /-- In a monoid, an element `a` divides an element `b` iff all associates of `a` divide `b`. -/ theorem mul_right_dvd : a * u ∣ b ↔ a ∣ b := Iff.intro (fun ⟨c, Eq⟩ => ⟨↑u * c, Eq.trans (mul_assoc _ _ _)⟩) fun h => dvd_trans (Dvd.intro (↑u⁻¹) (by rw [mul_assoc, u.mul_inv, mul_one])) h end Monoid section CommMonoid variable [CommMonoid α] {a b : α} {u : αˣ} /-- In a commutative monoid, an element `a` divides an element `b` iff `a` divides all left associates of `b`. -/ theorem dvd_mul_left : a ∣ u * b ↔ a ∣ b := by rw [mul_comm] apply dvd_mul_right /-- In a commutative monoid, an element `a` divides an element `b` iff all left associates of `a` divide `b`. -/ theorem mul_left_dvd : ↑u * a ∣ b ↔ a ∣ b := by rw [mul_comm] apply mul_right_dvd end CommMonoid end Units namespace IsUnit section Monoid variable [Monoid α] {a b u : α} /-- Units of a monoid divide any element of the monoid. -/ @[simp] theorem dvd (hu : IsUnit u) : u ∣ a := by rcases hu with ⟨u, rfl⟩ apply Units.coe_dvd @[simp] theorem dvd_mul_right (hu : IsUnit u) : a ∣ b * u ↔ a ∣ b := by rcases hu with ⟨u, rfl⟩ apply Units.dvd_mul_right /-- In a monoid, an element a divides an element b iff all associates of `a` divide `b`. -/ @[simp] theorem mul_right_dvd (hu : IsUnit u) : a * u ∣ b ↔ a ∣ b := by rcases hu with ⟨u, rfl⟩ apply Units.mul_right_dvd theorem isPrimal (hu : IsUnit u) : IsPrimal u := fun _ _ _ ↦ ⟨u, 1, hu.dvd, one_dvd _, (mul_one u).symm⟩ end Monoid section CommMonoid variable [CommMonoid α] {a b u : α} /-- In a commutative monoid, an element `a` divides an element `b` iff `a` divides all left associates of `b`. -/ @[simp] theorem dvd_mul_left (hu : IsUnit u) : a ∣ u * b ↔ a ∣ b := by rcases hu with ⟨u, rfl⟩ apply Units.dvd_mul_left /-- In a commutative monoid, an element `a` divides an element `b` iff all left associates of `a` divide `b`. -/ @[simp] theorem mul_left_dvd (hu : IsUnit u) : u * a ∣ b ↔ a ∣ b := by rcases hu with ⟨u, rfl⟩ apply Units.mul_left_dvd end CommMonoid end IsUnit section CommMonoid variable [CommMonoid α] theorem isUnit_iff_dvd_one {x : α} : IsUnit x ↔ x ∣ 1 := ⟨IsUnit.dvd, fun ⟨y, h⟩ => ⟨⟨x, y, h.symm, by rw [h, mul_comm]⟩, rfl⟩⟩ theorem isUnit_iff_forall_dvd {x : α} : IsUnit x ↔ ∀ y, x ∣ y := isUnit_iff_dvd_one.trans ⟨fun h _ => h.trans (one_dvd _), fun h => h _⟩ theorem isUnit_of_dvd_unit {x y : α} (xy : x ∣ y) (hu : IsUnit y) : IsUnit x := isUnit_iff_dvd_one.2 <| xy.trans <| isUnit_iff_dvd_one.1 hu theorem isUnit_of_dvd_one {a : α} (h : a ∣ 1) : IsUnit (a : α) := isUnit_iff_dvd_one.mpr h theorem not_isUnit_of_not_isUnit_dvd {a b : α} (ha : ¬IsUnit a) (hb : a ∣ b) : ¬IsUnit b := mt (isUnit_of_dvd_unit hb) ha end CommMonoid section RelPrime /-- `x` and `y` are relatively prime if every common divisor is a unit. -/ def IsRelPrime [Monoid α] (x y : α) : Prop := ∀ ⦃d⦄, d ∣ x → d ∣ y → IsUnit d variable [CommMonoid α] {x y z : α} @[symm] theorem IsRelPrime.symm (H : IsRelPrime x y) : IsRelPrime y x := fun _ hx hy ↦ H hy hx theorem isRelPrime_comm : IsRelPrime x y ↔ IsRelPrime y x := ⟨IsRelPrime.symm, IsRelPrime.symm⟩ theorem isRelPrime_self : IsRelPrime x x ↔ IsUnit x := ⟨(· dvd_rfl dvd_rfl), fun hu _ _ dvd ↦ isUnit_of_dvd_unit dvd hu⟩ theorem IsUnit.isRelPrime_left (h : IsUnit x) : IsRelPrime x y := fun _ hx _ ↦ isUnit_of_dvd_unit hx h theorem IsUnit.isRelPrime_right (h : IsUnit y) : IsRelPrime x y := h.isRelPrime_left.symm theorem isRelPrime_one_left : IsRelPrime 1 x := isUnit_one.isRelPrime_left theorem isRelPrime_one_right : IsRelPrime x 1 := isUnit_one.isRelPrime_right theorem IsRelPrime.of_mul_left_left (H : IsRelPrime (x * y) z) : IsRelPrime x z := fun _ hx ↦ H (dvd_mul_of_dvd_left hx _) theorem IsRelPrime.of_mul_left_right (H : IsRelPrime (x * y) z) : IsRelPrime y z := (mul_comm x y ▸ H).of_mul_left_left theorem IsRelPrime.of_mul_right_left (H : IsRelPrime x (y * z)) : IsRelPrime x y := by rw [isRelPrime_comm] at H ⊢ exact H.of_mul_left_left theorem IsRelPrime.of_mul_right_right (H : IsRelPrime x (y * z)) : IsRelPrime x z := (mul_comm y z ▸ H).of_mul_right_left theorem IsRelPrime.of_dvd_left (h : IsRelPrime y z) (dvd : x ∣ y) : IsRelPrime x z := by obtain ⟨d, rfl⟩ := dvd; exact IsRelPrime.of_mul_left_left h theorem IsRelPrime.of_dvd_right (h : IsRelPrime z y) (dvd : x ∣ y) : IsRelPrime z x := (h.symm.of_dvd_left dvd).symm theorem IsRelPrime.isUnit_of_dvd (H : IsRelPrime x y) (d : x ∣ y) : IsUnit x := H dvd_rfl d section IsUnit variable (hu : IsUnit x) theorem isRelPrime_mul_unit_left_left : IsRelPrime (x * y) z ↔ IsRelPrime y z := ⟨IsRelPrime.of_mul_left_right, fun H _ h ↦ H (hu.dvd_mul_left.mp h)⟩ theorem isRelPrime_mul_unit_left_right : IsRelPrime y (x * z) ↔ IsRelPrime y z := by rw [isRelPrime_comm, isRelPrime_mul_unit_left_left hu, isRelPrime_comm] theorem isRelPrime_mul_unit_left : IsRelPrime (x * y) (x * z) ↔ IsRelPrime y z := by rw [isRelPrime_mul_unit_left_left hu, isRelPrime_mul_unit_left_right hu] theorem isRelPrime_mul_unit_right_left : IsRelPrime (y * x) z ↔ IsRelPrime y z := by rw [mul_comm, isRelPrime_mul_unit_left_left hu] theorem isRelPrime_mul_unit_right_right : IsRelPrime y (z * x) ↔ IsRelPrime y z := by rw [mul_comm, isRelPrime_mul_unit_left_right hu] theorem isRelPrime_mul_unit_right : IsRelPrime (y * x) (z * x) ↔ IsRelPrime y z := by rw [isRelPrime_mul_unit_right_left hu, isRelPrime_mul_unit_right_right hu] end IsUnit theorem IsRelPrime.dvd_of_dvd_mul_right_of_isPrimal (H1 : IsRelPrime x z) (H2 : x ∣ y * z) (h : IsPrimal x) : x ∣ y := by obtain ⟨a, b, ha, hb, rfl⟩ := h H2 exact (H1.of_mul_left_right.isUnit_of_dvd hb).mul_right_dvd.mpr ha theorem IsRelPrime.dvd_of_dvd_mul_left_of_isPrimal (H1 : IsRelPrime x y) (H2 : x ∣ y * z) (h : IsPrimal x) : x ∣ z := H1.dvd_of_dvd_mul_right_of_isPrimal (mul_comm y z ▸ H2) h theorem IsRelPrime.mul_dvd_of_right_isPrimal (H : IsRelPrime x y) (H1 : x ∣ z) (H2 : y ∣ z) (hy : IsPrimal y) : x * y ∣ z := by obtain ⟨w, rfl⟩ := H1 exact mul_dvd_mul_left x (H.symm.dvd_of_dvd_mul_left_of_isPrimal H2 hy) theorem IsRelPrime.mul_dvd_of_left_isPrimal (H : IsRelPrime x y) (H1 : x ∣ z) (H2 : y ∣ z) (hx : IsPrimal x) : x * y ∣ z := by rw [mul_comm]; exact H.symm.mul_dvd_of_right_isPrimal H2 H1 hx /-! `IsRelPrime` enjoys desirable properties in a decomposition monoid. See Lemma 6.3 in *On properties of square-free elements in commutative cancellative monoids*, https://doi.org/10.1007/s00233-019-10022-3. -/ variable [DecompositionMonoid α] theorem IsRelPrime.dvd_of_dvd_mul_right (H1 : IsRelPrime x z) (H2 : x ∣ y * z) : x ∣ y := H1.dvd_of_dvd_mul_right_of_isPrimal H2 (DecompositionMonoid.primal x) theorem IsRelPrime.dvd_of_dvd_mul_left (H1 : IsRelPrime x y) (H2 : x ∣ y * z) : x ∣ z := H1.dvd_of_dvd_mul_right (mul_comm y z ▸ H2) theorem IsRelPrime.mul_left (H1 : IsRelPrime x z) (H2 : IsRelPrime y z) : IsRelPrime (x * y) z := fun _ h hz ↦ by obtain ⟨a, b, ha, hb, rfl⟩ := exists_dvd_and_dvd_of_dvd_mul h exact (H1 ha <| (dvd_mul_right a b).trans hz).mul (H2 hb <| (dvd_mul_left b a).trans hz) theorem IsRelPrime.mul_right (H1 : IsRelPrime x y) (H2 : IsRelPrime x z) : IsRelPrime x (y * z) := by rw [isRelPrime_comm] at H1 H2 ⊢; exact H1.mul_left H2 theorem IsRelPrime.mul_left_iff : IsRelPrime (x * y) z ↔ IsRelPrime x z ∧ IsRelPrime y z := ⟨fun H ↦ ⟨H.of_mul_left_left, H.of_mul_left_right⟩, fun ⟨H1, H2⟩ ↦ H1.mul_left H2⟩ theorem IsRelPrime.mul_right_iff : IsRelPrime x (y * z) ↔ IsRelPrime x y ∧ IsRelPrime x z := ⟨fun H ↦ ⟨H.of_mul_right_left, H.of_mul_right_right⟩, fun ⟨H1, H2⟩ ↦ H1.mul_right H2⟩ theorem IsRelPrime.mul_dvd (H : IsRelPrime x y) (H1 : x ∣ z) (H2 : y ∣ z) : x * y ∣ z := H.mul_dvd_of_left_isPrimal H1 H2 (DecompositionMonoid.primal x) end RelPrime
Algebra\EuclideanDomain\Basic.lean
/- Copyright (c) 2018 Louis Carlin. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Louis Carlin, Mario Carneiro -/ import Mathlib.Algebra.EuclideanDomain.Defs import Mathlib.Algebra.Ring.Divisibility.Basic import Mathlib.Algebra.Ring.Regular import Mathlib.Algebra.GroupWithZero.Divisibility import Mathlib.Algebra.Ring.Basic /-! # Lemmas about Euclidean domains ## Main statements * `gcd_eq_gcd_ab`: states Bézout's lemma for Euclidean domains. -/ universe u namespace EuclideanDomain variable {R : Type u} variable [EuclideanDomain R] /-- The well founded relation in a Euclidean Domain satisfying `a % b ≺ b` for `b ≠ 0` -/ local infixl:50 " ≺ " => EuclideanDomain.R -- See note [lower instance priority] instance (priority := 100) toMulDivCancelClass : MulDivCancelClass R where mul_div_cancel a b hb := by refine (eq_of_sub_eq_zero ?_).symm by_contra h have := mul_right_not_lt b h rw [sub_mul, mul_comm (_ / _), sub_eq_iff_eq_add'.2 (div_add_mod (a * b) b).symm] at this exact this (mod_lt _ hb) @[simp] theorem mod_eq_zero {a b : R} : a % b = 0 ↔ b ∣ a := ⟨fun h => by rw [← div_add_mod a b, h, add_zero] exact dvd_mul_right _ _, fun ⟨c, e⟩ => by rw [e, ← add_left_cancel_iff, div_add_mod, add_zero] haveI := Classical.dec by_cases b0 : b = 0 · simp only [b0, zero_mul] · rw [mul_div_cancel_left₀ _ b0]⟩ @[simp] theorem mod_self (a : R) : a % a = 0 := mod_eq_zero.2 dvd_rfl theorem dvd_mod_iff {a b c : R} (h : c ∣ b) : c ∣ a % b ↔ c ∣ a := by rw [← dvd_add_right (h.mul_right _), div_add_mod] @[simp] theorem mod_one (a : R) : a % 1 = 0 := mod_eq_zero.2 (one_dvd _) @[simp] theorem zero_mod (b : R) : 0 % b = 0 := mod_eq_zero.2 (dvd_zero _) @[simp] theorem zero_div {a : R} : 0 / a = 0 := by_cases (fun a0 : a = 0 => a0.symm ▸ div_zero 0) fun a0 => by simpa only [zero_mul] using mul_div_cancel_right₀ 0 a0 @[simp] theorem div_self {a : R} (a0 : a ≠ 0) : a / a = 1 := by simpa only [one_mul] using mul_div_cancel_right₀ 1 a0 theorem eq_div_of_mul_eq_left {a b c : R} (hb : b ≠ 0) (h : a * b = c) : a = c / b := by rw [← h, mul_div_cancel_right₀ _ hb] theorem eq_div_of_mul_eq_right {a b c : R} (ha : a ≠ 0) (h : a * b = c) : b = c / a := by rw [← h, mul_div_cancel_left₀ _ ha] theorem mul_div_assoc (x : R) {y z : R} (h : z ∣ y) : x * y / z = x * (y / z) := by by_cases hz : z = 0 · subst hz rw [div_zero, div_zero, mul_zero] rcases h with ⟨p, rfl⟩ rw [mul_div_cancel_left₀ _ hz, mul_left_comm, mul_div_cancel_left₀ _ hz] protected theorem mul_div_cancel' {a b : R} (hb : b ≠ 0) (hab : b ∣ a) : b * (a / b) = a := by rw [← mul_div_assoc _ hab, mul_div_cancel_left₀ _ hb] -- This generalizes `Int.div_one`, see note [simp-normal form] @[simp] theorem div_one (p : R) : p / 1 = p := (EuclideanDomain.eq_div_of_mul_eq_left (one_ne_zero' R) (mul_one p)).symm theorem div_dvd_of_dvd {p q : R} (hpq : q ∣ p) : p / q ∣ p := by by_cases hq : q = 0 · rw [hq, zero_dvd_iff] at hpq rw [hpq] exact dvd_zero _ use q rw [mul_comm, ← EuclideanDomain.mul_div_assoc _ hpq, mul_comm, mul_div_cancel_right₀ _ hq] theorem dvd_div_of_mul_dvd {a b c : R} (h : a * b ∣ c) : b ∣ c / a := by rcases eq_or_ne a 0 with (rfl | ha) · simp only [div_zero, dvd_zero] rcases h with ⟨d, rfl⟩ refine ⟨d, ?_⟩ rw [mul_assoc, mul_div_cancel_left₀ _ ha] section GCD variable [DecidableEq R] @[simp] theorem gcd_zero_right (a : R) : gcd a 0 = a := by rw [gcd] split_ifs with h <;> simp only [h, zero_mod, gcd_zero_left] theorem gcd_val (a b : R) : gcd a b = gcd (b % a) a := by rw [gcd] split_ifs with h <;> [simp only [h, mod_zero, gcd_zero_right]; rfl] theorem gcd_dvd (a b : R) : gcd a b ∣ a ∧ gcd a b ∣ b := GCD.induction a b (fun b => by rw [gcd_zero_left] exact ⟨dvd_zero _, dvd_rfl⟩) fun a b _ ⟨IH₁, IH₂⟩ => by rw [gcd_val] exact ⟨IH₂, (dvd_mod_iff IH₂).1 IH₁⟩ theorem gcd_dvd_left (a b : R) : gcd a b ∣ a := (gcd_dvd a b).left theorem gcd_dvd_right (a b : R) : gcd a b ∣ b := (gcd_dvd a b).right protected theorem gcd_eq_zero_iff {a b : R} : gcd a b = 0 ↔ a = 0 ∧ b = 0 := ⟨fun h => by simpa [h] using gcd_dvd a b, by rintro ⟨rfl, rfl⟩ exact gcd_zero_right _⟩ theorem dvd_gcd {a b c : R} : c ∣ a → c ∣ b → c ∣ gcd a b := GCD.induction a b (fun _ _ H => by simpa only [gcd_zero_left] using H) fun a b _ IH ca cb => by rw [gcd_val] exact IH ((dvd_mod_iff ca).2 cb) ca theorem gcd_eq_left {a b : R} : gcd a b = a ↔ a ∣ b := ⟨fun h => by rw [← h] apply gcd_dvd_right, fun h => by rw [gcd_val, mod_eq_zero.2 h, gcd_zero_left]⟩ @[simp] theorem gcd_one_left (a : R) : gcd 1 a = 1 := gcd_eq_left.2 (one_dvd _) @[simp] theorem gcd_self (a : R) : gcd a a = a := gcd_eq_left.2 dvd_rfl @[simp] theorem xgcdAux_fst (x y : R) : ∀ s t s' t', (xgcdAux x s t y s' t').1 = gcd x y := GCD.induction x y (by intros rw [xgcd_zero_left, gcd_zero_left]) fun x y h IH s t s' t' => by simp only [xgcdAux_rec h, if_neg h, IH] rw [← gcd_val] theorem xgcdAux_val (x y : R) : xgcdAux x 1 0 y 0 1 = (gcd x y, xgcd x y) := by rw [xgcd, ← xgcdAux_fst x y 1 0 0 1] private def P (a b : R) : R × R × R → Prop | (r, s, t) => (r : R) = a * s + b * t theorem xgcdAux_P (a b : R) {r r' : R} {s t s' t'} (p : P a b (r, s, t)) (p' : P a b (r', s', t')) : P a b (xgcdAux r s t r' s' t') := by induction r, r' using GCD.induction generalizing s t s' t' with | H0 n => simpa only [xgcd_zero_left] | H1 _ _ h IH => rw [xgcdAux_rec h] refine IH ?_ p unfold P at p p' ⊢ dsimp rw [mul_sub, mul_sub, add_sub, sub_add_eq_add_sub, ← p', sub_sub, mul_comm _ s, ← mul_assoc, mul_comm _ t, ← mul_assoc, ← add_mul, ← p, mod_eq_sub_mul_div] /-- An explicit version of **Bézout's lemma** for Euclidean domains. -/ theorem gcd_eq_gcd_ab (a b : R) : (gcd a b : R) = a * gcdA a b + b * gcdB a b := by have := @xgcdAux_P _ _ _ a b a b 1 0 0 1 (by dsimp [P]; rw [mul_one, mul_zero, add_zero]) (by dsimp [P]; rw [mul_one, mul_zero, zero_add]) rwa [xgcdAux_val, xgcd_val] at this -- see Note [lower instance priority] instance (priority := 70) (R : Type*) [e : EuclideanDomain R] : NoZeroDivisors R := haveI := Classical.decEq R { eq_zero_or_eq_zero_of_mul_eq_zero := fun {a b} h => or_iff_not_and_not.2 fun h0 => h0.1 <| by rw [← mul_div_cancel_right₀ a h0.2, h, zero_div] } -- see Note [lower instance priority] instance (priority := 70) (R : Type*) [e : EuclideanDomain R] : IsDomain R := { e, NoZeroDivisors.to_isDomain R with } end GCD section LCM variable [DecidableEq R] theorem dvd_lcm_left (x y : R) : x ∣ lcm x y := by_cases (fun hxy : gcd x y = 0 => by rw [lcm, hxy, div_zero] exact dvd_zero _) fun hxy => let ⟨z, hz⟩ := (gcd_dvd x y).2 ⟨z, Eq.symm <| eq_div_of_mul_eq_left hxy <| by rw [mul_right_comm, mul_assoc, ← hz]⟩ theorem dvd_lcm_right (x y : R) : y ∣ lcm x y := by_cases (fun hxy : gcd x y = 0 => by rw [lcm, hxy, div_zero] exact dvd_zero _) fun hxy => let ⟨z, hz⟩ := (gcd_dvd x y).1 ⟨z, Eq.symm <| eq_div_of_mul_eq_right hxy <| by rw [← mul_assoc, mul_right_comm, ← hz]⟩ theorem lcm_dvd {x y z : R} (hxz : x ∣ z) (hyz : y ∣ z) : lcm x y ∣ z := by rw [lcm] by_cases hxy : gcd x y = 0 · rw [hxy, div_zero] rw [EuclideanDomain.gcd_eq_zero_iff] at hxy rwa [hxy.1] at hxz rcases gcd_dvd x y with ⟨⟨r, hr⟩, ⟨s, hs⟩⟩ suffices x * y ∣ z * gcd x y by cases' this with p hp use p generalize gcd x y = g at hxy hs hp ⊢ subst hs rw [mul_left_comm, mul_div_cancel_left₀ _ hxy, ← mul_left_inj' hxy, hp] rw [← mul_assoc] simp only [mul_right_comm] rw [gcd_eq_gcd_ab, mul_add] apply dvd_add · rw [mul_left_comm] exact mul_dvd_mul_left _ (hyz.mul_right _) · rw [mul_left_comm, mul_comm] exact mul_dvd_mul_left _ (hxz.mul_right _) @[simp] theorem lcm_dvd_iff {x y z : R} : lcm x y ∣ z ↔ x ∣ z ∧ y ∣ z := ⟨fun hz => ⟨(dvd_lcm_left _ _).trans hz, (dvd_lcm_right _ _).trans hz⟩, fun ⟨hxz, hyz⟩ => lcm_dvd hxz hyz⟩ @[simp] theorem lcm_zero_left (x : R) : lcm 0 x = 0 := by rw [lcm, zero_mul, zero_div] @[simp] theorem lcm_zero_right (x : R) : lcm x 0 = 0 := by rw [lcm, mul_zero, zero_div] @[simp] theorem lcm_eq_zero_iff {x y : R} : lcm x y = 0 ↔ x = 0 ∨ y = 0 := by constructor · intro hxy rw [lcm, mul_div_assoc _ (gcd_dvd_right _ _), mul_eq_zero] at hxy apply Or.imp_right _ hxy intro hy by_cases hgxy : gcd x y = 0 · rw [EuclideanDomain.gcd_eq_zero_iff] at hgxy exact hgxy.2 · rcases gcd_dvd x y with ⟨⟨r, hr⟩, ⟨s, hs⟩⟩ generalize gcd x y = g at hr hs hy hgxy ⊢ subst hs rw [mul_div_cancel_left₀ _ hgxy] at hy rw [hy, mul_zero] rintro (hx | hy) · rw [hx, lcm_zero_left] · rw [hy, lcm_zero_right] @[simp] theorem gcd_mul_lcm (x y : R) : gcd x y * lcm x y = x * y := by rw [lcm]; by_cases h : gcd x y = 0 · rw [h, zero_mul] rw [EuclideanDomain.gcd_eq_zero_iff] at h rw [h.1, zero_mul] rcases gcd_dvd x y with ⟨⟨r, hr⟩, ⟨s, hs⟩⟩ generalize gcd x y = g at h hr ⊢; subst hr rw [mul_assoc, mul_div_cancel_left₀ _ h] end LCM section Div theorem mul_div_mul_cancel {a b c : R} (ha : a ≠ 0) (hcb : c ∣ b) : a * b / (a * c) = b / c := by by_cases hc : c = 0; · simp [hc] refine eq_div_of_mul_eq_right hc (mul_left_cancel₀ ha ?_) rw [← mul_assoc, ← mul_div_assoc _ (mul_dvd_mul_left a hcb), mul_div_cancel_left₀ _ (mul_ne_zero ha hc)] theorem mul_div_mul_comm_of_dvd_dvd {a b c d : R} (hac : c ∣ a) (hbd : d ∣ b) : a * b / (c * d) = a / c * (b / d) := by rcases eq_or_ne c 0 with (rfl | hc0); · simp rcases eq_or_ne d 0 with (rfl | hd0); · simp obtain ⟨k1, rfl⟩ := hac obtain ⟨k2, rfl⟩ := hbd rw [mul_div_cancel_left₀ _ hc0, mul_div_cancel_left₀ _ hd0, mul_mul_mul_comm, mul_div_cancel_left₀ _ (mul_ne_zero hc0 hd0)] end Div end EuclideanDomain
Algebra\EuclideanDomain\Defs.lean
/- Copyright (c) 2018 Louis Carlin. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Louis Carlin, Mario Carneiro -/ import Mathlib.Algebra.Divisibility.Basic import Mathlib.Algebra.Group.Basic import Mathlib.Algebra.Ring.Defs /-! # Euclidean domains This file introduces Euclidean domains and provides the extended Euclidean algorithm. To be precise, a slightly more general version is provided which is sometimes called a transfinite Euclidean domain and differs in the fact that the degree function need not take values in `ℕ` but can take values in any well-ordered set. Transfinite Euclidean domains were introduced by Motzkin and examples which don't satisfy the classical notion were provided independently by Hiblot and Nagata. ## Main definitions * `EuclideanDomain`: Defines Euclidean domain with functions `quotient` and `remainder`. Instances of `Div` and `Mod` are provided, so that one can write `a = b * (a / b) + a % b`. * `gcd`: defines the greatest common divisors of two elements of a Euclidean domain. * `xgcd`: given two elements `a b : R`, `xgcd a b` defines the pair `(x, y)` such that `x * a + y * b = gcd a b`. * `lcm`: defines the lowest common multiple of two elements `a` and `b` of a Euclidean domain as `a * b / (gcd a b)` ## Main statements See `Algebra.EuclideanDomain.Basic` for most of the theorems about Euclidean domains, including Bézout's lemma. See `Algebra.EuclideanDomain.Instances` for the fact that `ℤ` is a Euclidean domain, as is any field. ## Notation `≺` denotes the well founded relation on the Euclidean domain, e.g. in the example of the polynomial ring over a field, `p ≺ q` for polynomials `p` and `q` if and only if the degree of `p` is less than the degree of `q`. ## Implementation details Instead of working with a valuation, `EuclideanDomain` is implemented with the existence of a well founded relation `r` on the integral domain `R`, which in the example of `ℤ` would correspond to setting `i ≺ j` for integers `i` and `j` if the absolute value of `i` is smaller than the absolute value of `j`. ## References * [Th. Motzkin, *The Euclidean algorithm*][MR32592] * [J.-J. Hiblot, *Des anneaux euclidiens dont le plus petit algorithme n'est pas à valeurs finies*] [MR399081] * [M. Nagata, *On Euclid algorithm*][MR541021] ## Tags Euclidean domain, transfinite Euclidean domain, Bézout's lemma -/ universe u /-- A `EuclideanDomain` is a non-trivial commutative ring with a division and a remainder, satisfying `b * (a / b) + a % b = a`. The definition of a Euclidean domain usually includes a valuation function `R → ℕ`. This definition is slightly generalised to include a well founded relation `r` with the property that `r (a % b) b`, instead of a valuation. -/ class EuclideanDomain (R : Type u) extends CommRing R, Nontrivial R where /-- A division function (denoted `/`) on `R`. This satisfies the property `b * (a / b) + a % b = a`, where `%` denotes `remainder`. -/ protected quotient : R → R → R /-- Division by zero should always give zero by convention. -/ protected quotient_zero : ∀ a, quotient a 0 = 0 /-- A remainder function (denoted `%`) on `R`. This satisfies the property `b * (a / b) + a % b = a`, where `/` denotes `quotient`. -/ protected remainder : R → R → R /-- The property that links the quotient and remainder functions. This allows us to compute GCDs and LCMs. -/ protected quotient_mul_add_remainder_eq : ∀ a b, b * quotient a b + remainder a b = a /-- A well-founded relation on `R`, satisfying `r (a % b) b`. This ensures that the GCD algorithm always terminates. -/ protected r : R → R → Prop /-- The relation `r` must be well-founded. This ensures that the GCD algorithm always terminates. -/ r_wellFounded : WellFounded r /-- The relation `r` satisfies `r (a % b) b`. -/ protected remainder_lt : ∀ (a) {b}, b ≠ 0 → r (remainder a b) b /-- An additional constraint on `r`. -/ mul_left_not_lt : ∀ (a) {b}, b ≠ 0 → ¬r (a * b) a namespace EuclideanDomain variable {R : Type u} [EuclideanDomain R] /-- Abbreviated notation for the well-founded relation `r` in a Euclidean domain. -/ local infixl:50 " ≺ " => EuclideanDomain.r local instance wellFoundedRelation : WellFoundedRelation R where wf := r_wellFounded -- see Note [lower instance priority] instance (priority := 70) : Div R := ⟨EuclideanDomain.quotient⟩ -- see Note [lower instance priority] instance (priority := 70) : Mod R := ⟨EuclideanDomain.remainder⟩ theorem div_add_mod (a b : R) : b * (a / b) + a % b = a := EuclideanDomain.quotient_mul_add_remainder_eq _ _ theorem mod_add_div (a b : R) : a % b + b * (a / b) = a := (add_comm _ _).trans (div_add_mod _ _) theorem mod_add_div' (m k : R) : m % k + m / k * k = m := by rw [mul_comm] exact mod_add_div _ _ theorem div_add_mod' (m k : R) : m / k * k + m % k = m := by rw [mul_comm] exact div_add_mod _ _ theorem mod_eq_sub_mul_div {R : Type*} [EuclideanDomain R] (a b : R) : a % b = a - b * (a / b) := calc a % b = b * (a / b) + a % b - b * (a / b) := (add_sub_cancel_left _ _).symm _ = a - b * (a / b) := by rw [div_add_mod] theorem mod_lt : ∀ (a) {b : R}, b ≠ 0 → a % b ≺ b := EuclideanDomain.remainder_lt theorem mul_right_not_lt {a : R} (b) (h : a ≠ 0) : ¬a * b ≺ b := by rw [mul_comm] exact mul_left_not_lt b h @[simp] theorem mod_zero (a : R) : a % 0 = a := by simpa only [zero_mul, zero_add] using div_add_mod a 0 theorem lt_one (a : R) : a ≺ (1 : R) → a = 0 := haveI := Classical.dec not_imp_not.1 fun h => by simpa only [one_mul] using mul_left_not_lt 1 h theorem val_dvd_le : ∀ a b : R, b ∣ a → a ≠ 0 → ¬a ≺ b | _, b, ⟨d, rfl⟩, ha => mul_left_not_lt b (mt (by rintro rfl; exact mul_zero _) ha) @[simp] theorem div_zero (a : R) : a / 0 = 0 := EuclideanDomain.quotient_zero a section @[elab_as_elim] theorem GCD.induction {P : R → R → Prop} (a b : R) (H0 : ∀ x, P 0 x) (H1 : ∀ a b, a ≠ 0 → P (b % a) a → P a b) : P a b := by classical exact if a0 : a = 0 then by -- Porting note: required for hygiene, the equation compiler introduces a dummy variable `x` -- See https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/unnecessarily.20tombstoned.20argument/near/314573315 change P a b exact a0.symm ▸ H0 b else have _ := mod_lt b a0 H1 _ _ a0 (GCD.induction (b % a) a H0 H1) termination_by a end section GCD variable [DecidableEq R] /-- `gcd a b` is a (non-unique) element such that `gcd a b ∣ a` `gcd a b ∣ b`, and for any element `c` such that `c ∣ a` and `c ∣ b`, then `c ∣ gcd a b` -/ def gcd (a b : R) : R := if a0 : a = 0 then b else have _ := mod_lt b a0 gcd (b % a) a termination_by a @[simp] theorem gcd_zero_left (a : R) : gcd 0 a = a := by rw [gcd] exact if_pos rfl /-- An implementation of the extended GCD algorithm. At each step we are computing a triple `(r, s, t)`, where `r` is the next value of the GCD algorithm, to compute the greatest common divisor of the input (say `x` and `y`), and `s` and `t` are the coefficients in front of `x` and `y` to obtain `r` (i.e. `r = s * x + t * y`). The function `xgcdAux` takes in two triples, and from these recursively computes the next triple: ``` xgcdAux (r, s, t) (r', s', t') = xgcdAux (r' % r, s' - (r' / r) * s, t' - (r' / r) * t) (r, s, t) ``` -/ def xgcdAux (r s t r' s' t' : R) : R × R × R := if _hr : r = 0 then (r', s', t') else let q := r' / r have _ := mod_lt r' _hr xgcdAux (r' % r) (s' - q * s) (t' - q * t) r s t termination_by r @[simp] theorem xgcd_zero_left {s t r' s' t' : R} : xgcdAux 0 s t r' s' t' = (r', s', t') := by unfold xgcdAux exact if_pos rfl theorem xgcdAux_rec {r s t r' s' t' : R} (h : r ≠ 0) : xgcdAux r s t r' s' t' = xgcdAux (r' % r) (s' - r' / r * s) (t' - r' / r * t) r s t := by conv => lhs rw [xgcdAux] exact if_neg h /-- Use the extended GCD algorithm to generate the `a` and `b` values satisfying `gcd x y = x * a + y * b`. -/ def xgcd (x y : R) : R × R := (xgcdAux x 1 0 y 0 1).2 /-- The extended GCD `a` value in the equation `gcd x y = x * a + y * b`. -/ def gcdA (x y : R) : R := (xgcd x y).1 /-- The extended GCD `b` value in the equation `gcd x y = x * a + y * b`. -/ def gcdB (x y : R) : R := (xgcd x y).2 @[simp] theorem gcdA_zero_left {s : R} : gcdA 0 s = 0 := by unfold gcdA rw [xgcd, xgcd_zero_left] @[simp] theorem gcdB_zero_left {s : R} : gcdB 0 s = 1 := by unfold gcdB rw [xgcd, xgcd_zero_left] theorem xgcd_val (x y : R) : xgcd x y = (gcdA x y, gcdB x y) := rfl end GCD section LCM variable [DecidableEq R] /-- `lcm a b` is a (non-unique) element such that `a ∣ lcm a b` `b ∣ lcm a b`, and for any element `c` such that `a ∣ c` and `b ∣ c`, then `lcm a b ∣ c` -/ def lcm (x y : R) : R := x * y / gcd x y end LCM end EuclideanDomain
Algebra\EuclideanDomain\Field.lean
/- Copyright (c) 2018 Louis Carlin. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Louis Carlin, Mario Carneiro -/ import Mathlib.Algebra.EuclideanDomain.Defs import Mathlib.Algebra.Field.Defs import Mathlib.Algebra.GroupWithZero.Units.Basic /-! # Instances for Euclidean domains * `Field.toEuclideanDomain`: shows that any field is a Euclidean domain. -/ -- see Note [lower instance priority] instance (priority := 100) Field.toEuclideanDomain {K : Type*} [Field K] : EuclideanDomain K := { toCommRing := Field.toCommRing quotient := (· / ·), remainder := fun a b => a - a * b / b, quotient_zero := div_zero, quotient_mul_add_remainder_eq := fun a b => by by_cases h : b = 0 <;> simp [h, mul_div_cancel₀] r := fun a b => a = 0 ∧ b ≠ 0, r_wellFounded := WellFounded.intro fun a => (Acc.intro _) fun b ⟨hb, _⟩ => (Acc.intro _) fun c ⟨_, hnb⟩ => False.elim <| hnb hb, remainder_lt := fun a b hnb => by simp [hnb], mul_left_not_lt := fun a b hnb ⟨hab, hna⟩ => Or.casesOn (mul_eq_zero.1 hab) hna hnb }
Algebra\EuclideanDomain\Int.lean
/- Copyright (c) 2018 Louis Carlin. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Louis Carlin, Mario Carneiro -/ import Mathlib.Algebra.EuclideanDomain.Defs import Mathlib.Algebra.Order.Group.Int import Mathlib.Algebra.Ring.Int /-! # Instances for Euclidean domains * `Int.euclideanDomain`: shows that `ℤ` is a Euclidean domain. -/ instance Int.euclideanDomain : EuclideanDomain ℤ := { inferInstanceAs (CommRing Int), inferInstanceAs (Nontrivial Int) with quotient := (· / ·), quotient_zero := Int.ediv_zero, remainder := (· % ·), quotient_mul_add_remainder_eq := Int.ediv_add_emod, r := fun a b => a.natAbs < b.natAbs, r_wellFounded := (measure natAbs).wf remainder_lt := fun a b b0 => Int.ofNat_lt.1 <| by rw [Int.natAbs_of_nonneg (Int.emod_nonneg _ b0), ← Int.abs_eq_natAbs] exact Int.emod_lt _ b0 mul_left_not_lt := fun a b b0 => not_lt_of_ge <| by rw [← mul_one a.natAbs, Int.natAbs_mul] rw [← Int.natAbs_pos] at b0 exact Nat.mul_le_mul_left _ b0 }
Algebra\Field\Basic.lean
/- Copyright (c) 2014 Robert Lewis. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Robert Lewis, Leonardo de Moura, Johannes Hölzl, Mario Carneiro -/ import Mathlib.Algebra.Field.Defs import Mathlib.Algebra.GroupWithZero.Units.Lemmas import Mathlib.Algebra.Ring.Commute import Mathlib.Algebra.Ring.Invertible import Mathlib.Order.Synonym /-! # Lemmas about division (semi)rings and (semi)fields -/ open Function OrderDual Set universe u variable {α β K : Type*} section DivisionSemiring variable [DivisionSemiring α] {a b c d : α} theorem add_div (a b c : α) : (a + b) / c = a / c + b / c := by simp_rw [div_eq_mul_inv, add_mul] @[field_simps] theorem div_add_div_same (a b c : α) : a / c + b / c = (a + b) / c := (add_div _ _ _).symm theorem same_add_div (h : b ≠ 0) : (b + a) / b = 1 + a / b := by rw [← div_self h, add_div] theorem div_add_same (h : b ≠ 0) : (a + b) / b = a / b + 1 := by rw [← div_self h, add_div] theorem one_add_div (h : b ≠ 0) : 1 + a / b = (b + a) / b := (same_add_div h).symm theorem div_add_one (h : b ≠ 0) : a / b + 1 = (a + b) / b := (div_add_same h).symm /-- See `inv_add_inv` for the more convenient version when `K` is commutative. -/ theorem inv_add_inv' (ha : a ≠ 0) (hb : b ≠ 0) : a⁻¹ + b⁻¹ = a⁻¹ * (a + b) * b⁻¹ := let _ := invertibleOfNonzero ha; let _ := invertibleOfNonzero hb; invOf_add_invOf a b theorem one_div_mul_add_mul_one_div_eq_one_div_add_one_div (ha : a ≠ 0) (hb : b ≠ 0) : 1 / a * (a + b) * (1 / b) = 1 / a + 1 / b := by simpa only [one_div] using (inv_add_inv' ha hb).symm theorem add_div_eq_mul_add_div (a b : α) (hc : c ≠ 0) : a + b / c = (a * c + b) / c := (eq_div_iff_mul_eq hc).2 <| by rw [right_distrib, div_mul_cancel₀ _ hc] @[field_simps] theorem add_div' (a b c : α) (hc : c ≠ 0) : b + a / c = (b * c + a) / c := by rw [add_div, mul_div_cancel_right₀ _ hc] @[field_simps] theorem div_add' (a b c : α) (hc : c ≠ 0) : a / c + b = (a + b * c) / c := by rwa [add_comm, add_div', add_comm] protected theorem Commute.div_add_div (hbc : Commute b c) (hbd : Commute b d) (hb : b ≠ 0) (hd : d ≠ 0) : a / b + c / d = (a * d + b * c) / (b * d) := by rw [add_div, mul_div_mul_right _ b hd, hbc.eq, hbd.eq, mul_div_mul_right c d hb] protected theorem Commute.one_div_add_one_div (hab : Commute a b) (ha : a ≠ 0) (hb : b ≠ 0) : 1 / a + 1 / b = (a + b) / (a * b) := by rw [(Commute.one_right a).div_add_div hab ha hb, one_mul, mul_one, add_comm] protected theorem Commute.inv_add_inv (hab : Commute a b) (ha : a ≠ 0) (hb : b ≠ 0) : a⁻¹ + b⁻¹ = (a + b) / (a * b) := by rw [inv_eq_one_div, inv_eq_one_div, hab.one_div_add_one_div ha hb] end DivisionSemiring section DivisionMonoid variable [DivisionMonoid K] [HasDistribNeg K] {a b : K} theorem one_div_neg_one_eq_neg_one : (1 : K) / -1 = -1 := have : -1 * -1 = (1 : K) := by rw [neg_mul_neg, one_mul] Eq.symm (eq_one_div_of_mul_eq_one_right this) theorem one_div_neg_eq_neg_one_div (a : K) : 1 / -a = -(1 / a) := calc 1 / -a = 1 / (-1 * a) := by rw [neg_eq_neg_one_mul] _ = 1 / a * (1 / -1) := by rw [one_div_mul_one_div_rev] _ = 1 / a * -1 := by rw [one_div_neg_one_eq_neg_one] _ = -(1 / a) := by rw [mul_neg, mul_one] theorem div_neg_eq_neg_div (a b : K) : b / -a = -(b / a) := calc b / -a = b * (1 / -a) := by rw [← inv_eq_one_div, division_def] _ = b * -(1 / a) := by rw [one_div_neg_eq_neg_one_div] _ = -(b * (1 / a)) := by rw [neg_mul_eq_mul_neg] _ = -(b / a) := by rw [mul_one_div] theorem neg_div (a b : K) : -b / a = -(b / a) := by rw [neg_eq_neg_one_mul, mul_div_assoc, ← neg_eq_neg_one_mul] @[field_simps] theorem neg_div' (a b : K) : -(b / a) = -b / a := by simp [neg_div] @[simp] theorem neg_div_neg_eq (a b : K) : -a / -b = a / b := by rw [div_neg_eq_neg_div, neg_div, neg_neg] theorem neg_inv : -a⁻¹ = (-a)⁻¹ := by rw [inv_eq_one_div, inv_eq_one_div, div_neg_eq_neg_div] theorem div_neg (a : K) : a / -b = -(a / b) := by rw [← div_neg_eq_neg_div] theorem inv_neg : (-a)⁻¹ = -a⁻¹ := by rw [neg_inv] theorem inv_neg_one : (-1 : K)⁻¹ = -1 := by rw [← neg_inv, inv_one] end DivisionMonoid section DivisionRing variable [DivisionRing K] {a b c d : K} @[simp] theorem div_neg_self {a : K} (h : a ≠ 0) : a / -a = -1 := by rw [div_neg_eq_neg_div, div_self h] @[simp] theorem neg_div_self {a : K} (h : a ≠ 0) : -a / a = -1 := by rw [neg_div, div_self h] theorem div_sub_div_same (a b c : K) : a / c - b / c = (a - b) / c := by rw [sub_eq_add_neg, ← neg_div, div_add_div_same, sub_eq_add_neg] theorem same_sub_div {a b : K} (h : b ≠ 0) : (b - a) / b = 1 - a / b := by simpa only [← @div_self _ _ b h] using (div_sub_div_same b a b).symm theorem one_sub_div {a b : K} (h : b ≠ 0) : 1 - a / b = (b - a) / b := (same_sub_div h).symm theorem div_sub_same {a b : K} (h : b ≠ 0) : (a - b) / b = a / b - 1 := by simpa only [← @div_self _ _ b h] using (div_sub_div_same a b b).symm theorem div_sub_one {a b : K} (h : b ≠ 0) : a / b - 1 = (a - b) / b := (div_sub_same h).symm theorem sub_div (a b c : K) : (a - b) / c = a / c - b / c := (div_sub_div_same _ _ _).symm /-- See `inv_sub_inv` for the more convenient version when `K` is commutative. -/ theorem inv_sub_inv' {a b : K} (ha : a ≠ 0) (hb : b ≠ 0) : a⁻¹ - b⁻¹ = a⁻¹ * (b - a) * b⁻¹ := let _ := invertibleOfNonzero ha; let _ := invertibleOfNonzero hb; invOf_sub_invOf a b theorem one_div_mul_sub_mul_one_div_eq_one_div_add_one_div (ha : a ≠ 0) (hb : b ≠ 0) : 1 / a * (b - a) * (1 / b) = 1 / a - 1 / b := by simpa only [one_div] using (inv_sub_inv' ha hb).symm -- see Note [lower instance priority] instance (priority := 100) DivisionRing.isDomain : IsDomain K := NoZeroDivisors.to_isDomain _ protected theorem Commute.div_sub_div (hbc : Commute b c) (hbd : Commute b d) (hb : b ≠ 0) (hd : d ≠ 0) : a / b - c / d = (a * d - b * c) / (b * d) := by simpa only [mul_neg, neg_div, ← sub_eq_add_neg] using hbc.neg_right.div_add_div hbd hb hd protected theorem Commute.inv_sub_inv (hab : Commute a b) (ha : a ≠ 0) (hb : b ≠ 0) : a⁻¹ - b⁻¹ = (b - a) / (a * b) := by simp only [inv_eq_one_div, (Commute.one_right a).div_sub_div hab ha hb, one_mul, mul_one] end DivisionRing section Semifield variable [Semifield α] {a b c d : α} theorem div_add_div (a : α) (c : α) (hb : b ≠ 0) (hd : d ≠ 0) : a / b + c / d = (a * d + b * c) / (b * d) := (Commute.all b _).div_add_div (Commute.all _ _) hb hd theorem one_div_add_one_div (ha : a ≠ 0) (hb : b ≠ 0) : 1 / a + 1 / b = (a + b) / (a * b) := (Commute.all a _).one_div_add_one_div ha hb theorem inv_add_inv (ha : a ≠ 0) (hb : b ≠ 0) : a⁻¹ + b⁻¹ = (a + b) / (a * b) := (Commute.all a _).inv_add_inv ha hb end Semifield section Field variable [Field K] attribute [local simp] mul_assoc mul_comm mul_left_comm @[field_simps] theorem div_sub_div (a : K) {b : K} (c : K) {d : K} (hb : b ≠ 0) (hd : d ≠ 0) : a / b - c / d = (a * d - b * c) / (b * d) := (Commute.all b _).div_sub_div (Commute.all _ _) hb hd theorem inv_sub_inv {a b : K} (ha : a ≠ 0) (hb : b ≠ 0) : a⁻¹ - b⁻¹ = (b - a) / (a * b) := by rw [inv_eq_one_div, inv_eq_one_div, div_sub_div _ _ ha hb, one_mul, mul_one] @[field_simps] theorem sub_div' (a b c : K) (hc : c ≠ 0) : b - a / c = (b * c - a) / c := by simpa using div_sub_div b a one_ne_zero hc @[field_simps] theorem div_sub' (a b c : K) (hc : c ≠ 0) : a / c - b = (a - c * b) / c := by simpa using div_sub_div a b hc one_ne_zero -- see Note [lower instance priority] instance (priority := 100) Field.isDomain : IsDomain K := { DivisionRing.isDomain with } end Field namespace RingHom protected theorem injective [DivisionRing α] [Semiring β] [Nontrivial β] (f : α →+* β) : Injective f := (injective_iff_map_eq_zero f).2 fun _ ↦ (map_eq_zero f).1 end RingHom section NoncomputableDefs variable {R : Type*} [Nontrivial R] /-- Constructs a `DivisionRing` structure on a `Ring` consisting only of units and 0. -/ -- See note [reducible non-instances] noncomputable abbrev DivisionRing.ofIsUnitOrEqZero [Ring R] (h : ∀ a : R, IsUnit a ∨ a = 0) : DivisionRing R where toRing := ‹Ring R› __ := groupWithZeroOfIsUnitOrEqZero h nnqsmul := _ nnqsmul_def := fun q a => rfl qsmul := _ qsmul_def := fun q a => rfl /-- Constructs a `Field` structure on a `CommRing` consisting only of units and 0. -/ -- See note [reducible non-instances] noncomputable abbrev Field.ofIsUnitOrEqZero [CommRing R] (h : ∀ a : R, IsUnit a ∨ a = 0) : Field R where toCommRing := ‹CommRing R› __ := DivisionRing.ofIsUnitOrEqZero h end NoncomputableDefs namespace Function.Injective variable [Zero α] [Add α] [Neg α] [Sub α] [One α] [Mul α] [Inv α] [Div α] [SMul ℕ α] [SMul ℤ α] [SMul ℚ≥0 α] [SMul ℚ α] [Pow α ℕ] [Pow α ℤ] [NatCast α] [IntCast α] [NNRatCast α] [RatCast α] (f : α → β) (hf : Injective f) /-- Pullback a `DivisionSemiring` along an injective function. -/ -- See note [reducible non-instances] protected abbrev divisionSemiring [DivisionSemiring β] (zero : f 0 = 0) (one : f 1 = 1) (add : ∀ x y, f (x + y) = f x + f y) (mul : ∀ x y, f (x * y) = f x * f y) (inv : ∀ x, f x⁻¹ = (f x)⁻¹) (div : ∀ x y, f (x / y) = f x / f y) (nsmul : ∀ (n : ℕ) (x), f (n • x) = n • f x) (nnqsmul : ∀ (q : ℚ≥0) (x), f (q • x) = q • f x) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) (zpow : ∀ (x) (n : ℤ), f (x ^ n) = f x ^ n) (natCast : ∀ n : ℕ, f n = n) (nnratCast : ∀ q : ℚ≥0, f q = q) : DivisionSemiring α where toSemiring := hf.semiring f zero one add mul nsmul npow natCast __ := hf.groupWithZero f zero one mul inv div npow zpow nnratCast_def q := hf $ by rw [nnratCast, NNRat.cast_def, div, natCast, natCast] nnqsmul := (· • ·) nnqsmul_def q a := hf $ by rw [nnqsmul, NNRat.smul_def, mul, nnratCast] /-- Pullback a `DivisionSemiring` along an injective function. -/ -- See note [reducible non-instances] protected abbrev divisionRing [DivisionRing β] (zero : f 0 = 0) (one : f 1 = 1) (add : ∀ x y, f (x + y) = f x + f y) (mul : ∀ x y, f (x * y) = f x * f y) (neg : ∀ x, f (-x) = -f x) (sub : ∀ x y, f (x - y) = f x - f y) (inv : ∀ x, f x⁻¹ = (f x)⁻¹) (div : ∀ x y, f (x / y) = f x / f y) (nsmul : ∀ (n : ℕ) (x), f (n • x) = n • f x) (zsmul : ∀ (n : ℤ) (x), f (n • x) = n • f x) (nnqsmul : ∀ (q : ℚ≥0) (x), f (q • x) = q • f x) (qsmul : ∀ (q : ℚ) (x), f (q • x) = q • f x) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) (zpow : ∀ (x) (n : ℤ), f (x ^ n) = f x ^ n) (natCast : ∀ n : ℕ, f n = n) (intCast : ∀ n : ℤ, f n = n) (nnratCast : ∀ q : ℚ≥0, f q = q) (ratCast : ∀ q : ℚ, f q = q) : DivisionRing α where toRing := hf.ring f zero one add mul neg sub nsmul zsmul npow natCast intCast __ := hf.groupWithZero f zero one mul inv div npow zpow __ := hf.divisionSemiring f zero one add mul inv div nsmul nnqsmul npow zpow natCast nnratCast ratCast_def q := hf $ by erw [ratCast, div, intCast, natCast, Rat.cast_def] qsmul := (· • ·) qsmul_def q a := hf $ by erw [qsmul, mul, Rat.smul_def, ratCast] /-- Pullback a `Field` along an injective function. -/ -- See note [reducible non-instances] protected abbrev semifield [Semifield β] (zero : f 0 = 0) (one : f 1 = 1) (add : ∀ x y, f (x + y) = f x + f y) (mul : ∀ x y, f (x * y) = f x * f y) (inv : ∀ x, f x⁻¹ = (f x)⁻¹) (div : ∀ x y, f (x / y) = f x / f y) (nsmul : ∀ (n : ℕ) (x), f (n • x) = n • f x) (nnqsmul : ∀ (q : ℚ≥0) (x), f (q • x) = q • f x) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) (zpow : ∀ (x) (n : ℤ), f (x ^ n) = f x ^ n) (natCast : ∀ n : ℕ, f n = n) (nnratCast : ∀ q : ℚ≥0, f q = q) : Semifield α where toCommSemiring := hf.commSemiring f zero one add mul nsmul npow natCast __ := hf.commGroupWithZero f zero one mul inv div npow zpow __ := hf.divisionSemiring f zero one add mul inv div nsmul nnqsmul npow zpow natCast nnratCast /-- Pullback a `Field` along an injective function. -/ -- See note [reducible non-instances] protected abbrev field [Field β] (zero : f 0 = 0) (one : f 1 = 1) (add : ∀ x y, f (x + y) = f x + f y) (mul : ∀ x y, f (x * y) = f x * f y) (neg : ∀ x, f (-x) = -f x) (sub : ∀ x y, f (x - y) = f x - f y) (inv : ∀ x, f x⁻¹ = (f x)⁻¹) (div : ∀ x y, f (x / y) = f x / f y) (nsmul : ∀ (n : ℕ) (x), f (n • x) = n • f x) (zsmul : ∀ (n : ℤ) (x), f (n • x) = n • f x) (nnqsmul : ∀ (q : ℚ≥0) (x), f (q • x) = q • f x) (qsmul : ∀ (q : ℚ) (x), f (q • x) = q • f x) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) (zpow : ∀ (x) (n : ℤ), f (x ^ n) = f x ^ n) (natCast : ∀ n : ℕ, f n = n) (intCast : ∀ n : ℤ, f n = n) (nnratCast : ∀ q : ℚ≥0, f q = q) (ratCast : ∀ q : ℚ, f q = q) : Field α where toCommRing := hf.commRing f zero one add mul neg sub nsmul zsmul npow natCast intCast __ := hf.divisionRing f zero one add mul neg sub inv div nsmul zsmul nnqsmul qsmul npow zpow natCast intCast nnratCast ratCast end Function.Injective /-! ### Order dual -/ namespace OrderDual instance instRatCast [RatCast α] : RatCast αᵒᵈ := ‹_› instance instDivisionSemiring [DivisionSemiring α] : DivisionSemiring αᵒᵈ := ‹_› instance instDivisionRing [DivisionRing α] : DivisionRing αᵒᵈ := ‹_› instance instSemifield [Semifield α] : Semifield αᵒᵈ := ‹_› instance instField [Field α] : Field αᵒᵈ := ‹_› end OrderDual @[simp] lemma toDual_ratCast [RatCast α] (n : ℚ) : toDual (n : α) = n := rfl @[simp] lemma ofDual_ratCast [RatCast α] (n : ℚ) : (ofDual n : α) = n := rfl /-! ### Lexicographic order -/ namespace Lex instance instRatCast [RatCast α] : RatCast (Lex α) := ‹_› instance instDivisionSemiring [DivisionSemiring α] : DivisionSemiring (Lex α) := ‹_› instance instDivisionRing [DivisionRing α] : DivisionRing (Lex α) := ‹_› instance instSemifield [Semifield α] : Semifield (Lex α) := ‹_› instance instField [Field α] : Field (Lex α) := ‹_› end Lex @[simp] lemma toLex_ratCast [RatCast α] (n : ℚ) : toLex (n : α) = n := rfl @[simp] lemma ofLex_ratCast [RatCast α] (n : ℚ) : (ofLex n : α) = n := rfl
Algebra\Field\Defs.lean
/- Copyright (c) 2014 Robert Lewis. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Robert Lewis, Leonardo de Moura, Johannes Hölzl, Mario Carneiro, Yaël Dillies -/ import Mathlib.Algebra.Ring.Defs import Mathlib.Data.Rat.Init /-! # Division (semi)rings and (semi)fields This file introduces fields and division rings (also known as skewfields) and proves some basic statements about them. For a more extensive theory of fields, see the `FieldTheory` folder. ## Main definitions * `DivisionSemiring`: Nontrivial semiring with multiplicative inverses for nonzero elements. * `DivisionRing`: Nontrivial ring with multiplicative inverses for nonzero elements. * `Semifield`: Commutative division semiring. * `Field`: Commutative division ring. * `IsField`: Predicate on a (semi)ring that it is a (semi)field, i.e. that the multiplication is commutative, that it has more than one element and that all non-zero elements have a multiplicative inverse. In contrast to `Field`, which contains the data of a function associating to an element of the field its multiplicative inverse, this predicate only assumes the existence and can therefore more easily be used to e.g. transfer along ring isomorphisms. ## Implementation details By convention `0⁻¹ = 0` in a field or division ring. This is due to the fact that working with total functions has the advantage of not constantly having to check that `x ≠ 0` when writing `x⁻¹`. With this convention in place, some statements like `(a + b) * c⁻¹ = a * c⁻¹ + b * c⁻¹` still remain true, while others like the defining property `a * a⁻¹ = 1` need the assumption `a ≠ 0`. If you are a beginner in using Lean and are confused by that, you can read more about why this convention is taken in Kevin Buzzard's [blogpost](https://xenaproject.wordpress.com/2020/07/05/division-by-zero-in-type-theory-a-faq/) A division ring or field is an example of a `GroupWithZero`. If you cannot find a division ring / field lemma that does not involve `+`, you can try looking for a `GroupWithZero` lemma instead. ## Tags field, division ring, skew field, skew-field, skewfield -/ -- `NeZero` should not be needed in the basic algebraic hierarchy. assert_not_exists NeZero -- Check that we have not imported `Mathlib.Tactic.Common` yet. assert_not_exists Mathlib.Tactic.LibrarySearch.librarySearch assert_not_exists MonoidHom open Function Set universe u variable {α β K : Type*} /-- The default definition of the coercion `ℚ≥0 → K` for a division semiring `K`. `↑q : K` is defined as `(q.num : K) / (q.den : K)`. Do not use this directly (instances of `DivisionSemiring` are allowed to override that default for better definitional properties). Instead, use the coercion. -/ def NNRat.castRec [NatCast K] [Div K] (q : ℚ≥0) : K := q.num / q.den /-- The default definition of the coercion `ℚ → K` for a division ring `K`. `↑q : K` is defined as `(q.num : K) / (q.den : K)`. Do not use this directly (instances of `DivisionRing` are allowed to override that default for better definitional properties). Instead, use the coercion. -/ def Rat.castRec [NatCast K] [IntCast K] [Div K] (q : ℚ) : K := q.num / q.den /-- A `DivisionSemiring` is a `Semiring` with multiplicative inverses for nonzero elements. An instance of `DivisionSemiring K` includes maps `nnratCast : ℚ≥0 → K` and `nnqsmul : ℚ≥0 → K → K`. Those two fields are needed to implement the `DivisionSemiring K → Algebra ℚ≥0 K` instance since we need to control the specific definitions for some special cases of `K` (in particular `K = ℚ≥0` itself). See also note [forgetful inheritance]. If the division semiring has positive characteristic `p`, our division by zero convention forces `nnratCast (1 / p) = 1 / 0 = 0`. -/ class DivisionSemiring (α : Type*) extends Semiring α, GroupWithZero α, NNRatCast α where protected nnratCast := NNRat.castRec /-- However `NNRat.cast` is defined, it must be propositionally equal to `a / b`. Do not use this lemma directly. Use `NNRat.cast_def` instead. -/ protected nnratCast_def (q : ℚ≥0) : (NNRat.cast q : α) = q.num / q.den := by intros; rfl /-- Scalar multiplication by a nonnegative rational number. Unless there is a risk of a `Module ℚ≥0 _` instance diamond, write `nnqsmul := _`. This will set `nnqsmul` to `(NNRat.cast · * ·)` thanks to unification in the default proof of `nnqsmul_def`. Do not use directly. Instead use the `•` notation. -/ protected nnqsmul : ℚ≥0 → α → α /-- However `qsmul` is defined, it must be propositionally equal to multiplication by `Rat.cast`. Do not use this lemma directly. Use `NNRat.smul_def` instead. -/ protected nnqsmul_def (q : ℚ≥0) (a : α) : nnqsmul q a = NNRat.cast q * a := by intros; rfl /-- A `DivisionRing` is a `Ring` with multiplicative inverses for nonzero elements. An instance of `DivisionRing K` includes maps `ratCast : ℚ → K` and `qsmul : ℚ → K → K`. Those two fields are needed to implement the `DivisionRing K → Algebra ℚ K` instance since we need to control the specific definitions for some special cases of `K` (in particular `K = ℚ` itself). See also note [forgetful inheritance]. Similarly, there are maps `nnratCast ℚ≥0 → K` and `nnqsmul : ℚ≥0 → K → K` to implement the `DivisionSemiring K → Algebra ℚ≥0 K` instance. If the division ring has positive characteristic `p`, our division by zero convention forces `ratCast (1 / p) = 1 / 0 = 0`. -/ class DivisionRing (α : Type*) extends Ring α, DivInvMonoid α, Nontrivial α, NNRatCast α, RatCast α where /-- For a nonzero `a`, `a⁻¹` is a right multiplicative inverse. -/ protected mul_inv_cancel : ∀ (a : α), a ≠ 0 → a * a⁻¹ = 1 /-- The inverse of `0` is `0` by convention. -/ protected inv_zero : (0 : α)⁻¹ = 0 protected nnratCast := NNRat.castRec /-- However `NNRat.cast` is defined, it must be equal to `a / b`. Do not use this lemma directly. Use `NNRat.cast_def` instead. -/ protected nnratCast_def (q : ℚ≥0) : (NNRat.cast q : α) = q.num / q.den := by intros; rfl /-- Scalar multiplication by a nonnegative rational number. Unless there is a risk of a `Module ℚ≥0 _` instance diamond, write `nnqsmul := _`. This will set `nnqsmul` to `(NNRat.cast · * ·)` thanks to unification in the default proof of `nnqsmul_def`. Do not use directly. Instead use the `•` notation. -/ protected nnqsmul : ℚ≥0 → α → α /-- However `qsmul` is defined, it must be propositionally equal to multiplication by `Rat.cast`. Do not use this lemma directly. Use `NNRat.smul_def` instead. -/ protected nnqsmul_def (q : ℚ≥0) (a : α) : nnqsmul q a = NNRat.cast q * a := by intros; rfl protected ratCast := Rat.castRec /-- However `Rat.cast q` is defined, it must be propositionally equal to `q.num / q.den`. Do not use this lemma directly. Use `Rat.cast_def` instead. -/ protected ratCast_def (q : ℚ) : (Rat.cast q : α) = q.num / q.den := by intros; rfl /-- Scalar multiplication by a rational number. Unless there is a risk of a `Module ℚ _` instance diamond, write `qsmul := _`. This will set `qsmul` to `(Rat.cast · * ·)` thanks to unification in the default proof of `qsmul_def`. Do not use directly. Instead use the `•` notation. -/ protected qsmul : ℚ → α → α /-- However `qsmul` is defined, it must be propositionally equal to multiplication by `Rat.cast`. Do not use this lemma directly. Use `Rat.cast_def` instead. -/ protected qsmul_def (a : ℚ) (x : α) : qsmul a x = Rat.cast a * x := by intros; rfl -- see Note [lower instance priority] instance (priority := 100) DivisionRing.toDivisionSemiring [DivisionRing α] : DivisionSemiring α := { ‹DivisionRing α› with } /-- A `Semifield` is a `CommSemiring` with multiplicative inverses for nonzero elements. An instance of `Semifield K` includes maps `nnratCast : ℚ≥0 → K` and `nnqsmul : ℚ≥0 → K → K`. Those two fields are needed to implement the `DivisionSemiring K → Algebra ℚ≥0 K` instance since we need to control the specific definitions for some special cases of `K` (in particular `K = ℚ≥0` itself). See also note [forgetful inheritance]. If the semifield has positive characteristic `p`, our division by zero convention forces `nnratCast (1 / p) = 1 / 0 = 0`. -/ class Semifield (α : Type*) extends CommSemiring α, DivisionSemiring α, CommGroupWithZero α /-- A `Field` is a `CommRing` with multiplicative inverses for nonzero elements. An instance of `Field K` includes maps `ratCast : ℚ → K` and `qsmul : ℚ → K → K`. Those two fields are needed to implement the `DivisionRing K → Algebra ℚ K` instance since we need to control the specific definitions for some special cases of `K` (in particular `K = ℚ` itself). See also note [forgetful inheritance]. If the field has positive characteristic `p`, our division by zero convention forces `ratCast (1 / p) = 1 / 0 = 0`. -/ class Field (K : Type u) extends CommRing K, DivisionRing K -- see Note [lower instance priority] instance (priority := 100) Field.toSemifield [Field α] : Semifield α := { ‹Field α› with } namespace NNRat variable [DivisionSemiring α] instance (priority := 100) smulDivisionSemiring : SMul ℚ≥0 α := ⟨DivisionSemiring.nnqsmul⟩ lemma cast_def (q : ℚ≥0) : (q : α) = q.num / q.den := DivisionSemiring.nnratCast_def _ lemma smul_def (q : ℚ≥0) (a : α) : q • a = q * a := DivisionSemiring.nnqsmul_def q a variable (α) @[simp] lemma smul_one_eq_cast (q : ℚ≥0) : q • (1 : α) = q := by rw [NNRat.smul_def, mul_one] @[deprecated (since := "2024-05-03")] alias smul_one_eq_coe := smul_one_eq_cast end NNRat namespace Rat variable [DivisionRing K] {a b : K} lemma cast_def (q : ℚ) : (q : K) = q.num / q.den := DivisionRing.ratCast_def _ lemma cast_mk' (a b h1 h2) : ((⟨a, b, h1, h2⟩ : ℚ) : K) = a / b := cast_def _ instance (priority := 100) smulDivisionRing : SMul ℚ K := ⟨DivisionRing.qsmul⟩ theorem smul_def (a : ℚ) (x : K) : a • x = ↑a * x := DivisionRing.qsmul_def a x @[simp] theorem smul_one_eq_cast (A : Type*) [DivisionRing A] (m : ℚ) : m • (1 : A) = ↑m := by rw [Rat.smul_def, mul_one] @[deprecated (since := "2024-05-03")] alias smul_one_eq_coe := smul_one_eq_cast end Rat /-- `OfScientific.ofScientific` is the simp-normal form. -/ @[simp] theorem Rat.ofScientific_eq_ofScientific (m : ℕ) (s : Bool) (e : ℕ) : Rat.ofScientific (OfNat.ofNat m) s (OfNat.ofNat e) = OfScientific.ofScientific m s e := rfl
Algebra\Field\Equiv.lean
/- Copyright (c) 2023 Junyan Xu. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Junyan Xu -/ import Mathlib.Algebra.Field.IsField import Mathlib.Algebra.GroupWithZero.Hom /-! # If a semiring is a field, any isomorphic semiring is also a field. This is in a separate file to avoiding need to import `Field` in `Mathlib.Algebra.Ring.Equiv.` -/ namespace MulEquiv protected theorem isField {A : Type*} (B : Type*) [Semiring A] [Semiring B] (hB : IsField B) (e : A ≃* B) : IsField A where exists_pair_ne := have ⟨x, y, h⟩ := hB.exists_pair_ne; ⟨e.symm x, e.symm y, e.symm.injective.ne h⟩ mul_comm := fun x y => e.injective <| by rw [map_mul, map_mul, hB.mul_comm] mul_inv_cancel := fun h => by obtain ⟨a', he⟩ := hB.mul_inv_cancel ((e.injective.ne h).trans_eq <| map_zero e) exact ⟨e.symm a', e.injective <| by rw [map_mul, map_one, e.apply_symm_apply, he]⟩ end MulEquiv
Algebra\Field\IsField.lean
/- Copyright (c) 2014 Robert Lewis. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Robert Lewis, Leonardo de Moura, Johannes Hölzl, Mario Carneiro -/ import Mathlib.Algebra.Field.Defs import Mathlib.Tactic.Common /-! # `IsField` predicate Predicate on a (semi)ring that it is a (semi)field, i.e. that the multiplication is commutative, that it has more than one element and that all non-zero elements have a multiplicative inverse. In contrast to `Field`, which contains the data of a function associating to an element of the field its multiplicative inverse, this predicate only assumes the existence and can therefore more easily be used to e.g. transfer along ring isomorphisms. -/ universe u section IsField /-- A predicate to express that a (semi)ring is a (semi)field. This is mainly useful because such a predicate does not contain data, and can therefore be easily transported along ring isomorphisms. Additionally, this is useful when trying to prove that a particular ring structure extends to a (semi)field. -/ structure IsField (R : Type u) [Semiring R] : Prop where /-- For a semiring to be a field, it must have two distinct elements. -/ exists_pair_ne : ∃ x y : R, x ≠ y /-- Fields are commutative. -/ mul_comm : ∀ x y : R, x * y = y * x /-- Nonzero elements have multiplicative inverses. -/ mul_inv_cancel : ∀ {a : R}, a ≠ 0 → ∃ b, a * b = 1 /-- Transferring from `Semifield` to `IsField`. -/ theorem Semifield.toIsField (R : Type u) [Semifield R] : IsField R where __ := ‹Semifield R› mul_inv_cancel {a} ha := ⟨a⁻¹, mul_inv_cancel ha⟩ /-- Transferring from `Field` to `IsField`. -/ theorem Field.toIsField (R : Type u) [Field R] : IsField R := Semifield.toIsField _ @[simp] theorem IsField.nontrivial {R : Type u} [Semiring R] (h : IsField R) : Nontrivial R := ⟨h.exists_pair_ne⟩ @[simp] theorem not_isField_of_subsingleton (R : Type u) [Semiring R] [Subsingleton R] : ¬IsField R := fun h => let ⟨_, _, h⟩ := h.exists_pair_ne h (Subsingleton.elim _ _) open Classical in /-- Transferring from `IsField` to `Semifield`. -/ noncomputable def IsField.toSemifield {R : Type u} [Semiring R] (h : IsField R) : Semifield R where __ := ‹Semiring R› __ := h inv a := if ha : a = 0 then 0 else Classical.choose (h.mul_inv_cancel ha) inv_zero := dif_pos rfl mul_inv_cancel a ha := by convert Classical.choose_spec (h.mul_inv_cancel ha); exact dif_neg ha nnqsmul := _ nnqsmul_def q a := rfl /-- Transferring from `IsField` to `Field`. -/ noncomputable def IsField.toField {R : Type u} [Ring R] (h : IsField R) : Field R := { ‹Ring R›, IsField.toSemifield h with qsmul := _ qsmul_def := fun q a => rfl } /-- For each field, and for each nonzero element of said field, there is a unique inverse. Since `IsField` doesn't remember the data of an `inv` function and as such, a lemma that there is a unique inverse could be useful. -/ theorem uniq_inv_of_isField (R : Type u) [Ring R] (hf : IsField R) : ∀ x : R, x ≠ 0 → ∃! y : R, x * y = 1 := by intro x hx apply exists_unique_of_exists_of_unique · exact hf.mul_inv_cancel hx · intro y z hxy hxz calc y = y * (x * z) := by rw [hxz, mul_one] _ = x * y * z := by rw [← mul_assoc, hf.mul_comm y x] _ = z := by rw [hxy, one_mul] end IsField
Algebra\Field\MinimalAxioms.lean
/- Copyright (c) 2023 Chris Hughes. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Chris Hughes -/ import Mathlib.Algebra.Field.Defs import Mathlib.Algebra.Ring.MinimalAxioms /-! # Minimal Axioms for a Field This file defines constructors to define a `Field` structure on a Type, while proving a minimum number of equalities. ## Main Definitions * `Field.ofMinimalAxioms`: Define a `Field` structure on a Type by proving a minimized set of axioms -/ universe u /-- Define a `Field` structure on a Type by proving a minimized set of axioms. Note that this uses the default definitions for `npow`, `nsmul`, `zsmul`, `div` and `sub` See note [reducible non-instances]. -/ abbrev Field.ofMinimalAxioms (K : Type u) [Add K] [Mul K] [Neg K] [Inv K] [Zero K] [One K] (add_assoc : ∀ a b c : K, a + b + c = a + (b + c)) (zero_add : ∀ a : K, 0 + a = a) (add_left_neg : ∀ a : K, -a + a = 0) (mul_assoc : ∀ a b c : K, a * b * c = a * (b * c)) (mul_comm : ∀ a b : K, a * b = b * a) (one_mul : ∀ a : K, 1 * a = a) (mul_inv_cancel : ∀ a : K, a ≠ 0 → a * a⁻¹ = 1) (inv_zero : (0 : K)⁻¹ = 0) (left_distrib : ∀ a b c : K, a * (b + c) = a * b + a * c) (exists_pair_ne : ∃ x y : K, x ≠ y) : Field K := letI := CommRing.ofMinimalAxioms add_assoc zero_add add_left_neg mul_assoc mul_comm one_mul left_distrib { exists_pair_ne := exists_pair_ne mul_inv_cancel := mul_inv_cancel inv_zero := inv_zero nnqsmul := _ nnqsmul_def := fun q a => rfl qsmul := _ qsmul_def := fun q a => rfl }
Algebra\Field\Opposite.lean
/- Copyright (c) 2018 Kenny Lau. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Kenny Lau -/ import Mathlib.Algebra.Field.Defs import Mathlib.Algebra.Ring.Opposite import Mathlib.Data.Int.Cast.Lemmas /-! # Field structure on the multiplicative/additive opposite -/ variable {α : Type*} namespace MulOpposite @[to_additive] instance instNNRatCast [NNRatCast α] : NNRatCast αᵐᵒᵖ := ⟨fun q ↦ op q⟩ @[to_additive] instance instRatCast [RatCast α] : RatCast αᵐᵒᵖ := ⟨fun q ↦ op q⟩ @[to_additive (attr := simp, norm_cast)] lemma op_nnratCast [NNRatCast α] (q : ℚ≥0) : op (q : α) = q := rfl @[to_additive (attr := simp, norm_cast)] lemma unop_nnratCast [NNRatCast α] (q : ℚ≥0) : unop (q : αᵐᵒᵖ) = q := rfl @[to_additive (attr := simp, norm_cast)] lemma op_ratCast [RatCast α] (q : ℚ) : op (q : α) = q := rfl @[to_additive (attr := simp, norm_cast)] lemma unop_ratCast [RatCast α] (q : ℚ) : unop (q : αᵐᵒᵖ) = q := rfl instance instDivisionSemiring [DivisionSemiring α] : DivisionSemiring αᵐᵒᵖ where __ := instSemiring __ := instGroupWithZero nnqsmul := _ nnqsmul_def := fun q a => rfl nnratCast_def q := unop_injective $ by rw [unop_nnratCast, unop_div, unop_natCast, unop_natCast, NNRat.cast_def, div_eq_mul_inv, Nat.cast_comm] instance instDivisionRing [DivisionRing α] : DivisionRing αᵐᵒᵖ where __ := instRing __ := instDivisionSemiring qsmul := _ qsmul_def := fun q a => rfl ratCast_def q := unop_injective <| by rw [unop_ratCast, Rat.cast_def, unop_div, unop_natCast, unop_intCast, Int.commute_cast, div_eq_mul_inv] instance instSemifield [Semifield α] : Semifield αᵐᵒᵖ where __ := instCommSemiring __ := instDivisionSemiring instance instField [Field α] : Field αᵐᵒᵖ where __ := instCommRing __ := instDivisionRing end MulOpposite namespace AddOpposite instance instDivisionSemiring [DivisionSemiring α] : DivisionSemiring αᵃᵒᵖ where __ := instSemiring __ := instGroupWithZero nnqsmul := _ nnqsmul_def := fun q a => rfl nnratCast_def q := unop_injective $ by rw [unop_nnratCast, unop_div, unop_natCast, unop_natCast, NNRat.cast_def, div_eq_mul_inv] instance instDivisionRing [DivisionRing α] : DivisionRing αᵃᵒᵖ where __ := instRing __ := instDivisionSemiring qsmul := _ qsmul_def := fun q a => rfl ratCast_def q := unop_injective <| by rw [unop_ratCast, Rat.cast_def, unop_div, unop_natCast, unop_intCast, div_eq_mul_inv] instance instSemifield [Semifield α] : Semifield αᵃᵒᵖ where __ := instCommSemiring __ := instDivisionSemiring instance instField [Field α] : Field αᵃᵒᵖ where __ := instCommRing __ := instDivisionRing end AddOpposite
Algebra\Field\Power.lean
/- Copyright (c) 2014 Robert Lewis. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Robert Lewis, Leonardo de Moura, Johannes Hölzl, Mario Carneiro -/ import Mathlib.Algebra.Field.Defs import Mathlib.Algebra.Ring.Int /-! # Results about powers in fields or division rings. This file exists to ensure we can define `Field` with minimal imports, so contains some lemmas about powers of elements which need imports beyond those needed for the basic definition. -/ variable {α : Type*} section DivisionRing variable [DivisionRing α] {n : ℤ} theorem Odd.neg_zpow (h : Odd n) (a : α) : (-a) ^ n = -a ^ n := by have hn : n ≠ 0 := by rintro rfl; exact Int.odd_iff_not_even.1 h even_zero obtain ⟨k, rfl⟩ := h simp_rw [zpow_add' (.inr (.inl hn)), zpow_one, zpow_mul, zpow_two, neg_mul_neg, neg_mul_eq_mul_neg] theorem Odd.neg_one_zpow (h : Odd n) : (-1 : α) ^ n = -1 := by rw [h.neg_zpow, one_zpow] end DivisionRing
Algebra\Field\Rat.lean
/- Copyright (c) 2019 Johannes Hölzl. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Johannes Hölzl, Mario Carneiro -/ import Mathlib.Algebra.Field.Defs import Mathlib.Data.NNRat.Defs /-! # The rational numbers form a field This file contains the field instance on the rational numbers. See note [foundational algebra order theory]. ## TODO Move the `Semifield ℚ≥0` instance here. This will involve proving it by hand rather than relying on the `Nonneg` machinery. ## Tags rat, rationals, field, ℚ, numerator, denominator, num, denom -/ namespace Rat instance instField : Field ℚ where __ := commRing __ := commGroupWithZero nnqsmul := _ nnqsmul_def := fun q a => rfl qsmul := _ qsmul_def := fun q a => rfl nnratCast_def q := by rw [← NNRat.den_coe, ← Int.cast_natCast q.num, ← NNRat.num_coe]; exact(num_div_den _).symm ratCast_def q := (num_div_den _).symm /-! ### Extra instances to short-circuit type class resolution These also prevent non-computable instances being used to construct these instances non-computably. -/ instance instDivisionRing : DivisionRing ℚ := inferInstance end Rat
Algebra\Field\Subfield.lean
/- Copyright (c) 2020 Anne Baanen. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Anne Baanen -/ import Mathlib.Algebra.Ring.Subring.Basic import Mathlib.Algebra.Algebra.Defs import Mathlib.Data.Rat.Cast.Defs /-! # Subfields Let `K` be a division ring, for example a field. This file defines the "bundled" subfield type `Subfield K`, a type whose terms correspond to subfields of `K`. Note we do not require the "subfields" to be commutative, so they are really sub-division rings / skew fields. This is the preferred way to talk about subfields in mathlib. Unbundled subfields (`s : Set K` and `IsSubfield s`) are not in this file, and they will ultimately be deprecated. We prove that subfields are a complete lattice, and that you can `map` (pushforward) and `comap` (pull back) them along ring homomorphisms. We define the `closure` construction from `Set K` to `Subfield K`, sending a subset of `K` to the subfield it generates, and prove that it is a Galois insertion. ## Main definitions Notation used here: `(K : Type u) [DivisionRing K] (L : Type u) [DivisionRing L] (f g : K →+* L)` `(A : Subfield K) (B : Subfield L) (s : Set K)` * `Subfield K` : the type of subfields of a division ring `K`. * `instance : CompleteLattice (Subfield K)` : the complete lattice structure on the subfields. * `Subfield.closure` : subfield closure of a set, i.e., the smallest subfield that includes the set. * `Subfield.gi` : `closure : Set M → Subfield M` and coercion `(↑) : Subfield M → Set M` form a `GaloisInsertion`. * `comap f B : Subfield K` : the preimage of a subfield `B` along the ring homomorphism `f` * `map f A : Subfield L` : the image of a subfield `A` along the ring homomorphism `f`. * `f.fieldRange : Subfield L` : the range of the ring homomorphism `f`. * `eqLocusField f g : Subfield K` : given ring homomorphisms `f g : K →+* R`, the subfield of `K` where `f x = g x` ## Implementation notes A subfield is implemented as a subring which is closed under `⁻¹`. Lattice inclusion (e.g. `≤` and `⊓`) is used rather than set notation (`⊆` and `∩`), although `∈` is defined as membership of a subfield's underlying set. ## Tags subfield, subfields -/ universe u v w variable {K : Type u} {L : Type v} {M : Type w} variable [DivisionRing K] [DivisionRing L] [DivisionRing M] /-- `SubfieldClass S K` states `S` is a type of subsets `s ⊆ K` closed under field operations. -/ class SubfieldClass (S K : Type*) [DivisionRing K] [SetLike S K] extends SubringClass S K, InvMemClass S K : Prop namespace SubfieldClass variable (S : Type*) [SetLike S K] [h : SubfieldClass S K] -- See note [lower instance priority] /-- A subfield contains `1`, products and inverses. Be assured that we're not actually proving that subfields are subgroups: `SubgroupClass` is really an abbreviation of `SubgroupWithOrWithoutZeroClass`. -/ instance (priority := 100) toSubgroupClass : SubgroupClass S K := { h with } variable {S} {x : K} @[aesop safe apply (rule_sets := [SetLike])] lemma nnratCast_mem (s : S) (q : ℚ≥0) : (q : K) ∈ s := by simpa only [NNRat.cast_def] using div_mem (natCast_mem s q.num) (natCast_mem s q.den) @[aesop safe apply (rule_sets := [SetLike])] lemma ratCast_mem (s : S) (q : ℚ) : (q : K) ∈ s := by simpa only [Rat.cast_def] using div_mem (intCast_mem s q.num) (natCast_mem s q.den) instance instNNRatCast (s : S) : NNRatCast s where nnratCast q := ⟨q, nnratCast_mem s q⟩ instance instRatCast (s : S) : RatCast s where ratCast q := ⟨q, ratCast_mem s q⟩ @[simp, norm_cast] lemma coe_nnratCast (s : S) (q : ℚ≥0) : ((q : s) : K) = q := rfl @[simp, norm_cast] lemma coe_ratCast (s : S) (x : ℚ) : ((x : s) : K) = x := rfl @[aesop safe apply (rule_sets := [SetLike])] lemma nnqsmul_mem (s : S) (q : ℚ≥0) (hx : x ∈ s) : q • x ∈ s := by simpa only [NNRat.smul_def] using mul_mem (nnratCast_mem _ _) hx @[aesop safe apply (rule_sets := [SetLike])] lemma qsmul_mem (s : S) (q : ℚ) (hx : x ∈ s) : q • x ∈ s := by simpa only [Rat.smul_def] using mul_mem (ratCast_mem _ _) hx @[deprecated (since := "2024-04-05")] alias coe_rat_cast := coe_ratCast @[deprecated (since := "2024-04-05")] alias coe_rat_mem := ratCast_mem @[deprecated (since := "2024-04-05")] alias rat_smul_mem := qsmul_mem @[aesop safe apply (rule_sets := [SetLike])] lemma ofScientific_mem (s : S) {b : Bool} {n m : ℕ} : (OfScientific.ofScientific n b m : K) ∈ s := SubfieldClass.nnratCast_mem s (OfScientific.ofScientific n b m) instance instSMulNNRat (s : S) : SMul ℚ≥0 s where smul q x := ⟨q • x, nnqsmul_mem s q x.2⟩ instance instSMulRat (s : S) : SMul ℚ s where smul q x := ⟨q • x, qsmul_mem s q x.2⟩ @[simp, norm_cast] lemma coe_nnqsmul (s : S) (q : ℚ≥0) (x : s) : ↑(q • x) = q • (x : K) := rfl @[simp, norm_cast] lemma coe_qsmul (s : S) (q : ℚ) (x : s) : ↑(q • x) = q • (x : K) := rfl variable (S) /-- A subfield inherits a division ring structure -/ instance (priority := 75) toDivisionRing (s : S) : DivisionRing s := Subtype.coe_injective.divisionRing ((↑) : s → K) (by rfl) (by rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) (coe_nnqsmul _) (coe_qsmul _) (by intros; rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) -- Prefer subclasses of `Field` over subclasses of `SubfieldClass`. /-- A subfield of a field inherits a field structure -/ instance (priority := 75) toField {K} [Field K] [SetLike S K] [SubfieldClass S K] (s : S) : Field s := Subtype.coe_injective.field ((↑) : s → K) (by rfl) (by rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) (coe_nnqsmul _) (coe_qsmul _) (by intros; rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) (by intros; rfl) end SubfieldClass /-- `Subfield R` is the type of subfields of `R`. A subfield of `R` is a subset `s` that is a multiplicative submonoid and an additive subgroup. Note in particular that it shares the same 0 and 1 as R. -/ structure Subfield (K : Type u) [DivisionRing K] extends Subring K where /-- A subfield is closed under multiplicative inverses. -/ inv_mem' : ∀ x ∈ carrier, x⁻¹ ∈ carrier /-- Reinterpret a `Subfield` as a `Subring`. -/ add_decl_doc Subfield.toSubring namespace Subfield /-- The underlying `AddSubgroup` of a subfield. -/ def toAddSubgroup (s : Subfield K) : AddSubgroup K := { s.toSubring.toAddSubgroup with } -- Porting note: toSubmonoid already exists -- /-- The underlying submonoid of a subfield. -/ -- def toSubmonoid (s : Subfield K) : Submonoid K := -- { s.toSubring.toSubmonoid with } instance : SetLike (Subfield K) K where coe s := s.carrier coe_injective' p q h := by cases p; cases q; congr; exact SetLike.ext' h instance : SubfieldClass (Subfield K) K where add_mem {s} := s.add_mem' zero_mem s := s.zero_mem' neg_mem {s} := s.neg_mem' mul_mem {s} := s.mul_mem' one_mem s := s.one_mem' inv_mem {s} := s.inv_mem' _ -- @[simp] -- Porting note (#10618): simp can prove this (with `coe_toSubring`, which comes later) theorem mem_carrier {s : Subfield K} {x : K} : x ∈ s.carrier ↔ x ∈ s := Iff.rfl -- Porting note: in lean 3, `S` was type `Set K` @[simp] theorem mem_mk {S : Subring K} {x : K} (h) : x ∈ (⟨S, h⟩ : Subfield K) ↔ x ∈ S := Iff.rfl @[simp] theorem coe_set_mk (S : Subring K) (h) : ((⟨S, h⟩ : Subfield K) : Set K) = S := rfl @[simp] theorem mk_le_mk {S S' : Subring K} (h h') : (⟨S, h⟩ : Subfield K) ≤ (⟨S', h'⟩ : Subfield K) ↔ S ≤ S' := Iff.rfl /-- Two subfields are equal if they have the same elements. -/ @[ext] theorem ext {S T : Subfield K} (h : ∀ x, x ∈ S ↔ x ∈ T) : S = T := SetLike.ext h /-- Copy of a subfield with a new `carrier` equal to the old one. Useful to fix definitional equalities. -/ protected def copy (S : Subfield K) (s : Set K) (hs : s = ↑S) : Subfield K := { S.toSubring.copy s hs with carrier := s inv_mem' := hs.symm ▸ S.inv_mem' } @[simp] theorem coe_copy (S : Subfield K) (s : Set K) (hs : s = ↑S) : (S.copy s hs : Set K) = s := rfl theorem copy_eq (S : Subfield K) (s : Set K) (hs : s = ↑S) : S.copy s hs = S := SetLike.coe_injective hs @[simp] theorem coe_toSubring (s : Subfield K) : (s.toSubring : Set K) = s := rfl @[simp] theorem mem_toSubring (s : Subfield K) (x : K) : x ∈ s.toSubring ↔ x ∈ s := Iff.rfl end Subfield /-- A `Subring` containing inverses is a `Subfield`. -/ def Subring.toSubfield (s : Subring K) (hinv : ∀ x ∈ s, x⁻¹ ∈ s) : Subfield K := { s with inv_mem' := hinv } namespace Subfield variable (s t : Subfield K) section DerivedFromSubfieldClass /-- A subfield contains the field's 1. -/ protected theorem one_mem : (1 : K) ∈ s := one_mem s /-- A subfield contains the field's 0. -/ protected theorem zero_mem : (0 : K) ∈ s := zero_mem s /-- A subfield is closed under multiplication. -/ protected theorem mul_mem {x y : K} : x ∈ s → y ∈ s → x * y ∈ s := mul_mem /-- A subfield is closed under addition. -/ protected theorem add_mem {x y : K} : x ∈ s → y ∈ s → x + y ∈ s := add_mem /-- A subfield is closed under negation. -/ protected theorem neg_mem {x : K} : x ∈ s → -x ∈ s := neg_mem /-- A subfield is closed under subtraction. -/ protected theorem sub_mem {x y : K} : x ∈ s → y ∈ s → x - y ∈ s := sub_mem /-- A subfield is closed under inverses. -/ protected theorem inv_mem {x : K} : x ∈ s → x⁻¹ ∈ s := inv_mem /-- A subfield is closed under division. -/ protected theorem div_mem {x y : K} : x ∈ s → y ∈ s → x / y ∈ s := div_mem /-- Product of a list of elements in a subfield is in the subfield. -/ protected theorem list_prod_mem {l : List K} : (∀ x ∈ l, x ∈ s) → l.prod ∈ s := list_prod_mem /-- Sum of a list of elements in a subfield is in the subfield. -/ protected theorem list_sum_mem {l : List K} : (∀ x ∈ l, x ∈ s) → l.sum ∈ s := list_sum_mem /-- Sum of a multiset of elements in a `Subfield` is in the `Subfield`. -/ protected theorem multiset_sum_mem (m : Multiset K) : (∀ a ∈ m, a ∈ s) → m.sum ∈ s := multiset_sum_mem m /-- Sum of elements in a `Subfield` indexed by a `Finset` is in the `Subfield`. -/ protected theorem sum_mem {ι : Type*} {t : Finset ι} {f : ι → K} (h : ∀ c ∈ t, f c ∈ s) : (∑ i ∈ t, f i) ∈ s := sum_mem h protected theorem pow_mem {x : K} (hx : x ∈ s) (n : ℕ) : x ^ n ∈ s := pow_mem hx n protected theorem zsmul_mem {x : K} (hx : x ∈ s) (n : ℤ) : n • x ∈ s := zsmul_mem hx n protected theorem intCast_mem (n : ℤ) : (n : K) ∈ s := intCast_mem s n @[deprecated (since := "2024-04-05")] alias coe_int_mem := intCast_mem theorem zpow_mem {x : K} (hx : x ∈ s) (n : ℤ) : x ^ n ∈ s := by cases n · simpa using s.pow_mem hx _ · simpa [pow_succ'] using s.inv_mem (s.mul_mem hx (s.pow_mem hx _)) instance : Ring s := s.toSubring.toRing instance : Div s := ⟨fun x y => ⟨x / y, s.div_mem x.2 y.2⟩⟩ instance : Inv s := ⟨fun x => ⟨x⁻¹, s.inv_mem x.2⟩⟩ instance : Pow s ℤ := ⟨fun x z => ⟨x ^ z, s.zpow_mem x.2 z⟩⟩ -- TODO: Those are just special cases of `SubfieldClass.toDivisionRing`/`SubfieldClass.toField` instance toDivisionRing (s : Subfield K) : DivisionRing s := Subtype.coe_injective.divisionRing ((↑) : s → K) rfl rfl (fun _ _ ↦ rfl) (fun _ _ ↦ rfl) (fun _ ↦ rfl) (fun _ _ ↦ rfl) (fun _ ↦ rfl) (fun _ _ ↦ rfl) (fun _ _ ↦ rfl) (fun _ _ ↦ rfl) (fun _ _ ↦ rfl) (fun _ _ ↦ rfl) (fun _ _ ↦ rfl) (by intros; rfl) (fun _ ↦ rfl) (fun _ ↦ rfl) (by intros; rfl) fun _ ↦ rfl /-- A subfield inherits a field structure -/ instance toField {K} [Field K] (s : Subfield K) : Field s := Subtype.coe_injective.field ((↑) : s → K) rfl rfl (fun _ _ => rfl) (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) (by intros; rfl) (fun _ => rfl) (fun _ => rfl) (by intros; rfl) fun _ => rfl @[simp, norm_cast] theorem coe_add (x y : s) : (↑(x + y) : K) = ↑x + ↑y := rfl @[simp, norm_cast] theorem coe_sub (x y : s) : (↑(x - y) : K) = ↑x - ↑y := rfl @[simp, norm_cast] theorem coe_neg (x : s) : (↑(-x) : K) = -↑x := rfl @[simp, norm_cast] theorem coe_mul (x y : s) : (↑(x * y) : K) = ↑x * ↑y := rfl @[simp, norm_cast] theorem coe_div (x y : s) : (↑(x / y) : K) = ↑x / ↑y := rfl @[simp, norm_cast] theorem coe_inv (x : s) : (↑x⁻¹ : K) = (↑x)⁻¹ := rfl @[simp, norm_cast] theorem coe_zero : ((0 : s) : K) = 0 := rfl @[simp, norm_cast] theorem coe_one : ((1 : s) : K) = 1 := rfl end DerivedFromSubfieldClass /-- The embedding from a subfield of the field `K` to `K`. -/ def subtype (s : Subfield K) : s →+* K := { s.toSubmonoid.subtype, s.toAddSubgroup.subtype with toFun := (↑) } @[simp] theorem coe_subtype : ⇑(s.subtype) = ((↑) : s → K) := rfl variable (K) in theorem toSubring_subtype_eq_subtype (S : Subfield K) : S.toSubring.subtype = S.subtype := rfl /-! # Partial order -/ --@[simp] -- Porting note (#10618): simp can prove this theorem mem_toSubmonoid {s : Subfield K} {x : K} : x ∈ s.toSubmonoid ↔ x ∈ s := Iff.rfl @[simp] theorem coe_toSubmonoid : (s.toSubmonoid : Set K) = s := rfl @[simp] theorem mem_toAddSubgroup {s : Subfield K} {x : K} : x ∈ s.toAddSubgroup ↔ x ∈ s := Iff.rfl @[simp] theorem coe_toAddSubgroup : (s.toAddSubgroup : Set K) = s := rfl /-! # top -/ /-- The subfield of `K` containing all elements of `K`. -/ instance : Top (Subfield K) := ⟨{ (⊤ : Subring K) with inv_mem' := fun x _ => Subring.mem_top x }⟩ instance : Inhabited (Subfield K) := ⟨⊤⟩ @[simp] theorem mem_top (x : K) : x ∈ (⊤ : Subfield K) := Set.mem_univ x @[simp] theorem coe_top : ((⊤ : Subfield K) : Set K) = Set.univ := rfl /-- The ring equiv between the top element of `Subfield K` and `K`. -/ def topEquiv : (⊤ : Subfield K) ≃+* K := Subsemiring.topEquiv /-! # comap -/ variable (f : K →+* L) /-- The preimage of a subfield along a ring homomorphism is a subfield. -/ def comap (s : Subfield L) : Subfield K := { s.toSubring.comap f with inv_mem' := fun x hx => show f x⁻¹ ∈ s by rw [map_inv₀ f] exact s.inv_mem hx } @[simp] theorem coe_comap (s : Subfield L) : (s.comap f : Set K) = f ⁻¹' s := rfl @[simp] theorem mem_comap {s : Subfield L} {f : K →+* L} {x : K} : x ∈ s.comap f ↔ f x ∈ s := Iff.rfl theorem comap_comap (s : Subfield M) (g : L →+* M) (f : K →+* L) : (s.comap g).comap f = s.comap (g.comp f) := rfl /-! # map -/ /-- The image of a subfield along a ring homomorphism is a subfield. -/ def map (s : Subfield K) : Subfield L := { s.toSubring.map f with inv_mem' := by rintro _ ⟨x, hx, rfl⟩ exact ⟨x⁻¹, s.inv_mem hx, map_inv₀ f x⟩ } @[simp] theorem coe_map : (s.map f : Set L) = f '' s := rfl @[simp] theorem mem_map {f : K →+* L} {s : Subfield K} {y : L} : y ∈ s.map f ↔ ∃ x ∈ s, f x = y := by unfold map simp only [mem_mk, Subring.mem_mk, Subring.mem_toSubsemiring, Subring.mem_map, mem_toSubring] theorem map_map (g : L →+* M) (f : K →+* L) : (s.map f).map g = s.map (g.comp f) := SetLike.ext' <| Set.image_image _ _ _ theorem map_le_iff_le_comap {f : K →+* L} {s : Subfield K} {t : Subfield L} : s.map f ≤ t ↔ s ≤ t.comap f := Set.image_subset_iff theorem gc_map_comap (f : K →+* L) : GaloisConnection (map f) (comap f) := fun _ _ => map_le_iff_le_comap end Subfield namespace RingHom variable (g : L →+* M) (f : K →+* L) /-! # range -/ /-- The range of a ring homomorphism, as a subfield of the target. See Note [range copy pattern]. -/ def fieldRange : Subfield L := ((⊤ : Subfield K).map f).copy (Set.range f) Set.image_univ.symm @[simp] theorem coe_fieldRange : (f.fieldRange : Set L) = Set.range f := rfl @[simp] theorem mem_fieldRange {f : K →+* L} {y : L} : y ∈ f.fieldRange ↔ ∃ x, f x = y := Iff.rfl theorem fieldRange_eq_map : f.fieldRange = Subfield.map f ⊤ := by ext simp theorem map_fieldRange : f.fieldRange.map g = (g.comp f).fieldRange := by simpa only [fieldRange_eq_map] using (⊤ : Subfield K).map_map g f /-- The range of a morphism of fields is a fintype, if the domain is a fintype. Note that this instance can cause a diamond with `Subtype.Fintype` if `L` is also a fintype. -/ instance fintypeFieldRange [Fintype K] [DecidableEq L] (f : K →+* L) : Fintype f.fieldRange := Set.fintypeRange f end RingHom namespace Subfield /-! # inf -/ /-- The inf of two subfields is their intersection. -/ instance : Inf (Subfield K) := ⟨fun s t => { s.toSubring ⊓ t.toSubring with inv_mem' := fun _ hx => Subring.mem_inf.mpr ⟨s.inv_mem (Subring.mem_inf.mp hx).1, t.inv_mem (Subring.mem_inf.mp hx).2⟩ }⟩ @[simp] theorem coe_inf (p p' : Subfield K) : ((p ⊓ p' : Subfield K) : Set K) = p.carrier ∩ p'.carrier := rfl @[simp] theorem mem_inf {p p' : Subfield K} {x : K} : x ∈ p ⊓ p' ↔ x ∈ p ∧ x ∈ p' := Iff.rfl instance : InfSet (Subfield K) := ⟨fun S => { sInf (Subfield.toSubring '' S) with inv_mem' := by rintro x hx apply Subring.mem_sInf.mpr rintro _ ⟨p, p_mem, rfl⟩ exact p.inv_mem (Subring.mem_sInf.mp hx p.toSubring ⟨p, p_mem, rfl⟩) }⟩ @[simp, norm_cast] theorem coe_sInf (S : Set (Subfield K)) : ((sInf S : Subfield K) : Set K) = ⋂ s ∈ S, ↑s := show ((sInf (Subfield.toSubring '' S) : Subring K) : Set K) = ⋂ s ∈ S, ↑s by ext x rw [Subring.coe_sInf, Set.mem_iInter, Set.mem_iInter] exact ⟨fun h s s' ⟨s_mem, s'_eq⟩ => h s.toSubring _ ⟨⟨s, s_mem, rfl⟩, s'_eq⟩, fun h s s' ⟨⟨s'', s''_mem, s_eq⟩, (s'_eq : ↑s = s')⟩ => h s'' _ ⟨s''_mem, by simp [← s_eq, ← s'_eq]⟩⟩ theorem mem_sInf {S : Set (Subfield K)} {x : K} : x ∈ sInf S ↔ ∀ p ∈ S, x ∈ p := Subring.mem_sInf.trans ⟨fun h p hp => h p.toSubring ⟨p, hp, rfl⟩, fun h _ ⟨p', hp', p_eq⟩ => p_eq ▸ h p' hp'⟩ @[simp] theorem sInf_toSubring (s : Set (Subfield K)) : (sInf s).toSubring = ⨅ t ∈ s, Subfield.toSubring t := by ext x rw [mem_toSubring, mem_sInf] erw [Subring.mem_sInf] exact ⟨fun h p ⟨p', hp⟩ => hp ▸ Subring.mem_sInf.mpr fun p ⟨hp', hp⟩ => hp ▸ h _ hp', fun h p hp => h p.toSubring ⟨p, Subring.ext fun x => ⟨fun hx => Subring.mem_sInf.mp hx _ ⟨hp, rfl⟩, fun hx => Subring.mem_sInf.mpr fun p' ⟨_, p'_eq⟩ => p'_eq ▸ hx⟩⟩⟩ theorem isGLB_sInf (S : Set (Subfield K)) : IsGLB S (sInf S) := by have : ∀ {s t : Subfield K}, (s : Set K) ≤ t ↔ s ≤ t := by simp [SetLike.coe_subset_coe] refine IsGLB.of_image this ?_ convert isGLB_biInf (s := S) (f := SetLike.coe) exact coe_sInf _ /-- Subfields of a ring form a complete lattice. -/ instance : CompleteLattice (Subfield K) := { completeLatticeOfInf (Subfield K) isGLB_sInf with top := ⊤ le_top := fun _ _ _ => trivial inf := (· ⊓ ·) inf_le_left := fun _ _ _ => And.left inf_le_right := fun _ _ _ => And.right le_inf := fun _ _ _ h₁ h₂ _ hx => ⟨h₁ hx, h₂ hx⟩ } /-! # subfield closure of a subset -/ /-- The `Subfield` generated by a set. -/ def closure (s : Set K) : Subfield K := sInf {S | s ⊆ S} theorem mem_closure {x : K} {s : Set K} : x ∈ closure s ↔ ∀ S : Subfield K, s ⊆ S → x ∈ S := mem_sInf /-- The subfield generated by a set includes the set. -/ @[simp, aesop safe 20 apply (rule_sets := [SetLike])] theorem subset_closure {s : Set K} : s ⊆ closure s := fun _ hx => mem_closure.2 fun _ hS => hS hx theorem subring_closure_le (s : Set K) : Subring.closure s ≤ (closure s).toSubring := Subring.closure_le.mpr subset_closure theorem not_mem_of_not_mem_closure {s : Set K} {P : K} (hP : P ∉ closure s) : P ∉ s := fun h => hP (subset_closure h) /-- A subfield `t` includes `closure s` if and only if it includes `s`. -/ @[simp] theorem closure_le {s : Set K} {t : Subfield K} : closure s ≤ t ↔ s ⊆ t := ⟨Set.Subset.trans subset_closure, fun h _ hx => mem_closure.mp hx t h⟩ /-- Subfield closure of a set is monotone in its argument: if `s ⊆ t`, then `closure s ≤ closure t`. -/ theorem closure_mono ⦃s t : Set K⦄ (h : s ⊆ t) : closure s ≤ closure t := closure_le.2 <| Set.Subset.trans h subset_closure theorem closure_eq_of_le {s : Set K} {t : Subfield K} (h₁ : s ⊆ t) (h₂ : t ≤ closure s) : closure s = t := le_antisymm (closure_le.2 h₁) h₂ /-- An induction principle for closure membership. If `p` holds for `1`, and all elements of `s`, and is preserved under addition, negation, and multiplication, then `p` holds for all elements of the closure of `s`. -/ @[elab_as_elim] theorem closure_induction {s : Set K} {p : K → Prop} {x} (h : x ∈ closure s) (mem : ∀ x ∈ s, p x) (one : p 1) (add : ∀ x y, p x → p y → p (x + y)) (neg : ∀ x, p x → p (-x)) (inv : ∀ x, p x → p x⁻¹) (mul : ∀ x y, p x → p y → p (x * y)) : p x := by letI : Subfield K := ⟨⟨⟨⟨⟨p, by intro _ _; exact mul _ _⟩, one⟩, by intro _ _; exact add _ _, @add_neg_self K _ 1 ▸ add _ _ one (neg _ one)⟩, by intro _; exact neg _⟩, inv⟩ exact (closure_le (t := this)).2 mem h variable (K) /-- `closure` forms a Galois insertion with the coercion to set. -/ protected def gi : GaloisInsertion (@closure K _) (↑) where choice s _ := closure s gc _ _ := closure_le le_l_u _ := subset_closure choice_eq _ _ := rfl variable {K} /-- Closure of a subfield `S` equals `S`. -/ theorem closure_eq (s : Subfield K) : closure (s : Set K) = s := (Subfield.gi K).l_u_eq s @[simp] theorem closure_empty : closure (∅ : Set K) = ⊥ := (Subfield.gi K).gc.l_bot @[simp] theorem closure_univ : closure (Set.univ : Set K) = ⊤ := @coe_top K _ ▸ closure_eq ⊤ theorem closure_union (s t : Set K) : closure (s ∪ t) = closure s ⊔ closure t := (Subfield.gi K).gc.l_sup theorem closure_iUnion {ι} (s : ι → Set K) : closure (⋃ i, s i) = ⨆ i, closure (s i) := (Subfield.gi K).gc.l_iSup theorem closure_sUnion (s : Set (Set K)) : closure (⋃₀ s) = ⨆ t ∈ s, closure t := (Subfield.gi K).gc.l_sSup theorem map_sup (s t : Subfield K) (f : K →+* L) : (s ⊔ t).map f = s.map f ⊔ t.map f := (gc_map_comap f).l_sup theorem map_iSup {ι : Sort*} (f : K →+* L) (s : ι → Subfield K) : (iSup s).map f = ⨆ i, (s i).map f := (gc_map_comap f).l_iSup theorem comap_inf (s t : Subfield L) (f : K →+* L) : (s ⊓ t).comap f = s.comap f ⊓ t.comap f := (gc_map_comap f).u_inf theorem comap_iInf {ι : Sort*} (f : K →+* L) (s : ι → Subfield L) : (iInf s).comap f = ⨅ i, (s i).comap f := (gc_map_comap f).u_iInf @[simp] theorem map_bot (f : K →+* L) : (⊥ : Subfield K).map f = ⊥ := (gc_map_comap f).l_bot @[simp] theorem comap_top (f : K →+* L) : (⊤ : Subfield L).comap f = ⊤ := (gc_map_comap f).u_top /-- The underlying set of a non-empty directed sSup of subfields is just a union of the subfields. Note that this fails without the directedness assumption (the union of two subfields is typically not a subfield) -/ theorem mem_iSup_of_directed {ι} [hι : Nonempty ι] {S : ι → Subfield K} (hS : Directed (· ≤ ·) S) {x : K} : (x ∈ ⨆ i, S i) ↔ ∃ i, x ∈ S i := by let s : Subfield K := { __ := Subring.copy _ _ (Subring.coe_iSup_of_directed hS).symm inv_mem' := fun _ hx ↦ have ⟨i, hi⟩ := Set.mem_iUnion.mp hx Set.mem_iUnion.mpr ⟨i, (S i).inv_mem hi⟩ } have : iSup S = s := le_antisymm (iSup_le fun i ↦ le_iSup (fun i ↦ (S i : Set K)) i) (Set.iUnion_subset fun _ ↦ le_iSup S _) exact this ▸ Set.mem_iUnion theorem coe_iSup_of_directed {ι} [hι : Nonempty ι] {S : ι → Subfield K} (hS : Directed (· ≤ ·) S) : ((⨆ i, S i : Subfield K) : Set K) = ⋃ i, ↑(S i) := Set.ext fun x => by simp [mem_iSup_of_directed hS] theorem mem_sSup_of_directedOn {S : Set (Subfield K)} (Sne : S.Nonempty) (hS : DirectedOn (· ≤ ·) S) {x : K} : x ∈ sSup S ↔ ∃ s ∈ S, x ∈ s := by haveI : Nonempty S := Sne.to_subtype simp only [sSup_eq_iSup', mem_iSup_of_directed hS.directed_val, Subtype.exists, exists_prop] theorem coe_sSup_of_directedOn {S : Set (Subfield K)} (Sne : S.Nonempty) (hS : DirectedOn (· ≤ ·) S) : (↑(sSup S) : Set K) = ⋃ s ∈ S, ↑s := Set.ext fun x => by simp [mem_sSup_of_directedOn Sne hS] end Subfield namespace RingHom variable {s : Subfield K} open Subfield /-- Restriction of a ring homomorphism to its range interpreted as a subfield. -/ def rangeRestrictField (f : K →+* L) : K →+* f.fieldRange := f.rangeSRestrict @[simp] theorem coe_rangeRestrictField (f : K →+* L) (x : K) : (f.rangeRestrictField x : L) = f x := rfl section eqLocus variable {L : Type v} [Semiring L] /-- The subfield of elements `x : R` such that `f x = g x`, i.e., the equalizer of f and g as a subfield of R -/ def eqLocusField (f g : K →+* L) : Subfield K where __ := (f : K →+* L).eqLocus g inv_mem' _ := eq_on_inv₀ f g carrier := { x | f x = g x } /-- If two ring homomorphisms are equal on a set, then they are equal on its subfield closure. -/ theorem eqOn_field_closure {f g : K →+* L} {s : Set K} (h : Set.EqOn f g s) : Set.EqOn f g (closure s) := show closure s ≤ f.eqLocusField g from closure_le.2 h theorem eq_of_eqOn_subfield_top {f g : K →+* L} (h : Set.EqOn f g (⊤ : Subfield K)) : f = g := ext fun _ => h trivial theorem eq_of_eqOn_of_field_closure_eq_top {s : Set K} (hs : closure s = ⊤) {f g : K →+* L} (h : s.EqOn f g) : f = g := eq_of_eqOn_subfield_top <| hs ▸ eqOn_field_closure h end eqLocus theorem field_closure_preimage_le (f : K →+* L) (s : Set L) : closure (f ⁻¹' s) ≤ (closure s).comap f := closure_le.2 fun _ hx => SetLike.mem_coe.2 <| mem_comap.2 <| subset_closure hx /-- The image under a ring homomorphism of the subfield generated by a set equals the subfield generated by the image of the set. -/ theorem map_field_closure (f : K →+* L) (s : Set K) : (closure s).map f = closure (f '' s) := le_antisymm (map_le_iff_le_comap.2 <| le_trans (closure_mono <| Set.subset_preimage_image _ _) (field_closure_preimage_le _ _)) (closure_le.2 <| Set.image_subset _ subset_closure) end RingHom namespace Subfield open RingHom /-- The ring homomorphism associated to an inclusion of subfields. -/ def inclusion {S T : Subfield K} (h : S ≤ T) : S →+* T := S.subtype.codRestrict _ fun x => h x.2 @[simp] theorem fieldRange_subtype (s : Subfield K) : s.subtype.fieldRange = s := SetLike.ext' <| (coe_rangeS _).trans Subtype.range_coe end Subfield namespace RingEquiv variable {s t : Subfield K} /-- Makes the identity isomorphism from a proof two subfields of a multiplicative monoid are equal. -/ def subfieldCongr (h : s = t) : s ≃+* t := { Equiv.setCongr <| SetLike.ext'_iff.1 h with map_mul' := fun _ _ => rfl map_add' := fun _ _ => rfl } end RingEquiv namespace Subfield variable {s : Set K} theorem closure_preimage_le (f : K →+* L) (s : Set L) : closure (f ⁻¹' s) ≤ (closure s).comap f := closure_le.2 fun _ hx => SetLike.mem_coe.2 <| mem_comap.2 <| subset_closure hx section Commutative variable {K : Type u} [Field K] (s : Subfield K) /-- Product of a multiset of elements in a subfield is in the subfield. -/ protected theorem multiset_prod_mem (m : Multiset K) : (∀ a ∈ m, a ∈ s) → m.prod ∈ s := multiset_prod_mem m /-- Product of elements of a subfield indexed by a `Finset` is in the subfield. -/ protected theorem prod_mem {ι : Type*} {t : Finset ι} {f : ι → K} (h : ∀ c ∈ t, f c ∈ s) : (∏ i ∈ t, f i) ∈ s := prod_mem h instance toAlgebra : Algebra s K := RingHom.toAlgebra s.subtype /-- The `Subfield` generated by a set in a field. -/ private def commClosure (s : Set K) : Subfield K where carrier := {z : K | ∃ x ∈ Subring.closure s, ∃ y ∈ Subring.closure s, x / y = z} zero_mem' := ⟨0, Subring.zero_mem _, 1, Subring.one_mem _, div_one _⟩ one_mem' := ⟨1, Subring.one_mem _, 1, Subring.one_mem _, div_one _⟩ neg_mem' {x} := by rintro ⟨y, hy, z, hz, x_eq⟩ exact ⟨-y, Subring.neg_mem _ hy, z, hz, x_eq ▸ neg_div _ _⟩ inv_mem' x := by rintro ⟨y, hy, z, hz, x_eq⟩; exact ⟨z, hz, y, hy, x_eq ▸ (inv_div _ _).symm⟩ add_mem' x_mem y_mem := by -- Use `id` in the next 2 `obtain`s so that assumptions stay there for the `rwa`s below obtain ⟨nx, hnx, dx, hdx, rfl⟩ := id x_mem obtain ⟨ny, hny, dy, hdy, rfl⟩ := id y_mem by_cases hx0 : dx = 0; · rwa [hx0, div_zero, zero_add] by_cases hy0 : dy = 0; · rwa [hy0, div_zero, add_zero] exact ⟨nx * dy + dx * ny, Subring.add_mem _ (Subring.mul_mem _ hnx hdy) (Subring.mul_mem _ hdx hny), dx * dy, Subring.mul_mem _ hdx hdy, (div_add_div nx ny hx0 hy0).symm⟩ mul_mem' := by rintro _ _ ⟨nx, hnx, dx, hdx, rfl⟩ ⟨ny, hny, dy, hdy, rfl⟩ exact ⟨nx * ny, Subring.mul_mem _ hnx hny, dx * dy, Subring.mul_mem _ hdx hdy, (div_mul_div_comm _ _ _ _).symm⟩ private theorem commClosure_eq_closure {s : Set K} : commClosure s = closure s := le_antisymm (fun _ ⟨_, hy, _, hz, eq⟩ ↦ eq ▸ div_mem (subring_closure_le s hy) (subring_closure_le s hz)) (closure_le.mpr fun x hx ↦ ⟨x, Subring.subset_closure hx, 1, Subring.one_mem _, div_one x⟩) theorem mem_closure_iff {s : Set K} {x} : x ∈ closure s ↔ ∃ y ∈ Subring.closure s, ∃ z ∈ Subring.closure s, y / z = x := by rw [← commClosure_eq_closure]; rfl end Commutative end Subfield namespace Subfield theorem map_comap_eq (f : K →+* L) (s : Subfield L) : (s.comap f).map f = s ⊓ f.fieldRange := SetLike.coe_injective Set.image_preimage_eq_inter_range theorem map_comap_eq_self {f : K →+* L} {s : Subfield L} (h : s ≤ f.fieldRange) : (s.comap f).map f = s := by simpa only [inf_of_le_left h] using map_comap_eq f s theorem map_comap_eq_self_of_surjective {f : K →+* L} (hf : Function.Surjective f) (s : Subfield L) : (s.comap f).map f = s := SetLike.coe_injective (Set.image_preimage_eq _ hf) theorem comap_map (f : K →+* L) (s : Subfield K) : (s.map f).comap f = s := SetLike.coe_injective (Set.preimage_image_eq _ f.injective) end Subfield
Algebra\Field\ULift.lean
/- Copyright (c) 2023 Yaël Dillies. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Yaël Dillies -/ import Mathlib.Algebra.Field.Defs import Mathlib.Algebra.GroupWithZero.ULift import Mathlib.Algebra.Ring.ULift /-! # Field instances for `ULift` This file defines instances for field, semifield and related structures on `ULift` types. (Recall `ULift α` is just a "copy" of a type `α` in a higher universe.) -/ universe u v variable {α : Type u} {x y : ULift.{v} α} namespace ULift instance instNNRatCast [NNRatCast α] : NNRatCast (ULift α) where nnratCast q := up q instance instRatCast [RatCast α] : RatCast (ULift α) where ratCast q := up q @[simp, norm_cast] lemma up_nnratCast [NNRatCast α] (q : ℚ≥0) : up (q : α) = q := rfl @[simp, norm_cast] lemma down_nnratCast [NNRatCast α] (q : ℚ≥0) : down (q : ULift α) = q := rfl @[simp, norm_cast] lemma up_ratCast [RatCast α] (q : ℚ) : up (q : α) = q := rfl @[simp, norm_cast] lemma down_ratCast [RatCast α] (q : ℚ) : down (q : ULift α) = q := rfl instance divisionSemiring [DivisionSemiring α] : DivisionSemiring (ULift α) where toSemiring := semiring __ := groupWithZero nnqsmul_def _ _ := congrArg up <| DivisionSemiring.nnqsmul_def _ _ nnratCast_def _ := congrArg up <| DivisionSemiring.nnratCast_def _ instance semifield [Semifield α] : Semifield (ULift α) := { ULift.divisionSemiring, ULift.commGroupWithZero with } instance divisionRing [DivisionRing α] : DivisionRing (ULift α) where toRing := ring __ := groupWithZero nnqsmul_def _ _ := congrArg up <| DivisionSemiring.nnqsmul_def _ _ nnratCast_def _ := congrArg up <| DivisionSemiring.nnratCast_def _ qsmul_def _ _ := congrArg up <| DivisionRing.qsmul_def _ _ ratCast_def _ := congrArg up <| DivisionRing.ratCast_def _ instance field [Field α] : Field (ULift α) := { ULift.semifield, ULift.divisionRing with } end ULift
Algebra\FreeMonoid\Basic.lean
/- Copyright (c) 2019 Simon Hudon. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Simon Hudon, Yury Kudryashov -/ import Mathlib.Algebra.BigOperators.Group.List import Mathlib.Algebra.Group.Action.Defs import Mathlib.Algebra.Group.Units /-! # Free monoid over a given alphabet ## Main definitions * `FreeMonoid α`: free monoid over alphabet `α`; defined as a synonym for `List α` with multiplication given by `(++)`. * `FreeMonoid.of`: embedding `α → FreeMonoid α` sending each element `x` to `[x]`; * `FreeMonoid.lift`: natural equivalence between `α → M` and `FreeMonoid α →* M` * `FreeMonoid.map`: embedding of `α → β` into `FreeMonoid α →* FreeMonoid β` given by `List.map`. -/ variable {α : Type*} {β : Type*} {γ : Type*} {M : Type*} [Monoid M] {N : Type*} [Monoid N] /-- Free monoid over a given alphabet. -/ @[to_additive "Free nonabelian additive monoid over a given alphabet"] def FreeMonoid (α) := List α namespace FreeMonoid /-- The identity equivalence between `FreeMonoid α` and `List α`. -/ @[to_additive "The identity equivalence between `FreeAddMonoid α` and `List α`."] def toList : FreeMonoid α ≃ List α := Equiv.refl _ /-- The identity equivalence between `List α` and `FreeMonoid α`. -/ @[to_additive "The identity equivalence between `List α` and `FreeAddMonoid α`."] def ofList : List α ≃ FreeMonoid α := Equiv.refl _ @[to_additive (attr := simp)] theorem toList_symm : (@toList α).symm = ofList := rfl @[to_additive (attr := simp)] theorem ofList_symm : (@ofList α).symm = toList := rfl @[to_additive (attr := simp)] theorem toList_ofList (l : List α) : toList (ofList l) = l := rfl @[to_additive (attr := simp)] theorem ofList_toList (xs : FreeMonoid α) : ofList (toList xs) = xs := rfl @[to_additive (attr := simp)] theorem toList_comp_ofList : @toList α ∘ ofList = id := rfl @[to_additive (attr := simp)] theorem ofList_comp_toList : @ofList α ∘ toList = id := rfl @[to_additive] instance : CancelMonoid (FreeMonoid α) where one := ofList [] mul x y := ofList (toList x ++ toList y) mul_one := List.append_nil one_mul := List.nil_append mul_assoc := List.append_assoc mul_left_cancel _ _ _ := List.append_cancel_left mul_right_cancel _ _ _ := List.append_cancel_right @[to_additive] instance : Inhabited (FreeMonoid α) := ⟨1⟩ @[to_additive (attr := simp)] theorem toList_one : toList (1 : FreeMonoid α) = [] := rfl @[to_additive (attr := simp)] theorem ofList_nil : ofList ([] : List α) = 1 := rfl @[to_additive (attr := simp)] theorem toList_mul (xs ys : FreeMonoid α) : toList (xs * ys) = toList xs ++ toList ys := rfl @[to_additive (attr := simp)] theorem ofList_append (xs ys : List α) : ofList (xs ++ ys) = ofList xs * ofList ys := rfl @[to_additive (attr := simp)] theorem toList_prod (xs : List (FreeMonoid α)) : toList xs.prod = (xs.map toList).join := by induction xs <;> simp [*, List.join] @[to_additive (attr := simp)] theorem ofList_join (xs : List (List α)) : ofList xs.join = (xs.map ofList).prod := toList.injective <| by simp /-- Embeds an element of `α` into `FreeMonoid α` as a singleton list. -/ @[to_additive "Embeds an element of `α` into `FreeAddMonoid α` as a singleton list."] def of (x : α) : FreeMonoid α := ofList [x] @[to_additive (attr := simp)] theorem toList_of (x : α) : toList (of x) = [x] := rfl @[to_additive] theorem ofList_singleton (x : α) : ofList [x] = of x := rfl @[to_additive (attr := simp)] theorem ofList_cons (x : α) (xs : List α) : ofList (x :: xs) = of x * ofList xs := rfl @[to_additive] theorem toList_of_mul (x : α) (xs : FreeMonoid α) : toList (of x * xs) = x :: toList xs := rfl @[to_additive] theorem of_injective : Function.Injective (@of α) := List.singleton_injective /-- Recursor for `FreeMonoid` using `1` and `FreeMonoid.of x * xs` instead of `[]` and `x :: xs`. -/ @[to_additive (attr := elab_as_elim, induction_eliminator) "Recursor for `FreeAddMonoid` using `0` and FreeAddMonoid.of x + xs` instead of `[]` and `x :: xs`."] -- Porting note: change from `List.recOn` to `List.rec` since only the latter is computable def recOn {C : FreeMonoid α → Sort*} (xs : FreeMonoid α) (h0 : C 1) (ih : ∀ x xs, C xs → C (of x * xs)) : C xs := List.rec h0 ih xs @[to_additive (attr := simp)] theorem recOn_one {C : FreeMonoid α → Sort*} (h0 : C 1) (ih : ∀ x xs, C xs → C (of x * xs)) : @recOn α C 1 h0 ih = h0 := rfl @[to_additive (attr := simp)] theorem recOn_of_mul {C : FreeMonoid α → Sort*} (x : α) (xs : FreeMonoid α) (h0 : C 1) (ih : ∀ x xs, C xs → C (of x * xs)) : @recOn α C (of x * xs) h0 ih = ih x xs (recOn xs h0 ih) := rfl /-- A version of `List.cases_on` for `FreeMonoid` using `1` and `FreeMonoid.of x * xs` instead of `[]` and `x :: xs`. -/ @[to_additive (attr := elab_as_elim, cases_eliminator) "A version of `List.casesOn` for `FreeAddMonoid` using `0` and `FreeAddMonoid.of x + xs` instead of `[]` and `x :: xs`."] def casesOn {C : FreeMonoid α → Sort*} (xs : FreeMonoid α) (h0 : C 1) (ih : ∀ x xs, C (of x * xs)) : C xs := List.casesOn xs h0 ih @[to_additive (attr := simp)] theorem casesOn_one {C : FreeMonoid α → Sort*} (h0 : C 1) (ih : ∀ x xs, C (of x * xs)) : @casesOn α C 1 h0 ih = h0 := rfl @[to_additive (attr := simp)] theorem casesOn_of_mul {C : FreeMonoid α → Sort*} (x : α) (xs : FreeMonoid α) (h0 : C 1) (ih : ∀ x xs, C (of x * xs)) : @casesOn α C (of x * xs) h0 ih = ih x xs := rfl @[to_additive (attr := ext)] theorem hom_eq ⦃f g : FreeMonoid α →* M⦄ (h : ∀ x, f (of x) = g (of x)) : f = g := MonoidHom.ext fun l ↦ recOn l (f.map_one.trans g.map_one.symm) (fun x xs hxs ↦ by simp only [h, hxs, MonoidHom.map_mul]) /-- A variant of `List.prod` that has `[x].prod = x` true definitionally. The purpose is to make `FreeMonoid.lift_eval_of` true by `rfl`. -/ @[to_additive "A variant of `List.sum` that has `[x].sum = x` true definitionally. The purpose is to make `FreeAddMonoid.lift_eval_of` true by `rfl`."] def prodAux {M} [Monoid M] : List M → M | [] => 1 | (x :: xs) => List.foldl (· * ·) x xs @[to_additive] lemma prodAux_eq : ∀ l : List M, FreeMonoid.prodAux l = l.prod | [] => rfl | (_ :: xs) => congr_arg (fun x => List.foldl (· * ·) x xs) (one_mul _).symm /-- Equivalence between maps `α → M` and monoid homomorphisms `FreeMonoid α →* M`. -/ @[to_additive "Equivalence between maps `α → A` and additive monoid homomorphisms `FreeAddMonoid α →+ A`."] def lift : (α → M) ≃ (FreeMonoid α →* M) where toFun f := { toFun := fun l ↦ prodAux ((toList l).map f) map_one' := rfl map_mul' := fun _ _ ↦ by simp only [prodAux_eq, toList_mul, List.map_append, List.prod_append] } invFun f x := f (of x) left_inv f := rfl right_inv f := hom_eq fun x ↦ rfl @[to_additive (attr := simp)] theorem lift_ofList (f : α → M) (l : List α) : lift f (ofList l) = (l.map f).prod := prodAux_eq _ @[to_additive (attr := simp)] theorem lift_symm_apply (f : FreeMonoid α →* M) : lift.symm f = f ∘ of := rfl @[to_additive] theorem lift_apply (f : α → M) (l : FreeMonoid α) : lift f l = ((toList l).map f).prod := prodAux_eq _ @[to_additive] theorem lift_comp_of (f : α → M) : lift f ∘ of = f := rfl @[to_additive (attr := simp)] theorem lift_eval_of (f : α → M) (x : α) : lift f (of x) = f x := rfl @[to_additive (attr := simp)] theorem lift_restrict (f : FreeMonoid α →* M) : lift (f ∘ of) = f := lift.apply_symm_apply f @[to_additive] theorem comp_lift (g : M →* N) (f : α → M) : g.comp (lift f) = lift (g ∘ f) := by ext simp @[to_additive] theorem hom_map_lift (g : M →* N) (f : α → M) (x : FreeMonoid α) : g (lift f x) = lift (g ∘ f) x := DFunLike.ext_iff.1 (comp_lift g f) x /-- Define a multiplicative action of `FreeMonoid α` on `β`. -/ @[to_additive "Define an additive action of `FreeAddMonoid α` on `β`."] def mkMulAction (f : α → β → β) : MulAction (FreeMonoid α) β where smul l b := l.toList.foldr f b one_smul _ := rfl mul_smul _ _ _ := List.foldr_append _ _ _ _ @[to_additive] theorem smul_def (f : α → β → β) (l : FreeMonoid α) (b : β) : haveI := mkMulAction f l • b = l.toList.foldr f b := rfl @[to_additive] theorem ofList_smul (f : α → β → β) (l : List α) (b : β) : haveI := mkMulAction f ofList l • b = l.foldr f b := rfl @[to_additive (attr := simp)] theorem of_smul (f : α → β → β) (x : α) (y : β) : (haveI := mkMulAction f of x • y) = f x y := rfl /-- The unique monoid homomorphism `FreeMonoid α →* FreeMonoid β` that sends each `of x` to `of (f x)`. -/ @[to_additive "The unique additive monoid homomorphism `FreeAddMonoid α →+ FreeAddMonoid β` that sends each `of x` to `of (f x)`."] def map (f : α → β) : FreeMonoid α →* FreeMonoid β where toFun l := ofList <| l.toList.map f map_one' := rfl map_mul' _ _ := List.map_append _ _ _ @[to_additive (attr := simp)] theorem map_of (f : α → β) (x : α) : map f (of x) = of (f x) := rfl @[to_additive] theorem toList_map (f : α → β) (xs : FreeMonoid α) : toList (map f xs) = xs.toList.map f := rfl @[to_additive] theorem ofList_map (f : α → β) (xs : List α) : ofList (xs.map f) = map f (ofList xs) := rfl @[to_additive] theorem lift_of_comp_eq_map (f : α → β) : (lift fun x ↦ of (f x)) = map f := hom_eq fun _ ↦ rfl @[to_additive] theorem map_comp (g : β → γ) (f : α → β) : map (g ∘ f) = (map g).comp (map f) := hom_eq fun _ ↦ rfl @[to_additive (attr := simp)] theorem map_id : map (@id α) = MonoidHom.id (FreeMonoid α) := hom_eq fun _ ↦ rfl /-- The only invertible element of the free monoid is 1; this instance enables `units_eq_one`. -/ @[to_additive] instance uniqueUnits : Unique (FreeMonoid α)ˣ where uniq u := Units.ext <| toList.injective <| have : toList u.val ++ toList u.inv = [] := DFunLike.congr_arg toList u.val_inv (List.append_eq_nil.mp this).1 end FreeMonoid
Algebra\FreeMonoid\Count.lean
/- Copyright (c) 2022 Yury Kudryashov. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Yury Kudryashov -/ import Mathlib.Algebra.FreeMonoid.Basic /-! # `List.count` as a bundled homomorphism In this file we define `FreeMonoid.countP`, `FreeMonoid.count`, `FreeAddMonoid.countP`, and `FreeAddMonoid.count`. These are `List.countP` and `List.count` bundled as multiplicative and additive homomorphisms from `FreeMonoid` and `FreeAddMonoid`. We do not use `to_additive` because it can't map `Multiplicative ℕ` to `ℕ`. -/ variable {α : Type*} (p : α → Prop) [DecidablePred p] namespace FreeAddMonoid /-- `List.countP` as a bundled additive monoid homomorphism. -/ def countP : FreeAddMonoid α →+ ℕ where toFun := List.countP p map_zero' := List.countP_nil _ map_add' := List.countP_append _ theorem countP_of (x : α) : countP p (of x) = if p x = true then 1 else 0 := by simp [countP, List.countP, List.countP.go] theorem countP_apply (l : FreeAddMonoid α) : countP p l = List.countP p l := rfl /-- `List.count` as a bundled additive monoid homomorphism. -/ -- Porting note: was (x = ·) def count [DecidableEq α] (x : α) : FreeAddMonoid α →+ ℕ := countP (· = x) theorem count_of [DecidableEq α] (x y : α) : count x (of y) = (Pi.single x 1 : α → ℕ) y := by simp [Pi.single, Function.update, count, countP, List.countP, List.countP.go, Bool.beq_eq_decide_eq] theorem count_apply [DecidableEq α] (x : α) (l : FreeAddMonoid α) : count x l = List.count x l := rfl end FreeAddMonoid namespace FreeMonoid /-- `List.countP` as a bundled multiplicative monoid homomorphism. -/ def countP : FreeMonoid α →* Multiplicative ℕ := AddMonoidHom.toMultiplicative (FreeAddMonoid.countP p) theorem countP_of' (x : α) : countP p (of x) = if p x then Multiplicative.ofAdd 1 else Multiplicative.ofAdd 0 := by erw [FreeAddMonoid.countP_of] simp only [eq_iff_iff, iff_true, ofAdd_zero]; rfl theorem countP_of (x : α) : countP p (of x) = if p x then Multiplicative.ofAdd 1 else 1 := by rw [countP_of', ofAdd_zero] -- `rfl` is not transitive theorem countP_apply (l : FreeAddMonoid α) : countP p l = Multiplicative.ofAdd (List.countP p l) := rfl /-- `List.count` as a bundled additive monoid homomorphism. -/ def count [DecidableEq α] (x : α) : FreeMonoid α →* Multiplicative ℕ := countP (· = x) theorem count_apply [DecidableEq α] (x : α) (l : FreeAddMonoid α) : count x l = Multiplicative.ofAdd (List.count x l) := rfl theorem count_of [DecidableEq α] (x y : α) : count x (of y) = @Pi.mulSingle α (fun _ => Multiplicative ℕ) _ _ x (Multiplicative.ofAdd 1) y := by simp [count, countP_of, Pi.mulSingle_apply, eq_comm, Bool.beq_eq_decide_eq] end FreeMonoid
Algebra\GCDMonoid\Basic.lean
/- Copyright (c) 2018 Johannes Hölzl. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Johannes Hölzl, Jens Wagemaker -/ import Mathlib.Algebra.Associated.Basic import Mathlib.Algebra.Ring.Regular /-! # Monoids with normalization functions, `gcd`, and `lcm` This file defines extra structures on `CancelCommMonoidWithZero`s, including `IsDomain`s. ## Main Definitions * `NormalizationMonoid` * `GCDMonoid` * `NormalizedGCDMonoid` * `gcdMonoidOfGCD`, `gcdMonoidOfExistsGCD`, `normalizedGCDMonoidOfGCD`, `normalizedGCDMonoidOfExistsGCD` * `gcdMonoidOfLCM`, `gcdMonoidOfExistsLCM`, `normalizedGCDMonoidOfLCM`, `normalizedGCDMonoidOfExistsLCM` For the `NormalizedGCDMonoid` instances on `ℕ` and `ℤ`, see `Mathlib.Algebra.GCDMonoid.Nat`. ## Implementation Notes * `NormalizationMonoid` is defined by assigning to each element a `normUnit` such that multiplying by that unit normalizes the monoid, and `normalize` is an idempotent monoid homomorphism. This definition as currently implemented does casework on `0`. * `GCDMonoid` contains the definitions of `gcd` and `lcm` with the usual properties. They are both determined up to a unit. * `NormalizedGCDMonoid` extends `NormalizationMonoid`, so the `gcd` and `lcm` are always normalized. This makes `gcd`s of polynomials easier to work with, but excludes Euclidean domains, and monoids without zero. * `gcdMonoidOfGCD` and `normalizedGCDMonoidOfGCD` noncomputably construct a `GCDMonoid` (resp. `NormalizedGCDMonoid`) structure just from the `gcd` and its properties. * `gcdMonoidOfExistsGCD` and `normalizedGCDMonoidOfExistsGCD` noncomputably construct a `GCDMonoid` (resp. `NormalizedGCDMonoid`) structure just from a proof that any two elements have a (not necessarily normalized) `gcd`. * `gcdMonoidOfLCM` and `normalizedGCDMonoidOfLCM` noncomputably construct a `GCDMonoid` (resp. `NormalizedGCDMonoid`) structure just from the `lcm` and its properties. * `gcdMonoidOfExistsLCM` and `normalizedGCDMonoidOfExistsLCM` noncomputably construct a `GCDMonoid` (resp. `NormalizedGCDMonoid`) structure just from a proof that any two elements have a (not necessarily normalized) `lcm`. ## TODO * Port GCD facts about nats, definition of coprime * Generalize normalization monoids to commutative (cancellative) monoids with or without zero ## Tags divisibility, gcd, lcm, normalize -/ variable {α : Type*} -- Porting note: mathlib3 had a `@[protect_proj]` here, but adding `protected` to all the fields -- adds unnecessary clutter to later code /-- Normalization monoid: multiplying with `normUnit` gives a normal form for associated elements. -/ class NormalizationMonoid (α : Type*) [CancelCommMonoidWithZero α] where /-- `normUnit` assigns to each element of the monoid a unit of the monoid. -/ normUnit : α → αˣ /-- The proposition that `normUnit` maps `0` to the identity. -/ normUnit_zero : normUnit 0 = 1 /-- The proposition that `normUnit` respects multiplication of non-zero elements. -/ normUnit_mul : ∀ {a b}, a ≠ 0 → b ≠ 0 → normUnit (a * b) = normUnit a * normUnit b /-- The proposition that `normUnit` maps units to their inverses. -/ normUnit_coe_units : ∀ u : αˣ, normUnit u = u⁻¹ export NormalizationMonoid (normUnit normUnit_zero normUnit_mul normUnit_coe_units) attribute [simp] normUnit_coe_units normUnit_zero normUnit_mul section NormalizationMonoid variable [CancelCommMonoidWithZero α] [NormalizationMonoid α] @[simp] theorem normUnit_one : normUnit (1 : α) = 1 := normUnit_coe_units 1 -- Porting note (#11083): quite slow. Improve performance? /-- Chooses an element of each associate class, by multiplying by `normUnit` -/ def normalize : α →*₀ α where toFun x := x * normUnit x map_zero' := by simp only [normUnit_zero] exact mul_one (0 : α) map_one' := by dsimp only; rw [normUnit_one, one_mul]; rfl map_mul' x y := (by_cases fun hx : x = 0 => by dsimp only; rw [hx, zero_mul, zero_mul, zero_mul]) fun hx => (by_cases fun hy : y = 0 => by dsimp only; rw [hy, mul_zero, zero_mul, mul_zero]) fun hy => by simp only [normUnit_mul hx hy, Units.val_mul]; simp only [mul_assoc, mul_left_comm y] theorem associated_normalize (x : α) : Associated x (normalize x) := ⟨_, rfl⟩ theorem normalize_associated (x : α) : Associated (normalize x) x := (associated_normalize _).symm theorem associated_normalize_iff {x y : α} : Associated x (normalize y) ↔ Associated x y := ⟨fun h => h.trans (normalize_associated y), fun h => h.trans (associated_normalize y)⟩ theorem normalize_associated_iff {x y : α} : Associated (normalize x) y ↔ Associated x y := ⟨fun h => (associated_normalize _).trans h, fun h => (normalize_associated _).trans h⟩ theorem Associates.mk_normalize (x : α) : Associates.mk (normalize x) = Associates.mk x := Associates.mk_eq_mk_iff_associated.2 (normalize_associated _) @[simp] theorem normalize_apply (x : α) : normalize x = x * normUnit x := rfl -- Porting note (#10618): `simp` can prove this -- @[simp] theorem normalize_zero : normalize (0 : α) = 0 := normalize.map_zero -- Porting note (#10618): `simp` can prove this -- @[simp] theorem normalize_one : normalize (1 : α) = 1 := normalize.map_one theorem normalize_coe_units (u : αˣ) : normalize (u : α) = 1 := by simp theorem normalize_eq_zero {x : α} : normalize x = 0 ↔ x = 0 := ⟨fun hx => (associated_zero_iff_eq_zero x).1 <| hx ▸ associated_normalize _, by rintro rfl; exact normalize_zero⟩ theorem normalize_eq_one {x : α} : normalize x = 1 ↔ IsUnit x := ⟨fun hx => isUnit_iff_exists_inv.2 ⟨_, hx⟩, fun ⟨u, hu⟩ => hu ▸ normalize_coe_units u⟩ -- Porting note (#11083): quite slow. Improve performance? @[simp] theorem normUnit_mul_normUnit (a : α) : normUnit (a * normUnit a) = 1 := by nontriviality α using Subsingleton.elim a 0 obtain rfl | h := eq_or_ne a 0 · rw [normUnit_zero, zero_mul, normUnit_zero] · rw [normUnit_mul h (Units.ne_zero _), normUnit_coe_units, mul_inv_eq_one] theorem normalize_idem (x : α) : normalize (normalize x) = normalize x := by simp theorem normalize_eq_normalize {a b : α} (hab : a ∣ b) (hba : b ∣ a) : normalize a = normalize b := by nontriviality α rcases associated_of_dvd_dvd hab hba with ⟨u, rfl⟩ refine by_cases (by rintro rfl; simp only [zero_mul]) fun ha : a ≠ 0 => ?_ suffices a * ↑(normUnit a) = a * ↑u * ↑(normUnit a) * ↑u⁻¹ by simpa only [normalize_apply, mul_assoc, normUnit_mul ha u.ne_zero, normUnit_coe_units] calc a * ↑(normUnit a) = a * ↑(normUnit a) * ↑u * ↑u⁻¹ := (Units.mul_inv_cancel_right _ _).symm _ = a * ↑u * ↑(normUnit a) * ↑u⁻¹ := by rw [mul_right_comm a] theorem normalize_eq_normalize_iff {x y : α} : normalize x = normalize y ↔ x ∣ y ∧ y ∣ x := ⟨fun h => ⟨Units.dvd_mul_right.1 ⟨_, h.symm⟩, Units.dvd_mul_right.1 ⟨_, h⟩⟩, fun ⟨hxy, hyx⟩ => normalize_eq_normalize hxy hyx⟩ theorem dvd_antisymm_of_normalize_eq {a b : α} (ha : normalize a = a) (hb : normalize b = b) (hab : a ∣ b) (hba : b ∣ a) : a = b := ha ▸ hb ▸ normalize_eq_normalize hab hba theorem Associated.eq_of_normalized {a b : α} (h : Associated a b) (ha : normalize a = a) (hb : normalize b = b) : a = b := dvd_antisymm_of_normalize_eq ha hb h.dvd h.dvd' --can be proven by simp theorem dvd_normalize_iff {a b : α} : a ∣ normalize b ↔ a ∣ b := Units.dvd_mul_right --can be proven by simp theorem normalize_dvd_iff {a b : α} : normalize a ∣ b ↔ a ∣ b := Units.mul_right_dvd end NormalizationMonoid namespace Associates variable [CancelCommMonoidWithZero α] [NormalizationMonoid α] /-- Maps an element of `Associates` back to the normalized element of its associate class -/ protected def out : Associates α → α := (Quotient.lift (normalize : α → α)) fun a _ ⟨_, hu⟩ => hu ▸ normalize_eq_normalize ⟨_, rfl⟩ (Units.mul_right_dvd.2 <| dvd_refl a) @[simp] theorem out_mk (a : α) : (Associates.mk a).out = normalize a := rfl @[simp] theorem out_one : (1 : Associates α).out = 1 := normalize_one theorem out_mul (a b : Associates α) : (a * b).out = a.out * b.out := Quotient.inductionOn₂ a b fun _ _ => by simp only [Associates.quotient_mk_eq_mk, out_mk, mk_mul_mk, normalize.map_mul] theorem dvd_out_iff (a : α) (b : Associates α) : a ∣ b.out ↔ Associates.mk a ≤ b := Quotient.inductionOn b <| by simp [Associates.out_mk, Associates.quotient_mk_eq_mk, mk_le_mk_iff_dvd] theorem out_dvd_iff (a : α) (b : Associates α) : b.out ∣ a ↔ b ≤ Associates.mk a := Quotient.inductionOn b <| by simp [Associates.out_mk, Associates.quotient_mk_eq_mk, mk_le_mk_iff_dvd] @[simp] theorem out_top : (⊤ : Associates α).out = 0 := normalize_zero -- Porting note: lower priority to avoid linter complaints about simp-normal form @[simp 1100] theorem normalize_out (a : Associates α) : normalize a.out = a.out := Quotient.inductionOn a normalize_idem @[simp] theorem mk_out (a : Associates α) : Associates.mk a.out = a := Quotient.inductionOn a mk_normalize theorem out_injective : Function.Injective (Associates.out : _ → α) := Function.LeftInverse.injective mk_out end Associates -- Porting note: mathlib3 had a `@[protect_proj]` here, but adding `protected` to all the fields -- adds unnecessary clutter to later code /-- GCD monoid: a `CancelCommMonoidWithZero` with `gcd` (greatest common divisor) and `lcm` (least common multiple) operations, determined up to a unit. The type class focuses on `gcd` and we derive the corresponding `lcm` facts from `gcd`. -/ class GCDMonoid (α : Type*) [CancelCommMonoidWithZero α] where /-- The greatest common divisor between two elements. -/ gcd : α → α → α /-- The least common multiple between two elements. -/ lcm : α → α → α /-- The GCD is a divisor of the first element. -/ gcd_dvd_left : ∀ a b, gcd a b ∣ a /-- The GCD is a divisor of the second element. -/ gcd_dvd_right : ∀ a b, gcd a b ∣ b /-- Any common divisor of both elements is a divisor of the GCD. -/ dvd_gcd : ∀ {a b c}, a ∣ c → a ∣ b → a ∣ gcd c b /-- The product of two elements is `Associated` with the product of their GCD and LCM. -/ gcd_mul_lcm : ∀ a b, Associated (gcd a b * lcm a b) (a * b) /-- `0` is left-absorbing. -/ lcm_zero_left : ∀ a, lcm 0 a = 0 /-- `0` is right-absorbing. -/ lcm_zero_right : ∀ a, lcm a 0 = 0 /-- Normalized GCD monoid: a `CancelCommMonoidWithZero` with normalization and `gcd` (greatest common divisor) and `lcm` (least common multiple) operations. In this setting `gcd` and `lcm` form a bounded lattice on the associated elements where `gcd` is the infimum, `lcm` is the supremum, `1` is bottom, and `0` is top. The type class focuses on `gcd` and we derive the corresponding `lcm` facts from `gcd`. -/ class NormalizedGCDMonoid (α : Type*) [CancelCommMonoidWithZero α] extends NormalizationMonoid α, GCDMonoid α where /-- The GCD is normalized to itself. -/ normalize_gcd : ∀ a b, normalize (gcd a b) = gcd a b /-- The LCM is normalized to itself. -/ normalize_lcm : ∀ a b, normalize (lcm a b) = lcm a b export GCDMonoid (gcd lcm gcd_dvd_left gcd_dvd_right dvd_gcd lcm_zero_left lcm_zero_right) attribute [simp] lcm_zero_left lcm_zero_right section GCDMonoid variable [CancelCommMonoidWithZero α] instance [NormalizationMonoid α] : Nonempty (NormalizationMonoid α) := ⟨‹_›⟩ instance [GCDMonoid α] : Nonempty (GCDMonoid α) := ⟨‹_›⟩ instance [NormalizedGCDMonoid α] : Nonempty (NormalizedGCDMonoid α) := ⟨‹_›⟩ instance [h : Nonempty (NormalizedGCDMonoid α)] : Nonempty (NormalizationMonoid α) := h.elim fun _ ↦ inferInstance instance [h : Nonempty (NormalizedGCDMonoid α)] : Nonempty (GCDMonoid α) := h.elim fun _ ↦ inferInstance theorem gcd_isUnit_iff_isRelPrime [GCDMonoid α] {a b : α} : IsUnit (gcd a b) ↔ IsRelPrime a b := ⟨fun h _ ha hb ↦ isUnit_of_dvd_unit (dvd_gcd ha hb) h, (· (gcd_dvd_left a b) (gcd_dvd_right a b))⟩ -- Porting note: lower priority to avoid linter complaints about simp-normal form @[simp 1100] theorem normalize_gcd [NormalizedGCDMonoid α] : ∀ a b : α, normalize (gcd a b) = gcd a b := NormalizedGCDMonoid.normalize_gcd theorem gcd_mul_lcm [GCDMonoid α] : ∀ a b : α, Associated (gcd a b * lcm a b) (a * b) := GCDMonoid.gcd_mul_lcm section GCD theorem dvd_gcd_iff [GCDMonoid α] (a b c : α) : a ∣ gcd b c ↔ a ∣ b ∧ a ∣ c := Iff.intro (fun h => ⟨h.trans (gcd_dvd_left _ _), h.trans (gcd_dvd_right _ _)⟩) fun ⟨hab, hac⟩ => dvd_gcd hab hac theorem gcd_comm [NormalizedGCDMonoid α] (a b : α) : gcd a b = gcd b a := dvd_antisymm_of_normalize_eq (normalize_gcd _ _) (normalize_gcd _ _) (dvd_gcd (gcd_dvd_right _ _) (gcd_dvd_left _ _)) (dvd_gcd (gcd_dvd_right _ _) (gcd_dvd_left _ _)) theorem gcd_comm' [GCDMonoid α] (a b : α) : Associated (gcd a b) (gcd b a) := associated_of_dvd_dvd (dvd_gcd (gcd_dvd_right _ _) (gcd_dvd_left _ _)) (dvd_gcd (gcd_dvd_right _ _) (gcd_dvd_left _ _)) theorem gcd_assoc [NormalizedGCDMonoid α] (m n k : α) : gcd (gcd m n) k = gcd m (gcd n k) := dvd_antisymm_of_normalize_eq (normalize_gcd _ _) (normalize_gcd _ _) (dvd_gcd ((gcd_dvd_left (gcd m n) k).trans (gcd_dvd_left m n)) (dvd_gcd ((gcd_dvd_left (gcd m n) k).trans (gcd_dvd_right m n)) (gcd_dvd_right (gcd m n) k))) (dvd_gcd (dvd_gcd (gcd_dvd_left m (gcd n k)) ((gcd_dvd_right m (gcd n k)).trans (gcd_dvd_left n k))) ((gcd_dvd_right m (gcd n k)).trans (gcd_dvd_right n k))) theorem gcd_assoc' [GCDMonoid α] (m n k : α) : Associated (gcd (gcd m n) k) (gcd m (gcd n k)) := associated_of_dvd_dvd (dvd_gcd ((gcd_dvd_left (gcd m n) k).trans (gcd_dvd_left m n)) (dvd_gcd ((gcd_dvd_left (gcd m n) k).trans (gcd_dvd_right m n)) (gcd_dvd_right (gcd m n) k))) (dvd_gcd (dvd_gcd (gcd_dvd_left m (gcd n k)) ((gcd_dvd_right m (gcd n k)).trans (gcd_dvd_left n k))) ((gcd_dvd_right m (gcd n k)).trans (gcd_dvd_right n k))) instance [NormalizedGCDMonoid α] : Std.Commutative (α := α) gcd where comm := gcd_comm instance [NormalizedGCDMonoid α] : Std.Associative (α := α) gcd where assoc := gcd_assoc theorem gcd_eq_normalize [NormalizedGCDMonoid α] {a b c : α} (habc : gcd a b ∣ c) (hcab : c ∣ gcd a b) : gcd a b = normalize c := normalize_gcd a b ▸ normalize_eq_normalize habc hcab @[simp] theorem gcd_zero_left [NormalizedGCDMonoid α] (a : α) : gcd 0 a = normalize a := gcd_eq_normalize (gcd_dvd_right 0 a) (dvd_gcd (dvd_zero _) (dvd_refl a)) theorem gcd_zero_left' [GCDMonoid α] (a : α) : Associated (gcd 0 a) a := associated_of_dvd_dvd (gcd_dvd_right 0 a) (dvd_gcd (dvd_zero _) (dvd_refl a)) @[simp] theorem gcd_zero_right [NormalizedGCDMonoid α] (a : α) : gcd a 0 = normalize a := gcd_eq_normalize (gcd_dvd_left a 0) (dvd_gcd (dvd_refl a) (dvd_zero _)) theorem gcd_zero_right' [GCDMonoid α] (a : α) : Associated (gcd a 0) a := associated_of_dvd_dvd (gcd_dvd_left a 0) (dvd_gcd (dvd_refl a) (dvd_zero _)) @[simp] theorem gcd_eq_zero_iff [GCDMonoid α] (a b : α) : gcd a b = 0 ↔ a = 0 ∧ b = 0 := Iff.intro (fun h => by let ⟨ca, ha⟩ := gcd_dvd_left a b let ⟨cb, hb⟩ := gcd_dvd_right a b rw [h, zero_mul] at ha hb exact ⟨ha, hb⟩) fun ⟨ha, hb⟩ => by rw [ha, hb, ← zero_dvd_iff] apply dvd_gcd <;> rfl @[simp] theorem gcd_one_left [NormalizedGCDMonoid α] (a : α) : gcd 1 a = 1 := dvd_antisymm_of_normalize_eq (normalize_gcd _ _) normalize_one (gcd_dvd_left _ _) (one_dvd _) @[simp] theorem isUnit_gcd_one_left [GCDMonoid α] (a : α) : IsUnit (gcd 1 a) := isUnit_of_dvd_one (gcd_dvd_left _ _) theorem gcd_one_left' [GCDMonoid α] (a : α) : Associated (gcd 1 a) 1 := by simp @[simp] theorem gcd_one_right [NormalizedGCDMonoid α] (a : α) : gcd a 1 = 1 := dvd_antisymm_of_normalize_eq (normalize_gcd _ _) normalize_one (gcd_dvd_right _ _) (one_dvd _) @[simp] theorem isUnit_gcd_one_right [GCDMonoid α] (a : α) : IsUnit (gcd a 1) := isUnit_of_dvd_one (gcd_dvd_right _ _) theorem gcd_one_right' [GCDMonoid α] (a : α) : Associated (gcd a 1) 1 := by simp theorem gcd_dvd_gcd [GCDMonoid α] {a b c d : α} (hab : a ∣ b) (hcd : c ∣ d) : gcd a c ∣ gcd b d := dvd_gcd ((gcd_dvd_left _ _).trans hab) ((gcd_dvd_right _ _).trans hcd) protected theorem Associated.gcd [GCDMonoid α] {a₁ a₂ b₁ b₂ : α} (ha : Associated a₁ a₂) (hb : Associated b₁ b₂) : Associated (gcd a₁ b₁) (gcd a₂ b₂) := associated_of_dvd_dvd (gcd_dvd_gcd ha.dvd hb.dvd) (gcd_dvd_gcd ha.dvd' hb.dvd') @[simp] theorem gcd_same [NormalizedGCDMonoid α] (a : α) : gcd a a = normalize a := gcd_eq_normalize (gcd_dvd_left _ _) (dvd_gcd (dvd_refl a) (dvd_refl a)) @[simp] theorem gcd_mul_left [NormalizedGCDMonoid α] (a b c : α) : gcd (a * b) (a * c) = normalize a * gcd b c := (by_cases (by rintro rfl; simp only [zero_mul, gcd_zero_left, normalize_zero])) fun ha : a ≠ 0 => suffices gcd (a * b) (a * c) = normalize (a * gcd b c) by simpa let ⟨d, eq⟩ := dvd_gcd (dvd_mul_right a b) (dvd_mul_right a c) gcd_eq_normalize (eq.symm ▸ mul_dvd_mul_left a (show d ∣ gcd b c from dvd_gcd ((mul_dvd_mul_iff_left ha).1 <| eq ▸ gcd_dvd_left _ _) ((mul_dvd_mul_iff_left ha).1 <| eq ▸ gcd_dvd_right _ _))) (dvd_gcd (mul_dvd_mul_left a <| gcd_dvd_left _ _) (mul_dvd_mul_left a <| gcd_dvd_right _ _)) theorem gcd_mul_left' [GCDMonoid α] (a b c : α) : Associated (gcd (a * b) (a * c)) (a * gcd b c) := by obtain rfl | ha := eq_or_ne a 0 · simp only [zero_mul, gcd_zero_left'] obtain ⟨d, eq⟩ := dvd_gcd (dvd_mul_right a b) (dvd_mul_right a c) apply associated_of_dvd_dvd · rw [eq] apply mul_dvd_mul_left exact dvd_gcd ((mul_dvd_mul_iff_left ha).1 <| eq ▸ gcd_dvd_left _ _) ((mul_dvd_mul_iff_left ha).1 <| eq ▸ gcd_dvd_right _ _) · exact dvd_gcd (mul_dvd_mul_left a <| gcd_dvd_left _ _) (mul_dvd_mul_left a <| gcd_dvd_right _ _) @[simp] theorem gcd_mul_right [NormalizedGCDMonoid α] (a b c : α) : gcd (b * a) (c * a) = gcd b c * normalize a := by simp only [mul_comm, gcd_mul_left] @[simp] theorem gcd_mul_right' [GCDMonoid α] (a b c : α) : Associated (gcd (b * a) (c * a)) (gcd b c * a) := by simp only [mul_comm, gcd_mul_left'] theorem gcd_eq_left_iff [NormalizedGCDMonoid α] (a b : α) (h : normalize a = a) : gcd a b = a ↔ a ∣ b := (Iff.intro fun eq => eq ▸ gcd_dvd_right _ _) fun hab => dvd_antisymm_of_normalize_eq (normalize_gcd _ _) h (gcd_dvd_left _ _) (dvd_gcd (dvd_refl a) hab) theorem gcd_eq_right_iff [NormalizedGCDMonoid α] (a b : α) (h : normalize b = b) : gcd a b = b ↔ b ∣ a := by simpa only [gcd_comm a b] using gcd_eq_left_iff b a h theorem gcd_dvd_gcd_mul_left [GCDMonoid α] (m n k : α) : gcd m n ∣ gcd (k * m) n := gcd_dvd_gcd (dvd_mul_left _ _) dvd_rfl theorem gcd_dvd_gcd_mul_right [GCDMonoid α] (m n k : α) : gcd m n ∣ gcd (m * k) n := gcd_dvd_gcd (dvd_mul_right _ _) dvd_rfl theorem gcd_dvd_gcd_mul_left_right [GCDMonoid α] (m n k : α) : gcd m n ∣ gcd m (k * n) := gcd_dvd_gcd dvd_rfl (dvd_mul_left _ _) theorem gcd_dvd_gcd_mul_right_right [GCDMonoid α] (m n k : α) : gcd m n ∣ gcd m (n * k) := gcd_dvd_gcd dvd_rfl (dvd_mul_right _ _) theorem Associated.gcd_eq_left [NormalizedGCDMonoid α] {m n : α} (h : Associated m n) (k : α) : gcd m k = gcd n k := dvd_antisymm_of_normalize_eq (normalize_gcd _ _) (normalize_gcd _ _) (gcd_dvd_gcd h.dvd dvd_rfl) (gcd_dvd_gcd h.symm.dvd dvd_rfl) theorem Associated.gcd_eq_right [NormalizedGCDMonoid α] {m n : α} (h : Associated m n) (k : α) : gcd k m = gcd k n := dvd_antisymm_of_normalize_eq (normalize_gcd _ _) (normalize_gcd _ _) (gcd_dvd_gcd dvd_rfl h.dvd) (gcd_dvd_gcd dvd_rfl h.symm.dvd) theorem dvd_gcd_mul_of_dvd_mul [GCDMonoid α] {m n k : α} (H : k ∣ m * n) : k ∣ gcd k m * n := (dvd_gcd (dvd_mul_right _ n) H).trans (gcd_mul_right' n k m).dvd theorem dvd_gcd_mul_iff_dvd_mul [GCDMonoid α] {m n k : α} : k ∣ gcd k m * n ↔ k ∣ m * n := ⟨fun h => h.trans (mul_dvd_mul (gcd_dvd_right k m) dvd_rfl), dvd_gcd_mul_of_dvd_mul⟩ theorem dvd_mul_gcd_of_dvd_mul [GCDMonoid α] {m n k : α} (H : k ∣ m * n) : k ∣ m * gcd k n := by rw [mul_comm] at H ⊢ exact dvd_gcd_mul_of_dvd_mul H theorem dvd_mul_gcd_iff_dvd_mul [GCDMonoid α] {m n k : α} : k ∣ m * gcd k n ↔ k ∣ m * n := ⟨fun h => h.trans (mul_dvd_mul dvd_rfl (gcd_dvd_right k n)), dvd_mul_gcd_of_dvd_mul⟩ /-- Represent a divisor of `m * n` as a product of a divisor of `m` and a divisor of `n`. Note: In general, this representation is highly non-unique. See `Nat.prodDvdAndDvdOfDvdProd` for a constructive version on `ℕ`. -/ instance [h : Nonempty (GCDMonoid α)] : DecompositionMonoid α where primal k m n H := by cases h by_cases h0 : gcd k m = 0 · rw [gcd_eq_zero_iff] at h0 rcases h0 with ⟨rfl, rfl⟩ exact ⟨0, n, dvd_refl 0, dvd_refl n, by simp⟩ · obtain ⟨a, ha⟩ := gcd_dvd_left k m refine ⟨gcd k m, a, gcd_dvd_right _ _, ?_, ha⟩ rw [← mul_dvd_mul_iff_left h0, ← ha] exact dvd_gcd_mul_of_dvd_mul H theorem gcd_mul_dvd_mul_gcd [GCDMonoid α] (k m n : α) : gcd k (m * n) ∣ gcd k m * gcd k n := by obtain ⟨m', n', hm', hn', h⟩ := exists_dvd_and_dvd_of_dvd_mul (gcd_dvd_right k (m * n)) replace h : gcd k (m * n) = m' * n' := h rw [h] have hm'n' : m' * n' ∣ k := h ▸ gcd_dvd_left _ _ apply mul_dvd_mul · have hm'k : m' ∣ k := (dvd_mul_right m' n').trans hm'n' exact dvd_gcd hm'k hm' · have hn'k : n' ∣ k := (dvd_mul_left n' m').trans hm'n' exact dvd_gcd hn'k hn' theorem gcd_pow_right_dvd_pow_gcd [GCDMonoid α] {a b : α} {k : ℕ} : gcd a (b ^ k) ∣ gcd a b ^ k := by by_cases hg : gcd a b = 0 · rw [gcd_eq_zero_iff] at hg rcases hg with ⟨rfl, rfl⟩ exact (gcd_zero_left' (0 ^ k : α)).dvd.trans (pow_dvd_pow_of_dvd (gcd_zero_left' (0 : α)).symm.dvd _) · induction' k with k hk · rw [pow_zero, pow_zero] exact (gcd_one_right' a).dvd rw [pow_succ', pow_succ'] trans gcd a b * gcd a (b ^ k) · exact gcd_mul_dvd_mul_gcd a b (b ^ k) · exact (mul_dvd_mul_iff_left hg).mpr hk theorem gcd_pow_left_dvd_pow_gcd [GCDMonoid α] {a b : α} {k : ℕ} : gcd (a ^ k) b ∣ gcd a b ^ k := calc gcd (a ^ k) b ∣ gcd b (a ^ k) := (gcd_comm' _ _).dvd _ ∣ gcd b a ^ k := gcd_pow_right_dvd_pow_gcd _ ∣ gcd a b ^ k := pow_dvd_pow_of_dvd (gcd_comm' _ _).dvd _ theorem pow_dvd_of_mul_eq_pow [GCDMonoid α] {a b c d₁ d₂ : α} (ha : a ≠ 0) (hab : IsUnit (gcd a b)) {k : ℕ} (h : a * b = c ^ k) (hc : c = d₁ * d₂) (hd₁ : d₁ ∣ a) : d₁ ^ k ≠ 0 ∧ d₁ ^ k ∣ a := by have h1 : IsUnit (gcd (d₁ ^ k) b) := by apply isUnit_of_dvd_one trans gcd d₁ b ^ k · exact gcd_pow_left_dvd_pow_gcd · apply IsUnit.dvd apply IsUnit.pow apply isUnit_of_dvd_one apply dvd_trans _ hab.dvd apply gcd_dvd_gcd hd₁ (dvd_refl b) have h2 : d₁ ^ k ∣ a * b := by use d₂ ^ k rw [h, hc] exact mul_pow d₁ d₂ k rw [mul_comm] at h2 have h3 : d₁ ^ k ∣ a := by apply (dvd_gcd_mul_of_dvd_mul h2).trans rw [h1.mul_left_dvd] have h4 : d₁ ^ k ≠ 0 := by intro hdk rw [hdk] at h3 apply absurd (zero_dvd_iff.mp h3) ha exact ⟨h4, h3⟩ theorem exists_associated_pow_of_mul_eq_pow [GCDMonoid α] {a b c : α} (hab : IsUnit (gcd a b)) {k : ℕ} (h : a * b = c ^ k) : ∃ d : α, Associated (d ^ k) a := by cases subsingleton_or_nontrivial α · use 0 rw [Subsingleton.elim a (0 ^ k)] by_cases ha : a = 0 · use 0 obtain rfl | hk := eq_or_ne k 0 · simp [ha] at h · rw [ha, zero_pow hk] by_cases hb : b = 0 · use 1 rw [one_pow] apply (associated_one_iff_isUnit.mpr hab).symm.trans rw [hb] exact gcd_zero_right' a obtain rfl | hk := k.eq_zero_or_pos · use 1 rw [pow_zero] at h ⊢ use Units.mkOfMulEqOne _ _ h rw [Units.val_mkOfMulEqOne, one_mul] have hc : c ∣ a * b := by rw [h] exact dvd_pow_self _ hk.ne' obtain ⟨d₁, d₂, hd₁, hd₂, hc⟩ := exists_dvd_and_dvd_of_dvd_mul hc use d₁ obtain ⟨h0₁, ⟨a', ha'⟩⟩ := pow_dvd_of_mul_eq_pow ha hab h hc hd₁ rw [mul_comm] at h hc rw [(gcd_comm' a b).isUnit_iff] at hab obtain ⟨h0₂, ⟨b', hb'⟩⟩ := pow_dvd_of_mul_eq_pow hb hab h hc hd₂ rw [ha', hb', hc, mul_pow] at h have h' : a' * b' = 1 := by apply (mul_right_inj' h0₁).mp rw [mul_one] apply (mul_right_inj' h0₂).mp rw [← h] rw [mul_assoc, mul_comm a', ← mul_assoc _ b', ← mul_assoc b', mul_comm b'] use Units.mkOfMulEqOne _ _ h' rw [Units.val_mkOfMulEqOne, ha'] theorem exists_eq_pow_of_mul_eq_pow [GCDMonoid α] [Unique αˣ] {a b c : α} (hab : IsUnit (gcd a b)) {k : ℕ} (h : a * b = c ^ k) : ∃ d : α, a = d ^ k := let ⟨d, hd⟩ := exists_associated_pow_of_mul_eq_pow hab h ⟨d, (associated_iff_eq.mp hd).symm⟩ theorem gcd_greatest {α : Type*} [CancelCommMonoidWithZero α] [NormalizedGCDMonoid α] {a b d : α} (hda : d ∣ a) (hdb : d ∣ b) (hd : ∀ e : α, e ∣ a → e ∣ b → e ∣ d) : GCDMonoid.gcd a b = normalize d := haveI h := hd _ (GCDMonoid.gcd_dvd_left a b) (GCDMonoid.gcd_dvd_right a b) gcd_eq_normalize h (GCDMonoid.dvd_gcd hda hdb) theorem gcd_greatest_associated {α : Type*} [CancelCommMonoidWithZero α] [GCDMonoid α] {a b d : α} (hda : d ∣ a) (hdb : d ∣ b) (hd : ∀ e : α, e ∣ a → e ∣ b → e ∣ d) : Associated d (GCDMonoid.gcd a b) := haveI h := hd _ (GCDMonoid.gcd_dvd_left a b) (GCDMonoid.gcd_dvd_right a b) associated_of_dvd_dvd (GCDMonoid.dvd_gcd hda hdb) h theorem isUnit_gcd_of_eq_mul_gcd {α : Type*} [CancelCommMonoidWithZero α] [GCDMonoid α] {x y x' y' : α} (ex : x = gcd x y * x') (ey : y = gcd x y * y') (h : gcd x y ≠ 0) : IsUnit (gcd x' y') := by rw [← associated_one_iff_isUnit] refine Associated.of_mul_left ?_ (Associated.refl <| gcd x y) h convert (gcd_mul_left' (gcd x y) x' y').symm using 1 rw [← ex, ← ey, mul_one] theorem extract_gcd {α : Type*} [CancelCommMonoidWithZero α] [GCDMonoid α] (x y : α) : ∃ x' y', x = gcd x y * x' ∧ y = gcd x y * y' ∧ IsUnit (gcd x' y') := by by_cases h : gcd x y = 0 · obtain ⟨rfl, rfl⟩ := (gcd_eq_zero_iff x y).1 h simp_rw [← associated_one_iff_isUnit] exact ⟨1, 1, by rw [h, zero_mul], by rw [h, zero_mul], gcd_one_left' 1⟩ obtain ⟨x', ex⟩ := gcd_dvd_left x y obtain ⟨y', ey⟩ := gcd_dvd_right x y exact ⟨x', y', ex, ey, isUnit_gcd_of_eq_mul_gcd ex ey h⟩ theorem associated_gcd_left_iff [GCDMonoid α] {x y : α} : Associated x (gcd x y) ↔ x ∣ y := ⟨fun hx => hx.dvd.trans (gcd_dvd_right x y), fun hxy => associated_of_dvd_dvd (dvd_gcd dvd_rfl hxy) (gcd_dvd_left x y)⟩ theorem associated_gcd_right_iff [GCDMonoid α] {x y : α} : Associated y (gcd x y) ↔ y ∣ x := ⟨fun hx => hx.dvd.trans (gcd_dvd_left x y), fun hxy => associated_of_dvd_dvd (dvd_gcd hxy dvd_rfl) (gcd_dvd_right x y)⟩ theorem Irreducible.isUnit_gcd_iff [GCDMonoid α] {x y : α} (hx : Irreducible x) : IsUnit (gcd x y) ↔ ¬(x ∣ y) := by rw [hx.isUnit_iff_not_associated_of_dvd (gcd_dvd_left x y), not_iff_not, associated_gcd_left_iff] theorem Irreducible.gcd_eq_one_iff [NormalizedGCDMonoid α] {x y : α} (hx : Irreducible x) : gcd x y = 1 ↔ ¬(x ∣ y) := by rw [← hx.isUnit_gcd_iff, ← normalize_eq_one, NormalizedGCDMonoid.normalize_gcd] section Neg variable [HasDistribNeg α] lemma gcd_neg' [GCDMonoid α] {a b : α} : Associated (gcd a (-b)) (gcd a b) := Associated.gcd .rfl (.neg_left .rfl) lemma gcd_neg [NormalizedGCDMonoid α] {a b : α} : gcd a (-b) = gcd a b := gcd_neg'.eq_of_normalized (normalize_gcd _ _) (normalize_gcd _ _) lemma neg_gcd' [GCDMonoid α] {a b : α} : Associated (gcd (-a) b) (gcd a b) := Associated.gcd (.neg_left .rfl) .rfl lemma neg_gcd [NormalizedGCDMonoid α] {a b : α} : gcd (-a) b = gcd a b := neg_gcd'.eq_of_normalized (normalize_gcd _ _) (normalize_gcd _ _) end Neg end GCD section LCM theorem lcm_dvd_iff [GCDMonoid α] {a b c : α} : lcm a b ∣ c ↔ a ∣ c ∧ b ∣ c := by by_cases h : a = 0 ∨ b = 0 · rcases h with (rfl | rfl) <;> simp (config := { contextual := true }) only [iff_def, lcm_zero_left, lcm_zero_right, zero_dvd_iff, dvd_zero, eq_self_iff_true, and_true_iff, imp_true_iff] · obtain ⟨h1, h2⟩ := not_or.1 h have h : gcd a b ≠ 0 := fun H => h1 ((gcd_eq_zero_iff _ _).1 H).1 rw [← mul_dvd_mul_iff_left h, (gcd_mul_lcm a b).dvd_iff_dvd_left, ← (gcd_mul_right' c a b).dvd_iff_dvd_right, dvd_gcd_iff, mul_comm b c, mul_dvd_mul_iff_left h1, mul_dvd_mul_iff_right h2, and_comm] theorem dvd_lcm_left [GCDMonoid α] (a b : α) : a ∣ lcm a b := (lcm_dvd_iff.1 (dvd_refl (lcm a b))).1 theorem dvd_lcm_right [GCDMonoid α] (a b : α) : b ∣ lcm a b := (lcm_dvd_iff.1 (dvd_refl (lcm a b))).2 theorem lcm_dvd [GCDMonoid α] {a b c : α} (hab : a ∣ b) (hcb : c ∣ b) : lcm a c ∣ b := lcm_dvd_iff.2 ⟨hab, hcb⟩ @[simp] theorem lcm_eq_zero_iff [GCDMonoid α] (a b : α) : lcm a b = 0 ↔ a = 0 ∨ b = 0 := Iff.intro (fun h : lcm a b = 0 => by have : Associated (a * b) 0 := (gcd_mul_lcm a b).symm.trans <| by rw [h, mul_zero] rwa [← mul_eq_zero, ← associated_zero_iff_eq_zero]) (by rintro (rfl | rfl) <;> [apply lcm_zero_left; apply lcm_zero_right]) -- Porting note: lower priority to avoid linter complaints about simp-normal form @[simp 1100] theorem normalize_lcm [NormalizedGCDMonoid α] (a b : α) : normalize (lcm a b) = lcm a b := NormalizedGCDMonoid.normalize_lcm a b theorem lcm_comm [NormalizedGCDMonoid α] (a b : α) : lcm a b = lcm b a := dvd_antisymm_of_normalize_eq (normalize_lcm _ _) (normalize_lcm _ _) (lcm_dvd (dvd_lcm_right _ _) (dvd_lcm_left _ _)) (lcm_dvd (dvd_lcm_right _ _) (dvd_lcm_left _ _)) theorem lcm_comm' [GCDMonoid α] (a b : α) : Associated (lcm a b) (lcm b a) := associated_of_dvd_dvd (lcm_dvd (dvd_lcm_right _ _) (dvd_lcm_left _ _)) (lcm_dvd (dvd_lcm_right _ _) (dvd_lcm_left _ _)) theorem lcm_assoc [NormalizedGCDMonoid α] (m n k : α) : lcm (lcm m n) k = lcm m (lcm n k) := dvd_antisymm_of_normalize_eq (normalize_lcm _ _) (normalize_lcm _ _) (lcm_dvd (lcm_dvd (dvd_lcm_left _ _) ((dvd_lcm_left _ _).trans (dvd_lcm_right _ _))) ((dvd_lcm_right _ _).trans (dvd_lcm_right _ _))) (lcm_dvd ((dvd_lcm_left _ _).trans (dvd_lcm_left _ _)) (lcm_dvd ((dvd_lcm_right _ _).trans (dvd_lcm_left _ _)) (dvd_lcm_right _ _))) theorem lcm_assoc' [GCDMonoid α] (m n k : α) : Associated (lcm (lcm m n) k) (lcm m (lcm n k)) := associated_of_dvd_dvd (lcm_dvd (lcm_dvd (dvd_lcm_left _ _) ((dvd_lcm_left _ _).trans (dvd_lcm_right _ _))) ((dvd_lcm_right _ _).trans (dvd_lcm_right _ _))) (lcm_dvd ((dvd_lcm_left _ _).trans (dvd_lcm_left _ _)) (lcm_dvd ((dvd_lcm_right _ _).trans (dvd_lcm_left _ _)) (dvd_lcm_right _ _))) instance [NormalizedGCDMonoid α] : Std.Commutative (α := α) lcm where comm := lcm_comm instance [NormalizedGCDMonoid α] : Std.Associative (α := α) lcm where assoc := lcm_assoc theorem lcm_eq_normalize [NormalizedGCDMonoid α] {a b c : α} (habc : lcm a b ∣ c) (hcab : c ∣ lcm a b) : lcm a b = normalize c := normalize_lcm a b ▸ normalize_eq_normalize habc hcab theorem lcm_dvd_lcm [GCDMonoid α] {a b c d : α} (hab : a ∣ b) (hcd : c ∣ d) : lcm a c ∣ lcm b d := lcm_dvd (hab.trans (dvd_lcm_left _ _)) (hcd.trans (dvd_lcm_right _ _)) protected theorem Associated.lcm [GCDMonoid α] {a₁ a₂ b₁ b₂ : α} (ha : Associated a₁ a₂) (hb : Associated b₁ b₂) : Associated (lcm a₁ b₁) (lcm a₂ b₂) := associated_of_dvd_dvd (lcm_dvd_lcm ha.dvd hb.dvd) (lcm_dvd_lcm ha.dvd' hb.dvd') @[simp] theorem lcm_units_coe_left [NormalizedGCDMonoid α] (u : αˣ) (a : α) : lcm (↑u) a = normalize a := lcm_eq_normalize (lcm_dvd Units.coe_dvd dvd_rfl) (dvd_lcm_right _ _) @[simp] theorem lcm_units_coe_right [NormalizedGCDMonoid α] (a : α) (u : αˣ) : lcm a ↑u = normalize a := (lcm_comm a u).trans <| lcm_units_coe_left _ _ @[simp] theorem lcm_one_left [NormalizedGCDMonoid α] (a : α) : lcm 1 a = normalize a := lcm_units_coe_left 1 a @[simp] theorem lcm_one_right [NormalizedGCDMonoid α] (a : α) : lcm a 1 = normalize a := lcm_units_coe_right a 1 @[simp] theorem lcm_same [NormalizedGCDMonoid α] (a : α) : lcm a a = normalize a := lcm_eq_normalize (lcm_dvd dvd_rfl dvd_rfl) (dvd_lcm_left _ _) @[simp] theorem lcm_eq_one_iff [NormalizedGCDMonoid α] (a b : α) : lcm a b = 1 ↔ a ∣ 1 ∧ b ∣ 1 := Iff.intro (fun eq => eq ▸ ⟨dvd_lcm_left _ _, dvd_lcm_right _ _⟩) fun ⟨⟨c, hc⟩, ⟨d, hd⟩⟩ => show lcm (Units.mkOfMulEqOne a c hc.symm : α) (Units.mkOfMulEqOne b d hd.symm) = 1 by rw [lcm_units_coe_left, normalize_coe_units] @[simp] theorem lcm_mul_left [NormalizedGCDMonoid α] (a b c : α) : lcm (a * b) (a * c) = normalize a * lcm b c := (by_cases (by rintro rfl; simp only [zero_mul, lcm_zero_left, normalize_zero])) fun ha : a ≠ 0 => suffices lcm (a * b) (a * c) = normalize (a * lcm b c) by simpa have : a ∣ lcm (a * b) (a * c) := (dvd_mul_right _ _).trans (dvd_lcm_left _ _) let ⟨d, eq⟩ := this lcm_eq_normalize (lcm_dvd (mul_dvd_mul_left a (dvd_lcm_left _ _)) (mul_dvd_mul_left a (dvd_lcm_right _ _))) (eq.symm ▸ (mul_dvd_mul_left a <| lcm_dvd ((mul_dvd_mul_iff_left ha).1 <| eq ▸ dvd_lcm_left _ _) ((mul_dvd_mul_iff_left ha).1 <| eq ▸ dvd_lcm_right _ _))) @[simp] theorem lcm_mul_right [NormalizedGCDMonoid α] (a b c : α) : lcm (b * a) (c * a) = lcm b c * normalize a := by simp only [mul_comm, lcm_mul_left] theorem lcm_eq_left_iff [NormalizedGCDMonoid α] (a b : α) (h : normalize a = a) : lcm a b = a ↔ b ∣ a := (Iff.intro fun eq => eq ▸ dvd_lcm_right _ _) fun hab => dvd_antisymm_of_normalize_eq (normalize_lcm _ _) h (lcm_dvd (dvd_refl a) hab) (dvd_lcm_left _ _) theorem lcm_eq_right_iff [NormalizedGCDMonoid α] (a b : α) (h : normalize b = b) : lcm a b = b ↔ a ∣ b := by simpa only [lcm_comm b a] using lcm_eq_left_iff b a h theorem lcm_dvd_lcm_mul_left [GCDMonoid α] (m n k : α) : lcm m n ∣ lcm (k * m) n := lcm_dvd_lcm (dvd_mul_left _ _) dvd_rfl theorem lcm_dvd_lcm_mul_right [GCDMonoid α] (m n k : α) : lcm m n ∣ lcm (m * k) n := lcm_dvd_lcm (dvd_mul_right _ _) dvd_rfl theorem lcm_dvd_lcm_mul_left_right [GCDMonoid α] (m n k : α) : lcm m n ∣ lcm m (k * n) := lcm_dvd_lcm dvd_rfl (dvd_mul_left _ _) theorem lcm_dvd_lcm_mul_right_right [GCDMonoid α] (m n k : α) : lcm m n ∣ lcm m (n * k) := lcm_dvd_lcm dvd_rfl (dvd_mul_right _ _) theorem lcm_eq_of_associated_left [NormalizedGCDMonoid α] {m n : α} (h : Associated m n) (k : α) : lcm m k = lcm n k := dvd_antisymm_of_normalize_eq (normalize_lcm _ _) (normalize_lcm _ _) (lcm_dvd_lcm h.dvd dvd_rfl) (lcm_dvd_lcm h.symm.dvd dvd_rfl) theorem lcm_eq_of_associated_right [NormalizedGCDMonoid α] {m n : α} (h : Associated m n) (k : α) : lcm k m = lcm k n := dvd_antisymm_of_normalize_eq (normalize_lcm _ _) (normalize_lcm _ _) (lcm_dvd_lcm dvd_rfl h.dvd) (lcm_dvd_lcm dvd_rfl h.symm.dvd) end LCM @[deprecated (since := "2024-02-12")] alias GCDMonoid.prime_of_irreducible := Irreducible.prime @[deprecated (since := "2024-02-12")] alias GCDMonoid.irreducible_iff_prime := irreducible_iff_prime end GCDMonoid section UniqueUnit variable [CancelCommMonoidWithZero α] [Unique αˣ] -- see Note [lower instance priority] instance (priority := 100) normalizationMonoidOfUniqueUnits : NormalizationMonoid α where normUnit _ := 1 normUnit_zero := rfl normUnit_mul _ _ := (mul_one 1).symm normUnit_coe_units _ := Subsingleton.elim _ _ instance uniqueNormalizationMonoidOfUniqueUnits : Unique (NormalizationMonoid α) where default := normalizationMonoidOfUniqueUnits uniq := fun ⟨u, _, _, _⟩ => by congr; simp [eq_iff_true_of_subsingleton] instance subsingleton_gcdMonoid_of_unique_units : Subsingleton (GCDMonoid α) := ⟨fun g₁ g₂ => by have hgcd : g₁.gcd = g₂.gcd := by ext a b refine associated_iff_eq.mp (associated_of_dvd_dvd ?_ ?_) -- Porting note: Lean4 seems to need help specifying `g₁` and `g₂` · exact dvd_gcd (@gcd_dvd_left _ _ g₁ _ _) (@gcd_dvd_right _ _ g₁ _ _) · exact @dvd_gcd _ _ g₁ _ _ _ (@gcd_dvd_left _ _ g₂ _ _) (@gcd_dvd_right _ _ g₂ _ _) have hlcm : g₁.lcm = g₂.lcm := by ext a b -- Porting note: Lean4 seems to need help specifying `g₁` and `g₂` refine associated_iff_eq.mp (associated_of_dvd_dvd ?_ ?_) · exact (@lcm_dvd_iff _ _ g₁ ..).mpr ⟨@dvd_lcm_left _ _ g₂ _ _, @dvd_lcm_right _ _ g₂ _ _⟩ · exact lcm_dvd_iff.mpr ⟨@dvd_lcm_left _ _ g₁ _ _, @dvd_lcm_right _ _ g₁ _ _⟩ cases g₁ cases g₂ dsimp only at hgcd hlcm simp only [hgcd, hlcm]⟩ instance subsingleton_normalizedGCDMonoid_of_unique_units : Subsingleton (NormalizedGCDMonoid α) := ⟨by intro a b cases' a with a_norm a_gcd cases' b with b_norm b_gcd have := Subsingleton.elim a_gcd b_gcd subst this have := Subsingleton.elim a_norm b_norm subst this rfl⟩ @[simp] theorem normUnit_eq_one (x : α) : normUnit x = 1 := rfl -- Porting note (#10618): `simp` can prove this -- @[simp] theorem normalize_eq (x : α) : normalize x = x := mul_one x /-- If a monoid's only unit is `1`, then it is isomorphic to its associates. -/ @[simps] def associatesEquivOfUniqueUnits : Associates α ≃* α where toFun := Associates.out invFun := Associates.mk left_inv := Associates.mk_out right_inv _ := (Associates.out_mk _).trans <| normalize_eq _ map_mul' := Associates.out_mul end UniqueUnit section IsDomain variable [CommRing α] [IsDomain α] [NormalizedGCDMonoid α] theorem gcd_eq_of_dvd_sub_right {a b c : α} (h : a ∣ b - c) : gcd a b = gcd a c := by apply dvd_antisymm_of_normalize_eq (normalize_gcd _ _) (normalize_gcd _ _) <;> rw [dvd_gcd_iff] <;> refine ⟨gcd_dvd_left _ _, ?_⟩ · rcases h with ⟨d, hd⟩ rcases gcd_dvd_right a b with ⟨e, he⟩ rcases gcd_dvd_left a b with ⟨f, hf⟩ use e - f * d rw [mul_sub, ← he, ← mul_assoc, ← hf, ← hd, sub_sub_cancel] · rcases h with ⟨d, hd⟩ rcases gcd_dvd_right a c with ⟨e, he⟩ rcases gcd_dvd_left a c with ⟨f, hf⟩ use e + f * d rw [mul_add, ← he, ← mul_assoc, ← hf, ← hd, ← add_sub_assoc, add_comm c b, add_sub_cancel_right] theorem gcd_eq_of_dvd_sub_left {a b c : α} (h : a ∣ b - c) : gcd b a = gcd c a := by rw [gcd_comm _ a, gcd_comm _ a, gcd_eq_of_dvd_sub_right h] end IsDomain noncomputable section Constructors open Associates variable [CancelCommMonoidWithZero α] private theorem map_mk_unit_aux [DecidableEq α] {f : Associates α →* α} (hinv : Function.RightInverse f Associates.mk) (a : α) : a * ↑(Classical.choose (associated_map_mk hinv a)) = f (Associates.mk a) := Classical.choose_spec (associated_map_mk hinv a) /-- Define `NormalizationMonoid` on a structure from a `MonoidHom` inverse to `Associates.mk`. -/ def normalizationMonoidOfMonoidHomRightInverse [DecidableEq α] (f : Associates α →* α) (hinv : Function.RightInverse f Associates.mk) : NormalizationMonoid α where normUnit a := if a = 0 then 1 else Classical.choose (Associates.mk_eq_mk_iff_associated.1 (hinv (Associates.mk a)).symm) normUnit_zero := if_pos rfl normUnit_mul {a b} ha hb := by simp_rw [if_neg (mul_ne_zero ha hb), if_neg ha, if_neg hb, Units.ext_iff, Units.val_mul] suffices a * b * ↑(Classical.choose (associated_map_mk hinv (a * b))) = a * ↑(Classical.choose (associated_map_mk hinv a)) * (b * ↑(Classical.choose (associated_map_mk hinv b))) by apply mul_left_cancel₀ (mul_ne_zero ha hb) _ -- Porting note: original `simpa` fails with `unexpected bound variable #1` -- simpa only [mul_assoc, mul_comm, mul_left_comm] using this rw [this, mul_assoc, ← mul_assoc _ b, mul_comm _ b, ← mul_assoc, ← mul_assoc, mul_assoc (a * b)] rw [map_mk_unit_aux hinv a, map_mk_unit_aux hinv (a * b), map_mk_unit_aux hinv b, ← MonoidHom.map_mul, Associates.mk_mul_mk] normUnit_coe_units u := by nontriviality α simp_rw [if_neg (Units.ne_zero u), Units.ext_iff] apply mul_left_cancel₀ (Units.ne_zero u) rw [Units.mul_inv, map_mk_unit_aux hinv u, Associates.mk_eq_mk_iff_associated.2 (associated_one_iff_isUnit.2 ⟨u, rfl⟩), Associates.mk_one, MonoidHom.map_one] /-- Define `GCDMonoid` on a structure just from the `gcd` and its properties. -/ noncomputable def gcdMonoidOfGCD [DecidableEq α] (gcd : α → α → α) (gcd_dvd_left : ∀ a b, gcd a b ∣ a) (gcd_dvd_right : ∀ a b, gcd a b ∣ b) (dvd_gcd : ∀ {a b c}, a ∣ c → a ∣ b → a ∣ gcd c b) : GCDMonoid α := { gcd gcd_dvd_left gcd_dvd_right dvd_gcd := fun {a b c} => dvd_gcd lcm := fun a b => if a = 0 then 0 else Classical.choose ((gcd_dvd_left a b).trans (Dvd.intro b rfl)) gcd_mul_lcm := fun a b => by -- Porting note(#12129): additional beta reduction needed beta_reduce split_ifs with a0 · rw [mul_zero, a0, zero_mul] · rw [← Classical.choose_spec ((gcd_dvd_left a b).trans (Dvd.intro b rfl))] lcm_zero_left := fun a => if_pos rfl lcm_zero_right := fun a => by -- Porting note(#12129): additional beta reduction needed beta_reduce split_ifs with a0 · rfl have h := (Classical.choose_spec ((gcd_dvd_left a 0).trans (Dvd.intro 0 rfl))).symm have a0' : gcd a 0 ≠ 0 := by contrapose! a0 rw [← associated_zero_iff_eq_zero, ← a0] exact associated_of_dvd_dvd (dvd_gcd (dvd_refl a) (dvd_zero a)) (gcd_dvd_left _ _) apply Or.resolve_left (mul_eq_zero.1 _) a0' rw [h, mul_zero] } /-- Define `NormalizedGCDMonoid` on a structure just from the `gcd` and its properties. -/ noncomputable def normalizedGCDMonoidOfGCD [NormalizationMonoid α] [DecidableEq α] (gcd : α → α → α) (gcd_dvd_left : ∀ a b, gcd a b ∣ a) (gcd_dvd_right : ∀ a b, gcd a b ∣ b) (dvd_gcd : ∀ {a b c}, a ∣ c → a ∣ b → a ∣ gcd c b) (normalize_gcd : ∀ a b, normalize (gcd a b) = gcd a b) : NormalizedGCDMonoid α := { (inferInstance : NormalizationMonoid α) with gcd gcd_dvd_left gcd_dvd_right dvd_gcd := fun {a b c} => dvd_gcd normalize_gcd lcm := fun a b => if a = 0 then 0 else Classical.choose (dvd_normalize_iff.2 ((gcd_dvd_left a b).trans (Dvd.intro b rfl))) normalize_lcm := fun a b => by dsimp [normalize] split_ifs with a0 · exact @normalize_zero α _ _ · have := (Classical.choose_spec (dvd_normalize_iff.2 ((gcd_dvd_left a b).trans (Dvd.intro b rfl)))).symm set l := Classical.choose (dvd_normalize_iff.2 ((gcd_dvd_left a b).trans (Dvd.intro b rfl))) obtain rfl | hb := eq_or_ne b 0 -- Porting note: using `simp only` causes the propositions inside `Classical.choose` to -- differ, so `set` is unable to produce `l = 0` inside `this`. See -- https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/ -- Classical.2Echoose/near/317491179 · rw [mul_zero a, normalize_zero, mul_eq_zero] at this obtain ha | hl := this · apply (a0 _).elim rw [← zero_dvd_iff, ← ha] exact gcd_dvd_left _ _ · rw [hl, zero_mul] have h1 : gcd a b ≠ 0 := by have hab : a * b ≠ 0 := mul_ne_zero a0 hb contrapose! hab rw [← normalize_eq_zero, ← this, hab, zero_mul] have h2 : normalize (gcd a b * l) = gcd a b * l := by rw [this, normalize_idem] rw [← normalize_gcd] at this rwa [normalize.map_mul, normalize_gcd, mul_right_inj' h1] at h2 gcd_mul_lcm := fun a b => by -- Porting note(#12129): additional beta reduction needed beta_reduce split_ifs with a0 · rw [mul_zero, a0, zero_mul] · rw [← Classical.choose_spec (dvd_normalize_iff.2 ((gcd_dvd_left a b).trans (Dvd.intro b rfl)))] exact normalize_associated (a * b) lcm_zero_left := fun a => if_pos rfl lcm_zero_right := fun a => by -- Porting note(#12129): additional beta reduction needed beta_reduce split_ifs with a0 · rfl rw [← normalize_eq_zero] at a0 have h := (Classical.choose_spec (dvd_normalize_iff.2 ((gcd_dvd_left a 0).trans (Dvd.intro 0 rfl)))).symm have gcd0 : gcd a 0 = normalize a := by rw [← normalize_gcd] exact normalize_eq_normalize (gcd_dvd_left _ _) (dvd_gcd (dvd_refl a) (dvd_zero a)) rw [← gcd0] at a0 apply Or.resolve_left (mul_eq_zero.1 _) a0 rw [h, mul_zero, normalize_zero] } /-- Define `GCDMonoid` on a structure just from the `lcm` and its properties. -/ noncomputable def gcdMonoidOfLCM [DecidableEq α] (lcm : α → α → α) (dvd_lcm_left : ∀ a b, a ∣ lcm a b) (dvd_lcm_right : ∀ a b, b ∣ lcm a b) (lcm_dvd : ∀ {a b c}, c ∣ a → b ∣ a → lcm c b ∣ a) : GCDMonoid α := let exists_gcd a b := lcm_dvd (Dvd.intro b rfl) (Dvd.intro_left a rfl) { lcm gcd := fun a b => if a = 0 then b else if b = 0 then a else Classical.choose (exists_gcd a b) gcd_mul_lcm := fun a b => by -- Porting note(#12129): additional beta reduction needed beta_reduce split_ifs with h h_1 · rw [h, eq_zero_of_zero_dvd (dvd_lcm_left _ _), mul_zero, zero_mul] · rw [h_1, eq_zero_of_zero_dvd (dvd_lcm_right _ _)] rw [mul_comm, ← Classical.choose_spec (exists_gcd a b)] lcm_zero_left := fun a => eq_zero_of_zero_dvd (dvd_lcm_left _ _) lcm_zero_right := fun a => eq_zero_of_zero_dvd (dvd_lcm_right _ _) gcd_dvd_left := fun a b => by -- Porting note(#12129): additional beta reduction needed beta_reduce split_ifs with h h_1 · rw [h] apply dvd_zero · exact dvd_rfl have h0 : lcm a b ≠ 0 := by intro con have h := lcm_dvd (Dvd.intro b rfl) (Dvd.intro_left a rfl) rw [con, zero_dvd_iff, mul_eq_zero] at h cases h · exact absurd ‹a = 0› h · exact absurd ‹b = 0› h_1 rw [← mul_dvd_mul_iff_left h0, ← Classical.choose_spec (exists_gcd a b), mul_comm, mul_dvd_mul_iff_right h] apply dvd_lcm_right gcd_dvd_right := fun a b => by -- Porting note(#12129): additional beta reduction needed beta_reduce split_ifs with h h_1 · exact dvd_rfl · rw [h_1] apply dvd_zero have h0 : lcm a b ≠ 0 := by intro con have h := lcm_dvd (Dvd.intro b rfl) (Dvd.intro_left a rfl) rw [con, zero_dvd_iff, mul_eq_zero] at h cases h · exact absurd ‹a = 0› h · exact absurd ‹b = 0› h_1 rw [← mul_dvd_mul_iff_left h0, ← Classical.choose_spec (exists_gcd a b), mul_dvd_mul_iff_right h_1] apply dvd_lcm_left dvd_gcd := fun {a b c} ac ab => by -- Porting note(#12129): additional beta reduction needed beta_reduce split_ifs with h h_1 · exact ab · exact ac have h0 : lcm c b ≠ 0 := by intro con have h := lcm_dvd (Dvd.intro b rfl) (Dvd.intro_left c rfl) rw [con, zero_dvd_iff, mul_eq_zero] at h cases h · exact absurd ‹c = 0› h · exact absurd ‹b = 0› h_1 rw [← mul_dvd_mul_iff_left h0, ← Classical.choose_spec (exists_gcd c b)] rcases ab with ⟨d, rfl⟩ rw [mul_eq_zero] at ‹a * d ≠ 0› push_neg at h_1 rw [mul_comm a, ← mul_assoc, mul_dvd_mul_iff_right h_1.1] apply lcm_dvd (Dvd.intro d rfl) rw [mul_comm, mul_dvd_mul_iff_right h_1.2] apply ac } -- Porting note (#11083): very slow; improve performance? /-- Define `NormalizedGCDMonoid` on a structure just from the `lcm` and its properties. -/ noncomputable def normalizedGCDMonoidOfLCM [NormalizationMonoid α] [DecidableEq α] (lcm : α → α → α) (dvd_lcm_left : ∀ a b, a ∣ lcm a b) (dvd_lcm_right : ∀ a b, b ∣ lcm a b) (lcm_dvd : ∀ {a b c}, c ∣ a → b ∣ a → lcm c b ∣ a) (normalize_lcm : ∀ a b, normalize (lcm a b) = lcm a b) : NormalizedGCDMonoid α := let exists_gcd a b := dvd_normalize_iff.2 (lcm_dvd (Dvd.intro b rfl) (Dvd.intro_left a rfl)) { (inferInstance : NormalizationMonoid α) with lcm gcd := fun a b => if a = 0 then normalize b else if b = 0 then normalize a else Classical.choose (exists_gcd a b) gcd_mul_lcm := fun a b => by beta_reduce split_ifs with h h_1 · rw [h, eq_zero_of_zero_dvd (dvd_lcm_left _ _), mul_zero, zero_mul] · rw [h_1, eq_zero_of_zero_dvd (dvd_lcm_right _ _), mul_zero, mul_zero] rw [mul_comm, ← Classical.choose_spec (exists_gcd a b)] exact normalize_associated (a * b) normalize_lcm normalize_gcd := fun a b => by dsimp [normalize] split_ifs with h h_1 · apply normalize_idem · apply normalize_idem have h0 : lcm a b ≠ 0 := by intro con have h := lcm_dvd (Dvd.intro b rfl) (Dvd.intro_left a rfl) rw [con, zero_dvd_iff, mul_eq_zero] at h cases h · exact absurd ‹a = 0› h · exact absurd ‹b = 0› h_1 apply mul_left_cancel₀ h0 refine _root_.trans ?_ (Classical.choose_spec (exists_gcd a b)) conv_lhs => congr rw [← normalize_lcm a b] erw [← normalize.map_mul, ← Classical.choose_spec (exists_gcd a b), normalize_idem] lcm_zero_left := fun a => eq_zero_of_zero_dvd (dvd_lcm_left _ _) lcm_zero_right := fun a => eq_zero_of_zero_dvd (dvd_lcm_right _ _) gcd_dvd_left := fun a b => by beta_reduce split_ifs with h h_1 · rw [h] apply dvd_zero · exact (normalize_associated _).dvd have h0 : lcm a b ≠ 0 := by intro con have h := lcm_dvd (Dvd.intro b rfl) (Dvd.intro_left a rfl) rw [con, zero_dvd_iff, mul_eq_zero] at h cases h · exact absurd ‹a = 0› h · exact absurd ‹b = 0› h_1 rw [← mul_dvd_mul_iff_left h0, ← Classical.choose_spec (exists_gcd a b), normalize_dvd_iff, mul_comm, mul_dvd_mul_iff_right h] apply dvd_lcm_right gcd_dvd_right := fun a b => by beta_reduce split_ifs with h h_1 · exact (normalize_associated _).dvd · rw [h_1] apply dvd_zero have h0 : lcm a b ≠ 0 := by intro con have h := lcm_dvd (Dvd.intro b rfl) (Dvd.intro_left a rfl) rw [con, zero_dvd_iff, mul_eq_zero] at h cases h · exact absurd ‹a = 0› h · exact absurd ‹b = 0› h_1 rw [← mul_dvd_mul_iff_left h0, ← Classical.choose_spec (exists_gcd a b), normalize_dvd_iff, mul_dvd_mul_iff_right h_1] apply dvd_lcm_left dvd_gcd := fun {a b c} ac ab => by beta_reduce split_ifs with h h_1 · apply dvd_normalize_iff.2 ab · apply dvd_normalize_iff.2 ac have h0 : lcm c b ≠ 0 := by intro con have h := lcm_dvd (Dvd.intro b rfl) (Dvd.intro_left c rfl) rw [con, zero_dvd_iff, mul_eq_zero] at h cases h · exact absurd ‹c = 0› h · exact absurd ‹b = 0› h_1 rw [← mul_dvd_mul_iff_left h0, ← Classical.choose_spec (dvd_normalize_iff.2 (lcm_dvd (Dvd.intro b rfl) (Dvd.intro_left c rfl))), dvd_normalize_iff] rcases ab with ⟨d, rfl⟩ rw [mul_eq_zero] at h_1 push_neg at h_1 rw [mul_comm a, ← mul_assoc, mul_dvd_mul_iff_right h_1.1] apply lcm_dvd (Dvd.intro d rfl) rw [mul_comm, mul_dvd_mul_iff_right h_1.2] apply ac } /-- Define a `GCDMonoid` structure on a monoid just from the existence of a `gcd`. -/ noncomputable def gcdMonoidOfExistsGCD [DecidableEq α] (h : ∀ a b : α, ∃ c : α, ∀ d : α, d ∣ a ∧ d ∣ b ↔ d ∣ c) : GCDMonoid α := gcdMonoidOfGCD (fun a b => Classical.choose (h a b)) (fun a b => ((Classical.choose_spec (h a b) (Classical.choose (h a b))).2 dvd_rfl).1) (fun a b => ((Classical.choose_spec (h a b) (Classical.choose (h a b))).2 dvd_rfl).2) fun {a b c} ac ab => (Classical.choose_spec (h c b) a).1 ⟨ac, ab⟩ /-- Define a `NormalizedGCDMonoid` structure on a monoid just from the existence of a `gcd`. -/ noncomputable def normalizedGCDMonoidOfExistsGCD [NormalizationMonoid α] [DecidableEq α] (h : ∀ a b : α, ∃ c : α, ∀ d : α, d ∣ a ∧ d ∣ b ↔ d ∣ c) : NormalizedGCDMonoid α := normalizedGCDMonoidOfGCD (fun a b => normalize (Classical.choose (h a b))) (fun a b => normalize_dvd_iff.2 ((Classical.choose_spec (h a b) (Classical.choose (h a b))).2 dvd_rfl).1) (fun a b => normalize_dvd_iff.2 ((Classical.choose_spec (h a b) (Classical.choose (h a b))).2 dvd_rfl).2) (fun {a b c} ac ab => dvd_normalize_iff.2 ((Classical.choose_spec (h c b) a).1 ⟨ac, ab⟩)) fun _ _ => normalize_idem _ /-- Define a `GCDMonoid` structure on a monoid just from the existence of an `lcm`. -/ noncomputable def gcdMonoidOfExistsLCM [DecidableEq α] (h : ∀ a b : α, ∃ c : α, ∀ d : α, a ∣ d ∧ b ∣ d ↔ c ∣ d) : GCDMonoid α := gcdMonoidOfLCM (fun a b => Classical.choose (h a b)) (fun a b => ((Classical.choose_spec (h a b) (Classical.choose (h a b))).2 dvd_rfl).1) (fun a b => ((Classical.choose_spec (h a b) (Classical.choose (h a b))).2 dvd_rfl).2) fun {a b c} ac ab => (Classical.choose_spec (h c b) a).1 ⟨ac, ab⟩ /-- Define a `NormalizedGCDMonoid` structure on a monoid just from the existence of an `lcm`. -/ noncomputable def normalizedGCDMonoidOfExistsLCM [NormalizationMonoid α] [DecidableEq α] (h : ∀ a b : α, ∃ c : α, ∀ d : α, a ∣ d ∧ b ∣ d ↔ c ∣ d) : NormalizedGCDMonoid α := normalizedGCDMonoidOfLCM (fun a b => normalize (Classical.choose (h a b))) (fun a b => dvd_normalize_iff.2 ((Classical.choose_spec (h a b) (Classical.choose (h a b))).2 dvd_rfl).1) (fun a b => dvd_normalize_iff.2 ((Classical.choose_spec (h a b) (Classical.choose (h a b))).2 dvd_rfl).2) (fun {a b c} ac ab => normalize_dvd_iff.2 ((Classical.choose_spec (h c b) a).1 ⟨ac, ab⟩)) fun _ _ => normalize_idem _ end Constructors namespace CommGroupWithZero variable (G₀ : Type*) [CommGroupWithZero G₀] [DecidableEq G₀] -- Porting note (#11083): very slow; improve performance? -- see Note [lower instance priority] instance (priority := 100) : NormalizedGCDMonoid G₀ where normUnit x := if h : x = 0 then 1 else (Units.mk0 x h)⁻¹ normUnit_zero := dif_pos rfl normUnit_mul := fun {x y} x0 y0 => Units.eq_iff.1 (by -- Porting note(#12129): additional beta reduction needed -- Porting note: `simp` reaches maximum heartbeat -- by Units.eq_iff.mp (by simp only [x0, y0, mul_comm]) beta_reduce split_ifs with h · rw [mul_eq_zero] at h cases h · exact absurd ‹x = 0› x0 · exact absurd ‹y = 0› y0 · rw [Units.mk0_mul, mul_inv_rev, mul_comm] ) normUnit_coe_units u := by -- Porting note(#12129): additional beta reduction needed beta_reduce rw [dif_neg (Units.ne_zero _), Units.mk0_val] gcd a b := if a = 0 ∧ b = 0 then 0 else 1 lcm a b := if a = 0 ∨ b = 0 then 0 else 1 gcd_dvd_left a b := by -- Porting note(#12129): additional beta reduction needed beta_reduce split_ifs with h · rw [h.1] · exact one_dvd _ gcd_dvd_right a b := by -- Porting note(#12129): additional beta reduction needed beta_reduce split_ifs with h · rw [h.2] · exact one_dvd _ dvd_gcd := fun {a b c} hac hab => by -- Porting note(#12129): additional beta reduction needed beta_reduce split_ifs with h · apply dvd_zero · rw [not_and_or] at h cases h · refine isUnit_iff_dvd_one.mp (isUnit_of_dvd_unit ?_ (IsUnit.mk0 _ ‹c ≠ 0›)) exact hac · refine isUnit_iff_dvd_one.mp (isUnit_of_dvd_unit ?_ (IsUnit.mk0 _ ‹b ≠ 0›)) exact hab gcd_mul_lcm a b := by by_cases ha : a = 0 · simp only [ha, true_and, true_or, ite_true, mul_zero, zero_mul] exact Associated.refl _ · by_cases hb : b = 0 · simp only [hb, and_true, or_true, ite_true, mul_zero] exact Associated.refl _ -- Porting note(#12129): additional beta reduction needed · beta_reduce rw [if_neg (not_and_of_not_left _ ha), one_mul, if_neg (not_or_of_not ha hb)] exact (associated_one_iff_isUnit.mpr ((IsUnit.mk0 _ ha).mul (IsUnit.mk0 _ hb))).symm lcm_zero_left b := if_pos (Or.inl rfl) lcm_zero_right a := if_pos (Or.inr rfl) -- `split_ifs` wants to split `normalize`, so handle the cases manually normalize_gcd a b := if h : a = 0 ∧ b = 0 then by simp [if_pos h] else by simp [if_neg h] normalize_lcm a b := if h : a = 0 ∨ b = 0 then by simp [if_pos h] else by simp [if_neg h] @[simp] theorem coe_normUnit {a : G₀} (h0 : a ≠ 0) : (↑(normUnit a) : G₀) = a⁻¹ := by simp [normUnit, h0] theorem normalize_eq_one {a : G₀} (h0 : a ≠ 0) : normalize a = 1 := by simp [normalize_apply, h0] end CommGroupWithZero namespace Associates variable [CancelCommMonoidWithZero α] [GCDMonoid α] instance instGCDMonoid : GCDMonoid (Associates α) where gcd := Quotient.map₂' gcd fun a₁ a₂ (ha : Associated _ _) b₁ b₂ (hb : Associated _ _) => ha.gcd hb lcm := Quotient.map₂' lcm fun a₁ a₂ (ha : Associated _ _) b₁ b₂ (hb : Associated _ _) => ha.lcm hb gcd_dvd_left := by rintro ⟨a⟩ ⟨b⟩; exact mk_le_mk_of_dvd (gcd_dvd_left _ _) gcd_dvd_right := by rintro ⟨a⟩ ⟨b⟩; exact mk_le_mk_of_dvd (gcd_dvd_right _ _) dvd_gcd := by rintro ⟨a⟩ ⟨b⟩ ⟨c⟩ hac hbc exact mk_le_mk_of_dvd (dvd_gcd (dvd_of_mk_le_mk hac) (dvd_of_mk_le_mk hbc)) gcd_mul_lcm := by rintro ⟨a⟩ ⟨b⟩ rw [associated_iff_eq] exact Quotient.sound <| gcd_mul_lcm _ _ lcm_zero_left := by rintro ⟨a⟩; exact congr_arg Associates.mk <| lcm_zero_left _ lcm_zero_right := by rintro ⟨a⟩; exact congr_arg Associates.mk <| lcm_zero_right _ theorem gcd_mk_mk {a b : α} : gcd (Associates.mk a) (Associates.mk b) = Associates.mk (gcd a b) := rfl theorem lcm_mk_mk {a b : α} : lcm (Associates.mk a) (Associates.mk b) = Associates.mk (lcm a b) := rfl end Associates
Algebra\GCDMonoid\Finset.lean
/- Copyright (c) 2020 Aaron Anderson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Aaron Anderson -/ import Mathlib.Data.Finset.Fold import Mathlib.Algebra.GCDMonoid.Multiset /-! # GCD and LCM operations on finsets ## Main definitions - `Finset.gcd` - the greatest common denominator of a `Finset` of elements of a `GCDMonoid` - `Finset.lcm` - the least common multiple of a `Finset` of elements of a `GCDMonoid` ## Implementation notes Many of the proofs use the lemmas `gcd_def` and `lcm_def`, which relate `Finset.gcd` and `Finset.lcm` to `Multiset.gcd` and `Multiset.lcm`. TODO: simplify with a tactic and `Data.Finset.Lattice` ## Tags finset, gcd -/ variable {ι α β γ : Type*} namespace Finset open Multiset variable [CancelCommMonoidWithZero α] [NormalizedGCDMonoid α] /-! ### lcm -/ section lcm /-- Least common multiple of a finite set -/ def lcm (s : Finset β) (f : β → α) : α := s.fold GCDMonoid.lcm 1 f variable {s s₁ s₂ : Finset β} {f : β → α} theorem lcm_def : s.lcm f = (s.1.map f).lcm := rfl @[simp] theorem lcm_empty : (∅ : Finset β).lcm f = 1 := fold_empty @[simp] theorem lcm_dvd_iff {a : α} : s.lcm f ∣ a ↔ ∀ b ∈ s, f b ∣ a := by apply Iff.trans Multiset.lcm_dvd simp only [Multiset.mem_map, and_imp, exists_imp] exact ⟨fun k b hb ↦ k _ _ hb rfl, fun k a' b hb h ↦ h ▸ k _ hb⟩ theorem lcm_dvd {a : α} : (∀ b ∈ s, f b ∣ a) → s.lcm f ∣ a := lcm_dvd_iff.2 theorem dvd_lcm {b : β} (hb : b ∈ s) : f b ∣ s.lcm f := lcm_dvd_iff.1 dvd_rfl _ hb @[simp] theorem lcm_insert [DecidableEq β] {b : β} : (insert b s : Finset β).lcm f = GCDMonoid.lcm (f b) (s.lcm f) := by by_cases h : b ∈ s · rw [insert_eq_of_mem h, (lcm_eq_right_iff (f b) (s.lcm f) (Multiset.normalize_lcm (s.1.map f))).2 (dvd_lcm h)] apply fold_insert h @[simp] theorem lcm_singleton {b : β} : ({b} : Finset β).lcm f = normalize (f b) := Multiset.lcm_singleton -- Porting note: Priority changed for `simpNF` @[simp 1100] theorem normalize_lcm : normalize (s.lcm f) = s.lcm f := by simp [lcm_def] theorem lcm_union [DecidableEq β] : (s₁ ∪ s₂).lcm f = GCDMonoid.lcm (s₁.lcm f) (s₂.lcm f) := Finset.induction_on s₁ (by rw [empty_union, lcm_empty, lcm_one_left, normalize_lcm]) fun a s _ ih ↦ by rw [insert_union, lcm_insert, lcm_insert, ih, lcm_assoc] theorem lcm_congr {f g : β → α} (hs : s₁ = s₂) (hfg : ∀ a ∈ s₂, f a = g a) : s₁.lcm f = s₂.lcm g := by subst hs exact Finset.fold_congr hfg theorem lcm_mono_fun {g : β → α} (h : ∀ b ∈ s, f b ∣ g b) : s.lcm f ∣ s.lcm g := lcm_dvd fun b hb ↦ (h b hb).trans (dvd_lcm hb) theorem lcm_mono (h : s₁ ⊆ s₂) : s₁.lcm f ∣ s₂.lcm f := lcm_dvd fun _ hb ↦ dvd_lcm (h hb) theorem lcm_image [DecidableEq β] {g : γ → β} (s : Finset γ) : (s.image g).lcm f = s.lcm (f ∘ g) := by classical induction' s using Finset.induction with c s _ ih <;> simp [*] theorem lcm_eq_lcm_image [DecidableEq α] : s.lcm f = (s.image f).lcm id := Eq.symm <| lcm_image _ theorem lcm_eq_zero_iff [Nontrivial α] : s.lcm f = 0 ↔ 0 ∈ f '' s := by simp only [Multiset.mem_map, lcm_def, Multiset.lcm_eq_zero_iff, Set.mem_image, mem_coe, ← Finset.mem_def] end lcm /-! ### gcd -/ section gcd /-- Greatest common divisor of a finite set -/ def gcd (s : Finset β) (f : β → α) : α := s.fold GCDMonoid.gcd 0 f variable {s s₁ s₂ : Finset β} {f : β → α} theorem gcd_def : s.gcd f = (s.1.map f).gcd := rfl @[simp] theorem gcd_empty : (∅ : Finset β).gcd f = 0 := fold_empty theorem dvd_gcd_iff {a : α} : a ∣ s.gcd f ↔ ∀ b ∈ s, a ∣ f b := by apply Iff.trans Multiset.dvd_gcd simp only [Multiset.mem_map, and_imp, exists_imp] exact ⟨fun k b hb ↦ k _ _ hb rfl, fun k a' b hb h ↦ h ▸ k _ hb⟩ theorem gcd_dvd {b : β} (hb : b ∈ s) : s.gcd f ∣ f b := dvd_gcd_iff.1 dvd_rfl _ hb theorem dvd_gcd {a : α} : (∀ b ∈ s, a ∣ f b) → a ∣ s.gcd f := dvd_gcd_iff.2 @[simp] theorem gcd_insert [DecidableEq β] {b : β} : (insert b s : Finset β).gcd f = GCDMonoid.gcd (f b) (s.gcd f) := by by_cases h : b ∈ s · rw [insert_eq_of_mem h, (gcd_eq_right_iff (f b) (s.gcd f) (Multiset.normalize_gcd (s.1.map f))).2 (gcd_dvd h)] apply fold_insert h @[simp] theorem gcd_singleton {b : β} : ({b} : Finset β).gcd f = normalize (f b) := Multiset.gcd_singleton -- Porting note: Priority changed for `simpNF` @[simp 1100] theorem normalize_gcd : normalize (s.gcd f) = s.gcd f := by simp [gcd_def] theorem gcd_union [DecidableEq β] : (s₁ ∪ s₂).gcd f = GCDMonoid.gcd (s₁.gcd f) (s₂.gcd f) := Finset.induction_on s₁ (by rw [empty_union, gcd_empty, gcd_zero_left, normalize_gcd]) fun a s _ ih ↦ by rw [insert_union, gcd_insert, gcd_insert, ih, gcd_assoc] theorem gcd_congr {f g : β → α} (hs : s₁ = s₂) (hfg : ∀ a ∈ s₂, f a = g a) : s₁.gcd f = s₂.gcd g := by subst hs exact Finset.fold_congr hfg theorem gcd_mono_fun {g : β → α} (h : ∀ b ∈ s, f b ∣ g b) : s.gcd f ∣ s.gcd g := dvd_gcd fun b hb ↦ (gcd_dvd hb).trans (h b hb) theorem gcd_mono (h : s₁ ⊆ s₂) : s₂.gcd f ∣ s₁.gcd f := dvd_gcd fun _ hb ↦ gcd_dvd (h hb) theorem gcd_image [DecidableEq β] {g : γ → β} (s : Finset γ) : (s.image g).gcd f = s.gcd (f ∘ g) := by classical induction' s using Finset.induction with c s _ ih <;> simp [*] theorem gcd_eq_gcd_image [DecidableEq α] : s.gcd f = (s.image f).gcd id := Eq.symm <| gcd_image _ theorem gcd_eq_zero_iff : s.gcd f = 0 ↔ ∀ x : β, x ∈ s → f x = 0 := by rw [gcd_def, Multiset.gcd_eq_zero_iff] constructor <;> intro h · intro b bs apply h (f b) simp only [Multiset.mem_map, mem_def.1 bs] use b simp only [mem_def.1 bs, eq_self_iff_true, and_self] · intro a as rw [Multiset.mem_map] at as rcases as with ⟨b, ⟨bs, rfl⟩⟩ apply h b (mem_def.1 bs) /- Porting note: The change from `p : α → Prop` to `p : α → Bool` made this slightly less nice with all the `decide`s around. -/ theorem gcd_eq_gcd_filter_ne_zero [DecidablePred fun x : β ↦ f x = 0] : s.gcd f = (s.filter fun x ↦ f x ≠ 0).gcd f := by classical trans ((s.filter fun x ↦ f x = 0) ∪ s.filter fun x ↦ (f x ≠ 0)).gcd f · rw [filter_union_filter_neg_eq] rw [gcd_union] refine Eq.trans (?_ : _ = GCDMonoid.gcd (0 : α) ?_) (?_ : GCDMonoid.gcd (0 : α) _ = _) · exact (gcd (filter (fun x => (f x ≠ 0)) s) f) · refine congr (congr rfl <| s.induction_on ?_ ?_) (by simp) · simp · intro a s _ h rw [filter_insert] split_ifs with h1 <;> simp [h, h1] simp only [gcd_zero_left, normalize_gcd] nonrec theorem gcd_mul_left {a : α} : (s.gcd fun x ↦ a * f x) = normalize a * s.gcd f := by classical refine s.induction_on ?_ ?_ · simp · intro b t _ h rw [gcd_insert, gcd_insert, h, ← gcd_mul_left] apply ((normalize_associated a).mul_right _).gcd_eq_right nonrec theorem gcd_mul_right {a : α} : (s.gcd fun x ↦ f x * a) = s.gcd f * normalize a := by classical refine s.induction_on ?_ ?_ · simp · intro b t _ h rw [gcd_insert, gcd_insert, h, ← gcd_mul_right] apply ((normalize_associated a).mul_left _).gcd_eq_right theorem extract_gcd' (f g : β → α) (hs : ∃ x, x ∈ s ∧ f x ≠ 0) (hg : ∀ b ∈ s, f b = s.gcd f * g b) : s.gcd g = 1 := ((@mul_right_eq_self₀ _ _ (s.gcd f) _).1 <| by conv_lhs => rw [← normalize_gcd, ← gcd_mul_left, ← gcd_congr rfl hg]).resolve_right <| by contrapose! hs exact gcd_eq_zero_iff.1 hs theorem extract_gcd (f : β → α) (hs : s.Nonempty) : ∃ g : β → α, (∀ b ∈ s, f b = s.gcd f * g b) ∧ s.gcd g = 1 := by classical by_cases h : ∀ x ∈ s, f x = (0 : α) · refine ⟨fun _ ↦ 1, fun b hb ↦ by rw [h b hb, gcd_eq_zero_iff.2 h, mul_one], ?_⟩ rw [gcd_eq_gcd_image, image_const hs, gcd_singleton, id, normalize_one] · choose g' hg using @gcd_dvd _ _ _ _ s f push_neg at h refine ⟨fun b ↦ if hb : b ∈ s then g' hb else 0, fun b hb ↦ ?_, extract_gcd' f _ h fun b hb ↦ ?_⟩ · simp only [hb, hg, dite_true] rw [dif_pos hb, hg hb] variable [Div α] [MulDivCancelClass α] {f : ι → α} {s : Finset ι} {i : ι} /-- Given a nonempty Finset `s` and a function `f` from `s` to `ℕ`, if `d = s.gcd`, then the `gcd` of `(f i) / d` is equal to `1`. -/ lemma gcd_div_eq_one (his : i ∈ s) (hfi : f i ≠ 0) : s.gcd (fun j ↦ f j / s.gcd f) = 1 := by obtain ⟨g, he, hg⟩ := Finset.extract_gcd f ⟨i, his⟩ refine (Finset.gcd_congr rfl fun a ha ↦ ?_).trans hg rw [he a ha, mul_div_cancel_left₀] exact mt Finset.gcd_eq_zero_iff.1 fun h ↦ hfi <| h i his lemma gcd_div_id_eq_one {s : Finset α} {a : α} (has : a ∈ s) (ha : a ≠ 0) : s.gcd (fun b ↦ b / s.gcd id) = 1 := gcd_div_eq_one has ha end gcd end Finset namespace Finset section IsDomain variable [CommRing α] [IsDomain α] [NormalizedGCDMonoid α] theorem gcd_eq_of_dvd_sub {s : Finset β} {f g : β → α} {a : α} (h : ∀ x : β, x ∈ s → a ∣ f x - g x) : GCDMonoid.gcd a (s.gcd f) = GCDMonoid.gcd a (s.gcd g) := by classical revert h refine s.induction_on ?_ ?_ · simp intro b s _ hi h rw [gcd_insert, gcd_insert, gcd_comm (f b), ← gcd_assoc, hi fun x hx ↦ h _ (mem_insert_of_mem hx), gcd_comm a, gcd_assoc, gcd_comm a (GCDMonoid.gcd _ _), gcd_comm (g b), gcd_assoc _ _ a, gcd_comm _ a] exact congr_arg _ (gcd_eq_of_dvd_sub_right (h _ (mem_insert_self _ _))) end IsDomain end Finset
Algebra\GCDMonoid\IntegrallyClosed.lean
/- Copyright (c) 2022 Andrew Yang. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Andrew Yang -/ import Mathlib.Algebra.GCDMonoid.Basic import Mathlib.RingTheory.IntegralClosure.IntegrallyClosed import Mathlib.RingTheory.Polynomial.Eisenstein.Basic /-! # GCD domains are integrally closed -/ open scoped Polynomial variable {R A : Type*} [CommRing R] [IsDomain R] [CommRing A] [Algebra R A] theorem IsLocalization.surj_of_gcd_domain [GCDMonoid R] (M : Submonoid R) [IsLocalization M A] (z : A) : ∃ a b : R, IsUnit (gcd a b) ∧ z * algebraMap R A b = algebraMap R A a := by obtain ⟨x, ⟨y, hy⟩, rfl⟩ := IsLocalization.mk'_surjective M z obtain ⟨x', y', hx', hy', hu⟩ := extract_gcd x y use x', y', hu rw [mul_comm, IsLocalization.mul_mk'_eq_mk'_of_mul] convert IsLocalization.mk'_mul_cancel_left (M := M) (S := A) _ _ using 2 rw [Subtype.coe_mk, hy', ← mul_comm y', mul_assoc]; conv_lhs => rw [hx'] instance (priority := 100) GCDMonoid.toIsIntegrallyClosed [h : Nonempty (GCDMonoid R)] : IsIntegrallyClosed R := (isIntegrallyClosed_iff (FractionRing R)).mpr fun {X} ⟨p, hp₁, hp₂⟩ => by cases h obtain ⟨x, y, hg, he⟩ := IsLocalization.surj_of_gcd_domain (nonZeroDivisors R) X have := Polynomial.dvd_pow_natDegree_of_eval₂_eq_zero (IsFractionRing.injective R <| FractionRing R) hp₁ y x _ hp₂ (by rw [mul_comm, he]) have : IsUnit y := by rw [isUnit_iff_dvd_one, ← one_pow] exact (dvd_gcd this <| dvd_refl y).trans (gcd_pow_left_dvd_pow_gcd.trans <| pow_dvd_pow_of_dvd (isUnit_iff_dvd_one.1 hg) _) use x * (this.unit⁻¹ : _) erw [map_mul, ← Units.coe_map_inv, eq_comm, Units.eq_mul_inv_iff_mul_eq] exact he
Algebra\GCDMonoid\Multiset.lean
/- Copyright (c) 2020 Aaron Anderson. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Aaron Anderson -/ import Mathlib.Algebra.GCDMonoid.Basic import Mathlib.Data.Multiset.FinsetOps import Mathlib.Data.Multiset.Fold /-! # GCD and LCM operations on multisets ## Main definitions - `Multiset.gcd` - the greatest common denominator of a `Multiset` of elements of a `GCDMonoid` - `Multiset.lcm` - the least common multiple of a `Multiset` of elements of a `GCDMonoid` ## Implementation notes TODO: simplify with a tactic and `Data.Multiset.Lattice` ## Tags multiset, gcd -/ namespace Multiset variable {α : Type*} [CancelCommMonoidWithZero α] [NormalizedGCDMonoid α] /-! ### LCM -/ section lcm /-- Least common multiple of a multiset -/ def lcm (s : Multiset α) : α := s.fold GCDMonoid.lcm 1 @[simp] theorem lcm_zero : (0 : Multiset α).lcm = 1 := fold_zero _ _ @[simp] theorem lcm_cons (a : α) (s : Multiset α) : (a ::ₘ s).lcm = GCDMonoid.lcm a s.lcm := fold_cons_left _ _ _ _ @[simp] theorem lcm_singleton {a : α} : ({a} : Multiset α).lcm = normalize a := (fold_singleton _ _ _).trans <| lcm_one_right _ @[simp] theorem lcm_add (s₁ s₂ : Multiset α) : (s₁ + s₂).lcm = GCDMonoid.lcm s₁.lcm s₂.lcm := Eq.trans (by simp [lcm]) (fold_add _ _ _ _ _) theorem lcm_dvd {s : Multiset α} {a : α} : s.lcm ∣ a ↔ ∀ b ∈ s, b ∣ a := Multiset.induction_on s (by simp) (by simp (config := { contextual := true }) [or_imp, forall_and, lcm_dvd_iff]) theorem dvd_lcm {s : Multiset α} {a : α} (h : a ∈ s) : a ∣ s.lcm := lcm_dvd.1 dvd_rfl _ h theorem lcm_mono {s₁ s₂ : Multiset α} (h : s₁ ⊆ s₂) : s₁.lcm ∣ s₂.lcm := lcm_dvd.2 fun _ hb ↦ dvd_lcm (h hb) /- Porting note: Following `Algebra.GCDMonoid.Basic`'s version of `normalize_gcd`, I'm giving this lower priority to avoid linter complaints about simp-normal form -/ /- Porting note: Mathport seems to be replacing `Multiset.induction_on s $` with `(Multiset.induction_on s)`, when it should be `Multiset.induction_on s <|`. -/ @[simp 1100] theorem normalize_lcm (s : Multiset α) : normalize s.lcm = s.lcm := Multiset.induction_on s (by simp) fun a s _ ↦ by simp @[simp] nonrec theorem lcm_eq_zero_iff [Nontrivial α] (s : Multiset α) : s.lcm = 0 ↔ (0 : α) ∈ s := by induction' s using Multiset.induction_on with a s ihs · simp only [lcm_zero, one_ne_zero, not_mem_zero] · simp only [mem_cons, lcm_cons, lcm_eq_zero_iff, ihs, @eq_comm _ a] variable [DecidableEq α] @[simp] theorem lcm_dedup (s : Multiset α) : (dedup s).lcm = s.lcm := Multiset.induction_on s (by simp) fun a s IH ↦ by by_cases h : a ∈ s <;> simp [IH, h] unfold lcm rw [← cons_erase h, fold_cons_left, ← lcm_assoc, lcm_same] apply lcm_eq_of_associated_left (associated_normalize _) @[simp] theorem lcm_ndunion (s₁ s₂ : Multiset α) : (ndunion s₁ s₂).lcm = GCDMonoid.lcm s₁.lcm s₂.lcm := by rw [← lcm_dedup, dedup_ext.2, lcm_dedup, lcm_add] simp @[simp] theorem lcm_union (s₁ s₂ : Multiset α) : (s₁ ∪ s₂).lcm = GCDMonoid.lcm s₁.lcm s₂.lcm := by rw [← lcm_dedup, dedup_ext.2, lcm_dedup, lcm_add] simp @[simp] theorem lcm_ndinsert (a : α) (s : Multiset α) : (ndinsert a s).lcm = GCDMonoid.lcm a s.lcm := by rw [← lcm_dedup, dedup_ext.2, lcm_dedup, lcm_cons] simp end lcm /-! ### GCD -/ section gcd /-- Greatest common divisor of a multiset -/ def gcd (s : Multiset α) : α := s.fold GCDMonoid.gcd 0 @[simp] theorem gcd_zero : (0 : Multiset α).gcd = 0 := fold_zero _ _ @[simp] theorem gcd_cons (a : α) (s : Multiset α) : (a ::ₘ s).gcd = GCDMonoid.gcd a s.gcd := fold_cons_left _ _ _ _ @[simp] theorem gcd_singleton {a : α} : ({a} : Multiset α).gcd = normalize a := (fold_singleton _ _ _).trans <| gcd_zero_right _ @[simp] theorem gcd_add (s₁ s₂ : Multiset α) : (s₁ + s₂).gcd = GCDMonoid.gcd s₁.gcd s₂.gcd := Eq.trans (by simp [gcd]) (fold_add _ _ _ _ _) theorem dvd_gcd {s : Multiset α} {a : α} : a ∣ s.gcd ↔ ∀ b ∈ s, a ∣ b := Multiset.induction_on s (by simp) (by simp (config := { contextual := true }) [or_imp, forall_and, dvd_gcd_iff]) theorem gcd_dvd {s : Multiset α} {a : α} (h : a ∈ s) : s.gcd ∣ a := dvd_gcd.1 dvd_rfl _ h theorem gcd_mono {s₁ s₂ : Multiset α} (h : s₁ ⊆ s₂) : s₂.gcd ∣ s₁.gcd := dvd_gcd.2 fun _ hb ↦ gcd_dvd (h hb) /- Porting note: Following `Algebra.GCDMonoid.Basic`'s version of `normalize_gcd`, I'm giving this lower priority to avoid linter complaints about simp-normal form -/ @[simp 1100] theorem normalize_gcd (s : Multiset α) : normalize s.gcd = s.gcd := Multiset.induction_on s (by simp) fun a s _ ↦ by simp theorem gcd_eq_zero_iff (s : Multiset α) : s.gcd = 0 ↔ ∀ x : α, x ∈ s → x = 0 := by constructor · intro h x hx apply eq_zero_of_zero_dvd rw [← h] apply gcd_dvd hx · refine s.induction_on ?_ ?_ · simp intro a s sgcd h simp [h a (mem_cons_self a s), sgcd fun x hx ↦ h x (mem_cons_of_mem hx)] theorem gcd_map_mul (a : α) (s : Multiset α) : (s.map (a * ·)).gcd = normalize a * s.gcd := by refine s.induction_on ?_ fun b s ih ↦ ?_ · simp_rw [map_zero, gcd_zero, mul_zero] · simp_rw [map_cons, gcd_cons, ← gcd_mul_left] rw [ih] apply ((normalize_associated a).mul_right _).gcd_eq_right section variable [DecidableEq α] @[simp] theorem gcd_dedup (s : Multiset α) : (dedup s).gcd = s.gcd := Multiset.induction_on s (by simp) fun a s IH ↦ by by_cases h : a ∈ s <;> simp [IH, h] unfold gcd rw [← cons_erase h, fold_cons_left, ← gcd_assoc, gcd_same] apply (associated_normalize _).gcd_eq_left @[simp] theorem gcd_ndunion (s₁ s₂ : Multiset α) : (ndunion s₁ s₂).gcd = GCDMonoid.gcd s₁.gcd s₂.gcd := by rw [← gcd_dedup, dedup_ext.2, gcd_dedup, gcd_add] simp @[simp] theorem gcd_union (s₁ s₂ : Multiset α) : (s₁ ∪ s₂).gcd = GCDMonoid.gcd s₁.gcd s₂.gcd := by rw [← gcd_dedup, dedup_ext.2, gcd_dedup, gcd_add] simp @[simp] theorem gcd_ndinsert (a : α) (s : Multiset α) : (ndinsert a s).gcd = GCDMonoid.gcd a s.gcd := by rw [← gcd_dedup, dedup_ext.2, gcd_dedup, gcd_cons] simp end theorem extract_gcd' (s t : Multiset α) (hs : ∃ x, x ∈ s ∧ x ≠ (0 : α)) (ht : s = t.map (s.gcd * ·)) : t.gcd = 1 := ((@mul_right_eq_self₀ _ _ s.gcd _).1 <| by conv_lhs => rw [← normalize_gcd, ← gcd_map_mul, ← ht]).resolve_right <| by contrapose! hs exact s.gcd_eq_zero_iff.1 hs /- Porting note: Deprecated lemmas like `map_repeat` and `eq_repeat` weren't "officially" converted to `Multiset.replicate` format yet, so I made some ad hoc ones in `Data.Multiset.Basic` using the originals. -/ /- Porting note: The old proof used a strange form `have := _, refine ⟨s.pmap @f (fun _ ↦ id), this, extract_gcd' s _ h this⟩,` so I rearranged the proof slightly. -/ theorem extract_gcd (s : Multiset α) (hs : s ≠ 0) : ∃ t : Multiset α, s = t.map (s.gcd * ·) ∧ t.gcd = 1 := by classical by_cases h : ∀ x ∈ s, x = (0 : α) · use replicate (card s) 1 rw [map_replicate, eq_replicate, mul_one, s.gcd_eq_zero_iff.2 h, ← nsmul_singleton, ← gcd_dedup, dedup_nsmul (card_pos.2 hs).ne', dedup_singleton, gcd_singleton] exact ⟨⟨rfl, h⟩, normalize_one⟩ · choose f hf using @gcd_dvd _ _ _ s push_neg at h refine ⟨s.pmap @f fun _ ↦ id, ?_, extract_gcd' s _ h ?_⟩ <;> · rw [map_pmap] conv_lhs => rw [← s.map_id, ← s.pmap_eq_map _ _ fun _ ↦ id] congr with (x hx) rw [id, ← hf hx] end gcd end Multiset
Algebra\GCDMonoid\Nat.lean
/- Copyright (c) 2018 Johannes Hölzl. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Johannes Hölzl, Jens Wagemaker, Aaron Anderson -/ import Mathlib.Algebra.GCDMonoid.Basic import Mathlib.Algebra.Order.Ring.Int import Mathlib.Data.Int.GCD /-! # ℕ and ℤ are normalized GCD monoids. ## Main statements * ℕ is a `GCDMonoid` * ℕ is a `NormalizedGCDMonoid` * ℤ is a `NormalizationMonoid` * ℤ is a `GCDMonoid` * ℤ is a `NormalizedGCDMonoid` ## Tags natural numbers, integers, normalization monoid, gcd monoid, greatest common divisor -/ /-- `ℕ` is a gcd_monoid. -/ instance : GCDMonoid ℕ where gcd := Nat.gcd lcm := Nat.lcm gcd_dvd_left := Nat.gcd_dvd_left gcd_dvd_right := Nat.gcd_dvd_right dvd_gcd := Nat.dvd_gcd gcd_mul_lcm a b := by rw [Nat.gcd_mul_lcm]; rfl lcm_zero_left := Nat.lcm_zero_left lcm_zero_right := Nat.lcm_zero_right theorem gcd_eq_nat_gcd (m n : ℕ) : gcd m n = Nat.gcd m n := rfl theorem lcm_eq_nat_lcm (m n : ℕ) : lcm m n = Nat.lcm m n := rfl instance : NormalizedGCDMonoid ℕ := { (inferInstance : GCDMonoid ℕ), (inferInstance : NormalizationMonoid ℕ) with normalize_gcd := fun _ _ => normalize_eq _ normalize_lcm := fun _ _ => normalize_eq _ } namespace Int section NormalizationMonoid instance normalizationMonoid : NormalizationMonoid ℤ where normUnit a := if 0 ≤ a then 1 else -1 normUnit_zero := if_pos le_rfl normUnit_mul {a b} hna hnb := by cases' hna.lt_or_lt with ha ha <;> cases' hnb.lt_or_lt with hb hb <;> simp [mul_nonneg_iff, ha.le, ha.not_le, hb.le, hb.not_le] normUnit_coe_units u := (units_eq_one_or u).elim (fun eq => eq.symm ▸ if_pos zero_le_one) fun eq => eq.symm ▸ if_neg (not_le_of_gt <| show (-1 : ℤ) < 0 by decide) -- Porting note: added theorem normUnit_eq (z : ℤ) : normUnit z = if 0 ≤ z then 1 else -1 := rfl theorem normalize_of_nonneg {z : ℤ} (h : 0 ≤ z) : normalize z = z := by rw [normalize_apply, normUnit_eq, if_pos h, Units.val_one, mul_one] theorem normalize_of_nonpos {z : ℤ} (h : z ≤ 0) : normalize z = -z := by obtain rfl | h := h.eq_or_lt · simp · rw [normalize_apply, normUnit_eq, if_neg (not_le_of_gt h), Units.val_neg, Units.val_one, mul_neg_one] theorem normalize_coe_nat (n : ℕ) : normalize (n : ℤ) = n := normalize_of_nonneg (ofNat_le_ofNat_of_le <| Nat.zero_le n) theorem abs_eq_normalize (z : ℤ) : |z| = normalize z := by cases le_total 0 z <;> simp [-normalize_apply, normalize_of_nonneg, normalize_of_nonpos, *] theorem nonneg_of_normalize_eq_self {z : ℤ} (hz : normalize z = z) : 0 ≤ z := abs_eq_self.1 <| by rw [abs_eq_normalize, hz] theorem nonneg_iff_normalize_eq_self (z : ℤ) : normalize z = z ↔ 0 ≤ z := ⟨nonneg_of_normalize_eq_self, normalize_of_nonneg⟩ theorem eq_of_associated_of_nonneg {a b : ℤ} (h : Associated a b) (ha : 0 ≤ a) (hb : 0 ≤ b) : a = b := dvd_antisymm_of_normalize_eq (normalize_of_nonneg ha) (normalize_of_nonneg hb) h.dvd h.symm.dvd end NormalizationMonoid section GCDMonoid instance : GCDMonoid ℤ where gcd a b := Int.gcd a b lcm a b := Int.lcm a b gcd_dvd_left a b := Int.gcd_dvd_left gcd_dvd_right a b := Int.gcd_dvd_right dvd_gcd := dvd_gcd gcd_mul_lcm a b := by rw [← Int.ofNat_mul, gcd_mul_lcm, natCast_natAbs, abs_eq_normalize] exact normalize_associated (a * b) lcm_zero_left a := natCast_eq_zero.2 <| Nat.lcm_zero_left _ lcm_zero_right a := natCast_eq_zero.2 <| Nat.lcm_zero_right _ instance : NormalizedGCDMonoid ℤ := { Int.normalizationMonoid, (inferInstance : GCDMonoid ℤ) with normalize_gcd := fun _ _ => normalize_coe_nat _ normalize_lcm := fun _ _ => normalize_coe_nat _ } theorem coe_gcd (i j : ℤ) : ↑(Int.gcd i j) = GCDMonoid.gcd i j := rfl theorem coe_lcm (i j : ℤ) : ↑(Int.lcm i j) = GCDMonoid.lcm i j := rfl theorem natAbs_gcd (i j : ℤ) : natAbs (GCDMonoid.gcd i j) = Int.gcd i j := rfl theorem natAbs_lcm (i j : ℤ) : natAbs (GCDMonoid.lcm i j) = Int.lcm i j := rfl end GCDMonoid theorem exists_unit_of_abs (a : ℤ) : ∃ (u : ℤ) (_ : IsUnit u), (Int.natAbs a : ℤ) = u * a := by cases' natAbs_eq a with h h · use 1, isUnit_one rw [← h, one_mul] · use -1, isUnit_one.neg rw [← neg_eq_iff_eq_neg.mpr h] simp only [neg_mul, one_mul] theorem gcd_eq_natAbs {a b : ℤ} : Int.gcd a b = Nat.gcd a.natAbs b.natAbs := rfl end Int /-- Maps an associate class of integers consisting of `-n, n` to `n : ℕ` -/ def associatesIntEquivNat : Associates ℤ ≃ ℕ := by refine ⟨(·.out.natAbs), (Associates.mk ·), ?_, fun n ↦ ?_⟩ · refine Associates.forall_associated.2 fun a ↦ ?_ refine Associates.mk_eq_mk_iff_associated.2 <| Associated.symm <| ⟨normUnit a, ?_⟩ simp [Int.abs_eq_normalize] · dsimp only [Associates.out_mk] rw [← Int.abs_eq_normalize, Int.natAbs_abs, Int.natAbs_ofNat] theorem Int.associated_natAbs (k : ℤ) : Associated k k.natAbs := associated_of_dvd_dvd (Int.dvd_natCast.mpr dvd_rfl) (Int.natAbs_dvd.mpr dvd_rfl) theorem Int.associated_iff_natAbs {a b : ℤ} : Associated a b ↔ a.natAbs = b.natAbs := by rw [← dvd_dvd_iff_associated, ← Int.natAbs_dvd_natAbs, ← Int.natAbs_dvd_natAbs, dvd_dvd_iff_associated] exact associated_iff_eq theorem Int.associated_iff {a b : ℤ} : Associated a b ↔ a = b ∨ a = -b := by rw [Int.associated_iff_natAbs] exact Int.natAbs_eq_natAbs_iff
Algebra\Group\AddChar.lean
/- Copyright (c) 2022 Michael Stoll. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Michael Stoll -/ import Mathlib.Logic.Equiv.TransferInstance /-! # Characters from additive to multiplicative monoids Let `A` be an additive monoid, and `M` a multiplicative one. An *additive character* of `A` with values in `M` is simply a map `A → M` which intertwines the addition operation on `A` with the multiplicative operation on `M`. We define these objects, using the namespace `AddChar`, and show that if `A` is a commutative group under addition, then the additive characters are also a group (written multiplicatively). Note that we do not need `M` to be a group here. We also include some constructions specific to the case when `A = R` is a ring; then we define `mulShift ψ r`, where `ψ : AddChar R M` and `r : R`, to be the character defined by `x ↦ ψ (r * x)`. For more refined results of a number-theoretic nature (primitive characters, Gauss sums, etc) see `Mathlib.NumberTheory.LegendreSymbol.AddCharacter`. ## Tags additive character -/ /-! ### Definitions related to and results on additive characters -/ open Function Multiplicative section AddCharDef -- The domain of our additive characters variable (A : Type*) [AddMonoid A] -- The target variable (M : Type*) [Monoid M] /-- `AddChar A M` is the type of maps `A → M`, for `A` an additive monoid and `M` a multiplicative monoid, which intertwine addition in `A` with multiplication in `M`. We only put the typeclasses needed for the definition, although in practice we are usually interested in much more specific cases (e.g. when `A` is a group and `M` a commutative ring). -/ structure AddChar where /-- The underlying function. Do not use this function directly. Instead use the coercion coming from the `FunLike` instance. -/ toFun : A → M /-- The function maps `0` to `1`. Do not use this directly. Instead use `AddChar.map_zero_eq_one`. -/ map_zero_eq_one' : toFun 0 = 1 /-- The function maps addition in `A` to multiplication in `M`. Do not use this directly. Instead use `AddChar.map_add_eq_mul`. -/ map_add_eq_mul' : ∀ a b : A, toFun (a + b) = toFun a * toFun b end AddCharDef namespace AddChar section Basic -- results which don't require commutativity or inverses variable {A B M N : Type*} [AddMonoid A] [AddMonoid B] [Monoid M] [Monoid N] {ψ : AddChar A M} /-- Define coercion to a function. -/ instance instFunLike : FunLike (AddChar A M) A M where coe := AddChar.toFun coe_injective' φ ψ h := by cases φ; cases ψ; congr -- Porting note (#5229): added. @[ext] lemma ext (f g : AddChar A M) (h : ∀ x : A, f x = g x) : f = g := DFunLike.ext f g h @[simp] lemma coe_mk (f : A → M) (map_zero_eq_one' : f 0 = 1) (map_add_eq_mul' : ∀ a b : A, f (a + b) = f a * f b) : AddChar.mk f map_zero_eq_one' map_add_eq_mul' = f := by rfl /-- An additive character maps `0` to `1`. -/ @[simp] lemma map_zero_eq_one (ψ : AddChar A M) : ψ 0 = 1 := ψ.map_zero_eq_one' /-- An additive character maps sums to products. -/ lemma map_add_eq_mul (ψ : AddChar A M) (x y : A) : ψ (x + y) = ψ x * ψ y := ψ.map_add_eq_mul' x y @[deprecated (since := "2024-06-06")] alias map_zero_one := map_zero_eq_one @[deprecated (since := "2024-06-06")] alias map_add_mul := map_add_eq_mul /-- Interpret an additive character as a monoid homomorphism. -/ def toMonoidHom (φ : AddChar A M) : Multiplicative A →* M where toFun := φ.toFun map_one' := φ.map_zero_eq_one' map_mul' := φ.map_add_eq_mul' -- this instance was a bad idea and conflicted with `instFunLike` above @[simp] lemma toMonoidHom_apply (ψ : AddChar A M) (a : Multiplicative A) : ψ.toMonoidHom a = ψ (Multiplicative.toAdd a) := rfl /-- An additive character maps multiples by natural numbers to powers. -/ lemma map_nsmul_eq_pow (ψ : AddChar A M) (n : ℕ) (x : A) : ψ (n • x) = ψ x ^ n := ψ.toMonoidHom.map_pow x n @[deprecated (since := "2024-06-06")] alias map_nsmul_pow := map_nsmul_eq_pow /-- Additive characters `A → M` are the same thing as monoid homomorphisms from `Multiplicative A` to `M`. -/ def toMonoidHomEquiv : AddChar A M ≃ (Multiplicative A →* M) where toFun φ := φ.toMonoidHom invFun f := { toFun := f.toFun map_zero_eq_one' := f.map_one' map_add_eq_mul' := f.map_mul' } left_inv _ := rfl right_inv _ := rfl @[simp, norm_cast] lemma coe_toMonoidHomEquiv (ψ : AddChar A M) : ⇑(toMonoidHomEquiv ψ) = ψ ∘ Multiplicative.toAdd := rfl @[simp, norm_cast] lemma coe_toMonoidHomEquiv_symm (ψ : Multiplicative A →* M) : ⇑(toMonoidHomEquiv.symm ψ) = ψ ∘ Multiplicative.ofAdd := rfl @[simp] lemma toMonoidHomEquiv_apply (ψ : AddChar A M) (a : Multiplicative A) : toMonoidHomEquiv ψ a = ψ (Multiplicative.toAdd a) := rfl @[simp] lemma toMonoidHomEquiv_symm_apply (ψ : Multiplicative A →* M) (a : A) : toMonoidHomEquiv.symm ψ a = ψ (Multiplicative.ofAdd a) := rfl /-- Interpret an additive character as a monoid homomorphism. -/ def toAddMonoidHom (φ : AddChar A M) : A →+ Additive M where toFun := φ.toFun map_zero' := φ.map_zero_eq_one' map_add' := φ.map_add_eq_mul' @[simp] lemma coe_toAddMonoidHom (ψ : AddChar A M) : ⇑ψ.toAddMonoidHom = Additive.ofMul ∘ ψ := rfl @[simp] lemma toAddMonoidHom_apply (ψ : AddChar A M) (a : A) : ψ.toAddMonoidHom a = Additive.ofMul (ψ a) := rfl /-- Additive characters `A → M` are the same thing as additive homomorphisms from `A` to `Additive M`. -/ def toAddMonoidHomEquiv : AddChar A M ≃ (A →+ Additive M) where toFun φ := φ.toAddMonoidHom invFun f := { toFun := f.toFun map_zero_eq_one' := f.map_zero' map_add_eq_mul' := f.map_add' } left_inv _ := rfl right_inv _ := rfl @[simp, norm_cast] lemma coe_toAddMonoidHomEquiv (ψ : AddChar A M) : ⇑(toAddMonoidHomEquiv ψ) = Additive.ofMul ∘ ψ := rfl @[simp, norm_cast] lemma coe_toAddMonoidHomEquiv_symm (ψ : A →+ Additive M) : ⇑(toAddMonoidHomEquiv.symm ψ) = Additive.toMul ∘ ψ := rfl @[simp] lemma toAddMonoidHomEquiv_apply (ψ : AddChar A M) (a : A) : toAddMonoidHomEquiv ψ a = Additive.ofMul (ψ a) := rfl @[simp] lemma toAddMonoidHomEquiv_symm_apply (ψ : A →+ Additive M) (a : A) : toAddMonoidHomEquiv.symm ψ a = Additive.toMul (ψ a) := rfl /-- The trivial additive character (sending everything to `1`) is `(1 : AddChar A M).` -/ instance instOne : One (AddChar A M) := toMonoidHomEquiv.one @[simp, norm_cast] lemma coe_one : ⇑(1 : AddChar A M) = 1 := rfl @[simp] lemma one_apply (a : A) : (1 : AddChar A M) a = 1 := rfl instance instInhabited : Inhabited (AddChar A M) := ⟨1⟩ /-- Composing a `MonoidHom` with an `AddChar` yields another `AddChar`. -/ def _root_.MonoidHom.compAddChar {N : Type*} [Monoid N] (f : M →* N) (φ : AddChar A M) : AddChar A N := toMonoidHomEquiv.symm (f.comp φ.toMonoidHom) @[simp, norm_cast] lemma _root_.MonoidHom.coe_compAddChar {N : Type*} [Monoid N] (f : M →* N) (φ : AddChar A M) : f.compAddChar φ = f ∘ φ := rfl @[simp, norm_cast] lemma _root_.MonoidHom.compAddChar_apply (f : M →* N) (φ : AddChar A M) : f.compAddChar φ = f ∘ φ := rfl lemma _root_.MonoidHom.compAddChar_injective_left (ψ : AddChar A M) (hψ : Surjective ψ) : Injective fun f : M →* N ↦ f.compAddChar ψ := by rintro f g h; rw [DFunLike.ext'_iff] at h ⊢; exact hψ.injective_comp_right h lemma _root_.MonoidHom.compAddChar_injective_right (f : M →* N) (hf : Injective f) : Injective fun ψ : AddChar B M ↦ f.compAddChar ψ := by rintro ψ χ h; rw [DFunLike.ext'_iff] at h ⊢; exact hf.comp_left h /-- Composing an `AddChar` with an `AddMonoidHom` yields another `AddChar`. -/ def compAddMonoidHom (φ : AddChar B M) (f : A →+ B) : AddChar A M := toAddMonoidHomEquiv.symm (φ.toAddMonoidHom.comp f) @[simp, norm_cast] lemma coe_compAddMonoidHom (φ : AddChar B M) (f : A →+ B) : φ.compAddMonoidHom f = φ ∘ f := rfl @[simp] lemma compAddMonoidHom_apply (ψ : AddChar B M) (f : A →+ B) (a : A) : ψ.compAddMonoidHom f a = ψ (f a) := rfl lemma compAddMonoidHom_injective_left (f : A →+ B) (hf : Surjective f) : Injective fun ψ : AddChar B M ↦ ψ.compAddMonoidHom f := by rintro ψ χ h; rw [DFunLike.ext'_iff] at h ⊢; exact hf.injective_comp_right h lemma compAddMonoidHom_injective_right (ψ : AddChar B M) (hψ : Injective ψ) : Injective fun f : A →+ B ↦ ψ.compAddMonoidHom f := by rintro f g h rw [DFunLike.ext'_iff] at h ⊢; exact hψ.comp_left h lemma eq_one_iff : ψ = 1 ↔ ∀ x, ψ x = 1 := DFunLike.ext_iff lemma ne_one_iff : ψ ≠ 1 ↔ ∃ x, ψ x ≠ 1 := DFunLike.ne_iff /-- An additive character is *nontrivial* if it takes a value `≠ 1`. -/ @[deprecated (since := "2024-06-06")] def IsNontrivial (ψ : AddChar A M) : Prop := ∃ a : A, ψ a ≠ 1 set_option linter.deprecated false in /-- An additive character is nontrivial iff it is not the trivial character. -/ @[deprecated ne_one_iff (since := "2024-06-06")] lemma isNontrivial_iff_ne_trivial (ψ : AddChar A M) : IsNontrivial ψ ↔ ψ ≠ 1 := not_forall.symm.trans (DFunLike.ext_iff (f := ψ) (g := 1)).symm.not end Basic section toCommMonoid variable {A M : Type*} [AddMonoid A] [CommMonoid M] /-- When `M` is commutative, `AddChar A M` is a commutative monoid. -/ instance instCommMonoid : CommMonoid (AddChar A M) := toMonoidHomEquiv.commMonoid @[simp, norm_cast] lemma coe_mul (ψ χ : AddChar A M) : ⇑(ψ * χ) = ψ * χ := rfl @[simp, norm_cast] lemma coe_pow (ψ : AddChar A M) (n : ℕ) : ⇑(ψ ^ n) = ψ ^ n := rfl @[simp, norm_cast] lemma mul_apply (ψ φ : AddChar A M) (a : A) : (ψ * φ) a = ψ a * φ a := rfl @[simp, norm_cast] lemma pow_apply (ψ : AddChar A M) (n : ℕ) (a : A) : (ψ ^ n) a = (ψ a) ^ n := rfl /-- The natural equivalence to `(Multiplicative A →* M)` is a monoid isomorphism. -/ def toMonoidHomMulEquiv : AddChar A M ≃* (Multiplicative A →* M) := { toMonoidHomEquiv with map_mul' := fun φ ψ ↦ by rfl } /-- Additive characters `A → M` are the same thing as additive homomorphisms from `A` to `Additive M`. -/ def toAddMonoidAddEquiv : Additive (AddChar A M) ≃+ (A →+ Additive M) := { toAddMonoidHomEquiv with map_add' := fun φ ψ ↦ by rfl } end toCommMonoid /-! ## Additive characters of additive abelian groups -/ section fromAddCommGroup variable {A M : Type*} [AddCommGroup A] [CommMonoid M] /-- The additive characters on a commutative additive group form a commutative group. Note that the inverse is defined using negation on the domain; we do not assume `M` has an inversion operation for the definition (but see `AddChar.map_neg_eq_inv` below). -/ instance instCommGroup : CommGroup (AddChar A M) := { instCommMonoid with inv := fun ψ ↦ ψ.compAddMonoidHom negAddMonoidHom mul_left_inv := fun ψ ↦ by ext1 x; simp [negAddMonoidHom, ← map_add_eq_mul]} @[simp] lemma inv_apply (ψ : AddChar A M) (x : A) : ψ⁻¹ x = ψ (-x) := rfl end fromAddCommGroup section fromAddGrouptoCommMonoid /-- The values of an additive character on an additive group are units. -/ lemma val_isUnit {A M} [AddGroup A] [Monoid M] (φ : AddChar A M) (a : A) : IsUnit (φ a) := IsUnit.map φ.toMonoidHom <| Group.isUnit (Multiplicative.ofAdd a) end fromAddGrouptoCommMonoid section fromAddGrouptoDivisionMonoid variable {A M : Type*} [AddGroup A] [DivisionMonoid M] /-- An additive character maps negatives to inverses (when defined) -/ lemma map_neg_eq_inv (ψ : AddChar A M) (a : A) : ψ (-a) = (ψ a)⁻¹ := by apply eq_inv_of_mul_eq_one_left simp only [← map_add_eq_mul, add_left_neg, map_zero_eq_one] /-- An additive character maps integer scalar multiples to integer powers. -/ lemma map_zsmul_eq_zpow (ψ : AddChar A M) (n : ℤ) (a : A) : ψ (n • a) = (ψ a) ^ n := ψ.toMonoidHom.map_zpow a n @[deprecated (since := "2024-06-06")] alias map_neg_inv := map_neg_eq_inv @[deprecated (since := "2024-06-06")] alias map_zsmul_zpow := map_zsmul_eq_zpow end fromAddGrouptoDivisionMonoid section fromAddGrouptoDivisionCommMonoid variable {A M : Type*} [AddCommGroup A] [DivisionCommMonoid M] lemma inv_apply' (ψ : AddChar A M) (x : A) : ψ⁻¹ x = (ψ x)⁻¹ := by rw [inv_apply, map_neg_eq_inv] lemma map_sub_eq_div (ψ : AddChar A M) (a b : A) : ψ (a - b) = ψ a / ψ b := ψ.toMonoidHom.map_div _ _ lemma injective_iff {ψ : AddChar A M} : Injective ψ ↔ ∀ ⦃x⦄, ψ x = 1 → x = 0 := ψ.toMonoidHom.ker_eq_bot_iff.symm.trans eq_bot_iff end fromAddGrouptoDivisionCommMonoid /-! ## Additive characters of rings -/ section Ring -- The domain and target of our additive characters. Now we restrict to a ring in the domain. variable {R M : Type*} [Ring R] [CommMonoid M] /-- Define the multiplicative shift of an additive character. This satisfies `mulShift ψ a x = ψ (a * x)`. -/ def mulShift (ψ : AddChar R M) (r : R) : AddChar R M := ψ.compAddMonoidHom (AddMonoidHom.mulLeft r) @[simp] lemma mulShift_apply {ψ : AddChar R M} {r : R} {x : R} : mulShift ψ r x = ψ (r * x) := rfl /-- `ψ⁻¹ = mulShift ψ (-1))`. -/ theorem inv_mulShift (ψ : AddChar R M) : ψ⁻¹ = mulShift ψ (-1) := by ext rw [inv_apply, mulShift_apply, neg_mul, one_mul] /-- If `n` is a natural number, then `mulShift ψ n x = (ψ x) ^ n`. -/ theorem mulShift_spec' (ψ : AddChar R M) (n : ℕ) (x : R) : mulShift ψ n x = ψ x ^ n := by rw [mulShift_apply, ← nsmul_eq_mul, map_nsmul_eq_pow] /-- If `n` is a natural number, then `ψ ^ n = mulShift ψ n`. -/ theorem pow_mulShift (ψ : AddChar R M) (n : ℕ) : ψ ^ n = mulShift ψ n := by ext x rw [pow_apply, ← mulShift_spec'] /-- The product of `mulShift ψ r` and `mulShift ψ s` is `mulShift ψ (r + s)`. -/ theorem mulShift_mul (ψ : AddChar R M) (r s : R) : mulShift ψ r * mulShift ψ s = mulShift ψ (r + s) := by ext rw [mulShift_apply, right_distrib, map_add_eq_mul]; norm_cast lemma mulShift_mulShift (ψ : AddChar R M) (r s : R) : mulShift (mulShift ψ r) s = mulShift ψ (r * s) := by ext simp only [mulShift_apply, mul_assoc] /-- `mulShift ψ 0` is the trivial character. -/ @[simp] theorem mulShift_zero (ψ : AddChar R M) : mulShift ψ 0 = 1 := by ext; rw [mulShift_apply, zero_mul, map_zero_eq_one, one_apply] @[simp] lemma mulShift_one (ψ : AddChar R M) : mulShift ψ 1 = ψ := by ext; rw [mulShift_apply, one_mul] lemma mulShift_unit_eq_one_iff (ψ : AddChar R M) {u : R} (hu : IsUnit u) : ψ.mulShift u = 1 ↔ ψ = 1 := by refine ⟨fun h ↦ ?_, ?_⟩ · ext1 y rw [show y = u * (hu.unit⁻¹ * y) by rw [← mul_assoc, IsUnit.mul_val_inv, one_mul]] simpa only [mulShift_apply] using DFunLike.ext_iff.mp h (hu.unit⁻¹ * y) · rintro rfl ext1 y rw [mulShift_apply, one_apply, one_apply] end Ring end AddChar
Algebra\Group\Aut.lean
/- Copyright (c) 2018 Johannes Hölzl. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Johannes Hölzl, Callum Sutton, Yury Kudryashov -/ import Mathlib.Algebra.GroupWithZero.Action.Defs import Mathlib.GroupTheory.Perm.Basic /-! # Multiplicative and additive group automorphisms This file defines the automorphism group structure on `AddAut R := AddEquiv R R` and `MulAut R := MulEquiv R R`. ## Implementation notes The definition of multiplication in the automorphism groups agrees with function composition, multiplication in `Equiv.Perm`, and multiplication in `CategoryTheory.End`, but not with `CategoryTheory.comp`. This file is kept separate from `Data/Equiv/MulAdd` so that `GroupTheory.Perm` is free to use equivalences (and other files that use them) before the group structure is defined. ## Tags MulAut, AddAut -/ -- TODO after #13161 -- assert_not_exists MonoidWithZero assert_not_exists Ring variable {A : Type*} {M : Type*} {G : Type*} /-- The group of multiplicative automorphisms. -/ @[reducible, to_additive "The group of additive automorphisms."] def MulAut (M : Type*) [Mul M] := M ≃* M -- Note that `(attr := reducible)` in `to_additive` currently doesn't work, -- so we add the reducible attribute manually. attribute [reducible] AddAut namespace MulAut variable (M) [Mul M] /-- The group operation on multiplicative automorphisms is defined by `g h => MulEquiv.trans h g`. This means that multiplication agrees with composition, `(g*h)(x) = g (h x)`. -/ instance : Group (MulAut M) where mul g h := MulEquiv.trans h g one := MulEquiv.refl _ inv := MulEquiv.symm mul_assoc _ _ _ := rfl one_mul _ := rfl mul_one _ := rfl mul_left_inv := MulEquiv.self_trans_symm instance : Inhabited (MulAut M) := ⟨1⟩ @[simp] theorem coe_mul (e₁ e₂ : MulAut M) : ⇑(e₁ * e₂) = e₁ ∘ e₂ := rfl @[simp] theorem coe_one : ⇑(1 : MulAut M) = id := rfl theorem mul_def (e₁ e₂ : MulAut M) : e₁ * e₂ = e₂.trans e₁ := rfl theorem one_def : (1 : MulAut M) = MulEquiv.refl _ := rfl theorem inv_def (e₁ : MulAut M) : e₁⁻¹ = e₁.symm := rfl @[simp] theorem mul_apply (e₁ e₂ : MulAut M) (m : M) : (e₁ * e₂) m = e₁ (e₂ m) := rfl @[simp] theorem one_apply (m : M) : (1 : MulAut M) m = m := rfl @[simp] theorem apply_inv_self (e : MulAut M) (m : M) : e (e⁻¹ m) = m := MulEquiv.apply_symm_apply _ _ @[simp] theorem inv_apply_self (e : MulAut M) (m : M) : e⁻¹ (e m) = m := MulEquiv.apply_symm_apply _ _ /-- Monoid hom from the group of multiplicative automorphisms to the group of permutations. -/ def toPerm : MulAut M →* Equiv.Perm M where toFun := MulEquiv.toEquiv map_one' := rfl map_mul' _ _ := rfl /-- The tautological action by `MulAut M` on `M`. This generalizes `Function.End.applyMulAction`. -/ instance applyMulDistribMulAction {M} [Monoid M] : MulDistribMulAction (MulAut M) M where smul := (· <| ·) one_smul _ := rfl mul_smul _ _ _ := rfl smul_one := MulEquiv.map_one smul_mul := MulEquiv.map_mul @[simp] protected theorem smul_def {M} [Monoid M] (f : MulAut M) (a : M) : f • a = f a := rfl /-- `MulAut.applyDistribMulAction` is faithful. -/ instance apply_faithfulSMul {M} [Monoid M] : FaithfulSMul (MulAut M) M := ⟨ fun h => MulEquiv.ext h ⟩ /-- Group conjugation, `MulAut.conj g h = g * h * g⁻¹`, as a monoid homomorphism mapping multiplication in `G` into multiplication in the automorphism group `MulAut G`. See also the type `ConjAct G` for any group `G`, which has a `MulAction (ConjAct G) G` instance where `conj G` acts on `G` by conjugation. -/ def conj [Group G] : G →* MulAut G where toFun g := { toFun := fun h => g * h * g⁻¹ invFun := fun h => g⁻¹ * h * g left_inv := fun _ => by simp only [mul_assoc, inv_mul_cancel_left, mul_left_inv, mul_one] right_inv := fun _ => by simp only [mul_assoc, mul_inv_cancel_left, mul_right_inv, mul_one] map_mul' := by simp only [mul_assoc, inv_mul_cancel_left, forall_const] } map_mul' g₁ g₂ := by ext h show g₁ * g₂ * h * (g₁ * g₂)⁻¹ = g₁ * (g₂ * h * g₂⁻¹) * g₁⁻¹ simp only [mul_assoc, mul_inv_rev] map_one' := by ext; simp only [one_mul, inv_one, mul_one, one_apply]; rfl @[simp] theorem conj_apply [Group G] (g h : G) : conj g h = g * h * g⁻¹ := rfl @[simp] theorem conj_symm_apply [Group G] (g h : G) : (conj g).symm h = g⁻¹ * h * g := rfl @[simp] theorem conj_inv_apply [Group G] (g h : G) : (conj g)⁻¹ h = g⁻¹ * h * g := rfl end MulAut namespace AddAut variable (A) [Add A] /-- The group operation on additive automorphisms is defined by `g h => AddEquiv.trans h g`. This means that multiplication agrees with composition, `(g*h)(x) = g (h x)`. -/ instance group : Group (AddAut A) where mul g h := AddEquiv.trans h g one := AddEquiv.refl _ inv := AddEquiv.symm mul_assoc _ _ _ := rfl one_mul _ := rfl mul_one _ := rfl mul_left_inv := AddEquiv.self_trans_symm instance : Inhabited (AddAut A) := ⟨1⟩ @[simp] theorem coe_mul (e₁ e₂ : AddAut A) : ⇑(e₁ * e₂) = e₁ ∘ e₂ := rfl @[simp] theorem coe_one : ⇑(1 : AddAut A) = id := rfl theorem mul_def (e₁ e₂ : AddAut A) : e₁ * e₂ = e₂.trans e₁ := rfl theorem one_def : (1 : AddAut A) = AddEquiv.refl _ := rfl theorem inv_def (e₁ : AddAut A) : e₁⁻¹ = e₁.symm := rfl @[simp] theorem mul_apply (e₁ e₂ : AddAut A) (a : A) : (e₁ * e₂) a = e₁ (e₂ a) := rfl @[simp] theorem one_apply (a : A) : (1 : AddAut A) a = a := rfl @[simp] theorem apply_inv_self (e : AddAut A) (a : A) : e⁻¹ (e a) = a := AddEquiv.apply_symm_apply _ _ @[simp] theorem inv_apply_self (e : AddAut A) (a : A) : e (e⁻¹ a) = a := AddEquiv.apply_symm_apply _ _ /-- Monoid hom from the group of multiplicative automorphisms to the group of permutations. -/ def toPerm : AddAut A →* Equiv.Perm A where toFun := AddEquiv.toEquiv map_one' := rfl map_mul' _ _ := rfl /-- The tautological action by `AddAut A` on `A`. This generalizes `Function.End.applyMulAction`. -/ instance applyDistribMulAction {A} [AddMonoid A] : DistribMulAction (AddAut A) A where smul := (· <| ·) smul_zero := AddEquiv.map_zero smul_add := AddEquiv.map_add one_smul _ := rfl mul_smul _ _ _ := rfl @[simp] protected theorem smul_def {A} [AddMonoid A] (f : AddAut A) (a : A) : f • a = f a := rfl /-- `AddAut.applyDistribMulAction` is faithful. -/ instance apply_faithfulSMul {A} [AddMonoid A] : FaithfulSMul (AddAut A) A := ⟨fun h => AddEquiv.ext h⟩ /-- Additive group conjugation, `AddAut.conj g h = g + h - g`, as an additive monoid homomorphism mapping addition in `G` into multiplication in the automorphism group `AddAut G` (written additively in order to define the map). -/ def conj [AddGroup G] : G →+ Additive (AddAut G) where toFun g := @Additive.ofMul (AddAut G) { toFun := fun h => g + h + -g -- this definition is chosen to match `MulAut.conj` invFun := fun h => -g + h + g left_inv := fun _ => by simp only [add_assoc, neg_add_cancel_left, add_left_neg, add_zero] right_inv := fun _ => by simp only [add_assoc, add_neg_cancel_left, add_right_neg, add_zero] map_add' := by simp only [add_assoc, neg_add_cancel_left, forall_const] } map_add' g₁ g₂ := by apply Additive.toMul.injective; ext h show g₁ + g₂ + h + -(g₁ + g₂) = g₁ + (g₂ + h + -g₂) + -g₁ simp only [add_assoc, neg_add_rev] map_zero' := by apply Additive.toMul.injective; ext simp only [zero_add, neg_zero, add_zero, toMul_ofMul, toMul_zero, one_apply] rfl @[simp] theorem conj_apply [AddGroup G] (g h : G) : conj g h = g + h + -g := rfl @[simp] theorem conj_symm_apply [AddGroup G] (g h : G) : (conj g).symm h = -g + h + g := rfl -- Porting note: the exact translation of this mathlib3 lemma would be`(-conj g) h = -g + h + g`, -- but this no longer pass the simp_nf linter, as the LHS simplifies by `toMul_neg` to -- `(Additive.toMul (conj g))⁻¹`. @[simp] theorem conj_inv_apply [AddGroup G] (g h : G) : (Additive.toMul (conj g))⁻¹ h = -g + h + g := rfl end AddAut
Algebra\Group\Basic.lean
/- Copyright (c) 2014 Jeremy Avigad. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Jeremy Avigad, Leonardo de Moura, Simon Hudon, Mario Carneiro -/ import Aesop import Mathlib.Algebra.Group.Defs import Mathlib.Data.Nat.Defs import Mathlib.Data.Int.Defs import Mathlib.Logic.Function.Basic import Mathlib.Tactic.Cases import Mathlib.Tactic.SimpRw import Mathlib.Tactic.SplitIfs /-! # Basic lemmas about semigroups, monoids, and groups This file lists various basic lemmas about semigroups, monoids, and groups. Most proofs are one-liners from the corresponding axioms. For the definitions of semigroups, monoids and groups, see `Algebra/Group/Defs.lean`. -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered open Function universe u variable {α β G M : Type*} section ite variable [Pow α β] @[to_additive (attr := simp) dite_smul] lemma pow_dite (p : Prop) [Decidable p] (a : α) (b : p → β) (c : ¬ p → β) : a ^ (if h : p then b h else c h) = if h : p then a ^ b h else a ^ c h := by split_ifs <;> rfl @[to_additive (attr := simp) smul_dite] lemma dite_pow (p : Prop) [Decidable p] (a : p → α) (b : ¬ p → α) (c : β) : (if h : p then a h else b h) ^ c = if h : p then a h ^ c else b h ^ c := by split_ifs <;> rfl @[to_additive (attr := simp) ite_smul] lemma pow_ite (p : Prop) [Decidable p] (a : α) (b c : β) : a ^ (if p then b else c) = if p then a ^ b else a ^ c := pow_dite _ _ _ _ @[to_additive (attr := simp) smul_ite] lemma ite_pow (p : Prop) [Decidable p] (a b : α) (c : β) : (if p then a else b) ^ c = if p then a ^ c else b ^ c := dite_pow _ _ _ _ set_option linter.existingAttributeWarning false in attribute [to_additive (attr := simp)] dite_smul smul_dite ite_smul smul_ite end ite section IsLeftCancelMul variable [Mul G] [IsLeftCancelMul G] @[to_additive] theorem mul_right_injective (a : G) : Injective (a * ·) := fun _ _ ↦ mul_left_cancel @[to_additive (attr := simp)] theorem mul_right_inj (a : G) {b c : G} : a * b = a * c ↔ b = c := (mul_right_injective a).eq_iff @[to_additive] theorem mul_ne_mul_right (a : G) {b c : G} : a * b ≠ a * c ↔ b ≠ c := (mul_right_injective a).ne_iff end IsLeftCancelMul section IsRightCancelMul variable [Mul G] [IsRightCancelMul G] @[to_additive] theorem mul_left_injective (a : G) : Function.Injective (· * a) := fun _ _ ↦ mul_right_cancel @[to_additive (attr := simp)] theorem mul_left_inj (a : G) {b c : G} : b * a = c * a ↔ b = c := (mul_left_injective a).eq_iff @[to_additive] theorem mul_ne_mul_left (a : G) {b c : G} : b * a ≠ c * a ↔ b ≠ c := (mul_left_injective a).ne_iff end IsRightCancelMul section Semigroup variable [Semigroup α] @[to_additive] instance Semigroup.to_isAssociative : Std.Associative (α := α) (· * ·) := ⟨mul_assoc⟩ /-- Composing two multiplications on the left by `y` then `x` is equal to a multiplication on the left by `x * y`. -/ @[to_additive (attr := simp) "Composing two additions on the left by `y` then `x` is equal to an addition on the left by `x + y`."] theorem comp_mul_left (x y : α) : (x * ·) ∘ (y * ·) = (x * y * ·) := by ext z simp [mul_assoc] /-- Composing two multiplications on the right by `y` and `x` is equal to a multiplication on the right by `y * x`. -/ @[to_additive (attr := simp) "Composing two additions on the right by `y` and `x` is equal to an addition on the right by `y + x`."] theorem comp_mul_right (x y : α) : (· * x) ∘ (· * y) = (· * (y * x)) := by ext z simp [mul_assoc] end Semigroup @[to_additive] instance CommMagma.to_isCommutative [CommMagma G] : Std.Commutative (α := G) (· * ·) := ⟨mul_comm⟩ section MulOneClass variable {M : Type u} [MulOneClass M] @[to_additive] theorem ite_mul_one {P : Prop} [Decidable P] {a b : M} : ite P (a * b) 1 = ite P a 1 * ite P b 1 := by by_cases h : P <;> simp [h] @[to_additive] theorem ite_one_mul {P : Prop} [Decidable P] {a b : M} : ite P 1 (a * b) = ite P 1 a * ite P 1 b := by by_cases h : P <;> simp [h] @[to_additive] theorem eq_one_iff_eq_one_of_mul_eq_one {a b : M} (h : a * b = 1) : a = 1 ↔ b = 1 := by constructor <;> (rintro rfl; simpa using h) @[to_additive] theorem one_mul_eq_id : ((1 : M) * ·) = id := funext one_mul @[to_additive] theorem mul_one_eq_id : (· * (1 : M)) = id := funext mul_one end MulOneClass section CommSemigroup variable [CommSemigroup G] @[to_additive] theorem mul_left_comm : ∀ a b c : G, a * (b * c) = b * (a * c) := left_comm Mul.mul mul_comm mul_assoc @[to_additive] theorem mul_right_comm : ∀ a b c : G, a * b * c = a * c * b := right_comm Mul.mul mul_comm mul_assoc @[to_additive] theorem mul_mul_mul_comm (a b c d : G) : a * b * (c * d) = a * c * (b * d) := by simp only [mul_left_comm, mul_assoc] @[to_additive] theorem mul_rotate (a b c : G) : a * b * c = b * c * a := by simp only [mul_left_comm, mul_comm] @[to_additive] theorem mul_rotate' (a b c : G) : a * (b * c) = b * (c * a) := by simp only [mul_left_comm, mul_comm] end CommSemigroup attribute [local simp] mul_assoc sub_eq_add_neg section Monoid variable [Monoid M] {a b c : M} {m n : ℕ} @[to_additive boole_nsmul] lemma pow_boole (P : Prop) [Decidable P] (a : M) : (a ^ if P then 1 else 0) = if P then a else 1 := by simp only [pow_ite, pow_one, pow_zero] @[to_additive nsmul_add_sub_nsmul] lemma pow_mul_pow_sub (a : M) (h : m ≤ n) : a ^ m * a ^ (n - m) = a ^ n := by rw [← pow_add, Nat.add_comm, Nat.sub_add_cancel h] @[to_additive sub_nsmul_nsmul_add] lemma pow_sub_mul_pow (a : M) (h : m ≤ n) : a ^ (n - m) * a ^ m = a ^ n := by rw [← pow_add, Nat.sub_add_cancel h] @[to_additive sub_one_nsmul_add] lemma mul_pow_sub_one (hn : n ≠ 0) (a : M) : a * a ^ (n - 1) = a ^ n := by rw [← pow_succ', Nat.sub_add_cancel $ Nat.one_le_iff_ne_zero.2 hn] @[to_additive add_sub_one_nsmul] lemma pow_sub_one_mul (hn : n ≠ 0) (a : M) : a ^ (n - 1) * a = a ^ n := by rw [← pow_succ, Nat.sub_add_cancel $ Nat.one_le_iff_ne_zero.2 hn] /-- If `x ^ n = 1`, then `x ^ m` is the same as `x ^ (m % n)` -/ @[to_additive nsmul_eq_mod_nsmul "If `n • x = 0`, then `m • x` is the same as `(m % n) • x`"] lemma pow_eq_pow_mod (m : ℕ) (ha : a ^ n = 1) : a ^ m = a ^ (m % n) := by calc a ^ m = a ^ (m % n + n * (m / n)) := by rw [Nat.mod_add_div] _ = a ^ (m % n) := by simp [pow_add, pow_mul, ha] @[to_additive] lemma pow_mul_pow_eq_one : ∀ n, a * b = 1 → a ^ n * b ^ n = 1 | 0, _ => by simp | n + 1, h => calc a ^ n.succ * b ^ n.succ = a ^ n * a * (b * b ^ n) := by rw [pow_succ, pow_succ'] _ = a ^ n * (a * b) * b ^ n := by simp only [mul_assoc] _ = 1 := by simp [h, pow_mul_pow_eq_one] end Monoid section CommMonoid variable [CommMonoid M] {x y z : M} @[to_additive] theorem inv_unique (hy : x * y = 1) (hz : x * z = 1) : y = z := left_inv_eq_right_inv (Trans.trans (mul_comm _ _) hy) hz @[to_additive nsmul_add] lemma mul_pow (a b : M) : ∀ n, (a * b) ^ n = a ^ n * b ^ n | 0 => by rw [pow_zero, pow_zero, pow_zero, one_mul] | n + 1 => by rw [pow_succ', pow_succ', pow_succ', mul_pow, mul_mul_mul_comm] end CommMonoid section LeftCancelMonoid variable {M : Type u} [LeftCancelMonoid M] {a b : M} @[to_additive (attr := simp)] theorem mul_right_eq_self : a * b = a ↔ b = 1 := calc a * b = a ↔ a * b = a * 1 := by rw [mul_one] _ ↔ b = 1 := mul_left_cancel_iff @[to_additive (attr := simp)] theorem self_eq_mul_right : a = a * b ↔ b = 1 := eq_comm.trans mul_right_eq_self @[to_additive] theorem mul_right_ne_self : a * b ≠ a ↔ b ≠ 1 := mul_right_eq_self.not @[to_additive] theorem self_ne_mul_right : a ≠ a * b ↔ b ≠ 1 := self_eq_mul_right.not end LeftCancelMonoid section RightCancelMonoid variable {M : Type u} [RightCancelMonoid M] {a b : M} @[to_additive (attr := simp)] theorem mul_left_eq_self : a * b = b ↔ a = 1 := calc a * b = b ↔ a * b = 1 * b := by rw [one_mul] _ ↔ a = 1 := mul_right_cancel_iff @[to_additive (attr := simp)] theorem self_eq_mul_left : b = a * b ↔ a = 1 := eq_comm.trans mul_left_eq_self @[to_additive] theorem mul_left_ne_self : a * b ≠ b ↔ a ≠ 1 := mul_left_eq_self.not @[to_additive] theorem self_ne_mul_left : b ≠ a * b ↔ a ≠ 1 := self_eq_mul_left.not end RightCancelMonoid section CancelCommMonoid variable [CancelCommMonoid α] {a b c d : α} @[to_additive] lemma eq_iff_eq_of_mul_eq_mul (h : a * b = c * d) : a = c ↔ b = d := by aesop @[to_additive] lemma ne_iff_ne_of_mul_eq_mul (h : a * b = c * d) : a ≠ c ↔ b ≠ d := by aesop end CancelCommMonoid section InvolutiveInv variable [InvolutiveInv G] {a b : G} @[to_additive (attr := simp)] theorem inv_involutive : Function.Involutive (Inv.inv : G → G) := inv_inv @[to_additive (attr := simp)] theorem inv_surjective : Function.Surjective (Inv.inv : G → G) := inv_involutive.surjective @[to_additive] theorem inv_injective : Function.Injective (Inv.inv : G → G) := inv_involutive.injective @[to_additive (attr := simp)] theorem inv_inj : a⁻¹ = b⁻¹ ↔ a = b := inv_injective.eq_iff @[to_additive] theorem inv_eq_iff_eq_inv : a⁻¹ = b ↔ a = b⁻¹ := ⟨fun h => h ▸ (inv_inv a).symm, fun h => h.symm ▸ inv_inv b⟩ variable (G) @[to_additive] theorem inv_comp_inv : Inv.inv ∘ Inv.inv = @id G := inv_involutive.comp_self @[to_additive] theorem leftInverse_inv : LeftInverse (fun a : G ↦ a⁻¹) fun a ↦ a⁻¹ := inv_inv @[to_additive] theorem rightInverse_inv : RightInverse (fun a : G ↦ a⁻¹) fun a ↦ a⁻¹ := inv_inv end InvolutiveInv section DivInvMonoid variable [DivInvMonoid G] {a b c : G} @[to_additive, field_simps] -- The attributes are out of order on purpose theorem inv_eq_one_div (x : G) : x⁻¹ = 1 / x := by rw [div_eq_mul_inv, one_mul] @[to_additive] theorem mul_one_div (x y : G) : x * (1 / y) = x / y := by rw [div_eq_mul_inv, one_mul, div_eq_mul_inv] @[to_additive] theorem mul_div_assoc (a b c : G) : a * b / c = a * (b / c) := by rw [div_eq_mul_inv, div_eq_mul_inv, mul_assoc _ _ _] @[to_additive, field_simps] -- The attributes are out of order on purpose theorem mul_div_assoc' (a b c : G) : a * (b / c) = a * b / c := (mul_div_assoc _ _ _).symm @[to_additive (attr := simp)] theorem one_div (a : G) : 1 / a = a⁻¹ := (inv_eq_one_div a).symm @[to_additive] theorem mul_div (a b c : G) : a * (b / c) = a * b / c := by simp only [mul_assoc, div_eq_mul_inv] @[to_additive] theorem div_eq_mul_one_div (a b : G) : a / b = a * (1 / b) := by rw [div_eq_mul_inv, one_div] end DivInvMonoid section DivInvOneMonoid variable [DivInvOneMonoid G] @[to_additive (attr := simp)] theorem div_one (a : G) : a / 1 = a := by simp [div_eq_mul_inv] @[to_additive] theorem one_div_one : (1 : G) / 1 = 1 := div_one _ end DivInvOneMonoid section DivisionMonoid variable [DivisionMonoid α] {a b c d : α} attribute [local simp] mul_assoc div_eq_mul_inv @[to_additive] theorem eq_inv_of_mul_eq_one_right (h : a * b = 1) : b = a⁻¹ := (inv_eq_of_mul_eq_one_right h).symm @[to_additive] theorem eq_one_div_of_mul_eq_one_left (h : b * a = 1) : b = 1 / a := by rw [eq_inv_of_mul_eq_one_left h, one_div] @[to_additive] theorem eq_one_div_of_mul_eq_one_right (h : a * b = 1) : b = 1 / a := by rw [eq_inv_of_mul_eq_one_right h, one_div] @[to_additive] theorem eq_of_div_eq_one (h : a / b = 1) : a = b := inv_injective <| inv_eq_of_mul_eq_one_right <| by rwa [← div_eq_mul_inv] lemma eq_of_inv_mul_eq_one (h : a⁻¹ * b = 1) : a = b := by simpa using eq_inv_of_mul_eq_one_left h lemma eq_of_mul_inv_eq_one (h : a * b⁻¹ = 1) : a = b := by simpa using eq_inv_of_mul_eq_one_left h @[to_additive] theorem div_ne_one_of_ne : a ≠ b → a / b ≠ 1 := mt eq_of_div_eq_one variable (a b c) @[to_additive] theorem one_div_mul_one_div_rev : 1 / a * (1 / b) = 1 / (b * a) := by simp @[to_additive] theorem inv_div_left : a⁻¹ / b = (b * a)⁻¹ := by simp @[to_additive (attr := simp)] theorem inv_div : (a / b)⁻¹ = b / a := by simp @[to_additive] theorem one_div_div : 1 / (a / b) = b / a := by simp @[to_additive] theorem one_div_one_div : 1 / (1 / a) = a := by simp @[to_additive] theorem div_eq_div_iff_comm : a / b = c / d ↔ b / a = d / c := inv_inj.symm.trans <| by simp only [inv_div] @[to_additive SubtractionMonoid.toSubNegZeroMonoid] instance (priority := 100) DivisionMonoid.toDivInvOneMonoid : DivInvOneMonoid α := { DivisionMonoid.toDivInvMonoid with inv_one := by simpa only [one_div, inv_inv] using (inv_div (1 : α) 1).symm } @[to_additive (attr := simp)] lemma inv_pow (a : α) : ∀ n : ℕ, a⁻¹ ^ n = (a ^ n)⁻¹ | 0 => by rw [pow_zero, pow_zero, inv_one] | n + 1 => by rw [pow_succ', pow_succ, inv_pow _ n, mul_inv_rev] -- the attributes are intentionally out of order. `smul_zero` proves `zsmul_zero`. @[to_additive zsmul_zero, simp] lemma one_zpow : ∀ n : ℤ, (1 : α) ^ n = 1 | (n : ℕ) => by rw [zpow_natCast, one_pow] | .negSucc n => by rw [zpow_negSucc, one_pow, inv_one] @[to_additive (attr := simp) neg_zsmul] lemma zpow_neg (a : α) : ∀ n : ℤ, a ^ (-n) = (a ^ n)⁻¹ | (n + 1 : ℕ) => DivInvMonoid.zpow_neg' _ _ | 0 => by change a ^ (0 : ℤ) = (a ^ (0 : ℤ))⁻¹ simp | Int.negSucc n => by rw [zpow_negSucc, inv_inv, ← zpow_natCast] rfl @[to_additive neg_one_zsmul_add] lemma mul_zpow_neg_one (a b : α) : (a * b) ^ (-1 : ℤ) = b ^ (-1 : ℤ) * a ^ (-1 : ℤ) := by simp only [zpow_neg, zpow_one, mul_inv_rev] @[to_additive zsmul_neg] lemma inv_zpow (a : α) : ∀ n : ℤ, a⁻¹ ^ n = (a ^ n)⁻¹ | (n : ℕ) => by rw [zpow_natCast, zpow_natCast, inv_pow] | .negSucc n => by rw [zpow_negSucc, zpow_negSucc, inv_pow] @[to_additive (attr := simp) zsmul_neg'] lemma inv_zpow' (a : α) (n : ℤ) : a⁻¹ ^ n = a ^ (-n) := by rw [inv_zpow, zpow_neg] @[to_additive nsmul_zero_sub] lemma one_div_pow (a : α) (n : ℕ) : (1 / a) ^ n = 1 / a ^ n := by simp only [one_div, inv_pow] @[to_additive zsmul_zero_sub] lemma one_div_zpow (a : α) (n : ℤ) : (1 / a) ^ n = 1 / a ^ n := by simp only [one_div, inv_zpow] variable {a b c} @[to_additive (attr := simp)] theorem inv_eq_one : a⁻¹ = 1 ↔ a = 1 := inv_injective.eq_iff' inv_one @[to_additive (attr := simp)] theorem one_eq_inv : 1 = a⁻¹ ↔ a = 1 := eq_comm.trans inv_eq_one @[to_additive] theorem inv_ne_one : a⁻¹ ≠ 1 ↔ a ≠ 1 := inv_eq_one.not @[to_additive] theorem eq_of_one_div_eq_one_div (h : 1 / a = 1 / b) : a = b := by rw [← one_div_one_div a, h, one_div_one_div] -- Note that `mul_zsmul` and `zpow_mul` have the primes swapped -- when additivised since their argument order, -- and therefore the more "natural" choice of lemma, is reversed. @[to_additive mul_zsmul'] lemma zpow_mul (a : α) : ∀ m n : ℤ, a ^ (m * n) = (a ^ m) ^ n | (m : ℕ), (n : ℕ) => by rw [zpow_natCast, zpow_natCast, ← pow_mul, ← zpow_natCast] rfl | (m : ℕ), .negSucc n => by rw [zpow_natCast, zpow_negSucc, ← pow_mul, Int.ofNat_mul_negSucc, zpow_neg, inv_inj, ← zpow_natCast] | .negSucc m, (n : ℕ) => by rw [zpow_natCast, zpow_negSucc, ← inv_pow, ← pow_mul, Int.negSucc_mul_ofNat, zpow_neg, inv_pow, inv_inj, ← zpow_natCast] | .negSucc m, .negSucc n => by rw [zpow_negSucc, zpow_negSucc, Int.negSucc_mul_negSucc, inv_pow, inv_inv, ← pow_mul, ← zpow_natCast] rfl @[to_additive mul_zsmul] lemma zpow_mul' (a : α) (m n : ℤ) : a ^ (m * n) = (a ^ n) ^ m := by rw [Int.mul_comm, zpow_mul] variable (a b c) @[to_additive, field_simps] -- The attributes are out of order on purpose theorem div_div_eq_mul_div : a / (b / c) = a * c / b := by simp @[to_additive (attr := simp)] theorem div_inv_eq_mul : a / b⁻¹ = a * b := by simp @[to_additive] theorem div_mul_eq_div_div_swap : a / (b * c) = a / c / b := by simp only [mul_assoc, mul_inv_rev, div_eq_mul_inv] end DivisionMonoid section DivisionCommMonoid variable [DivisionCommMonoid α] (a b c d : α) attribute [local simp] mul_assoc mul_comm mul_left_comm div_eq_mul_inv @[to_additive neg_add] theorem mul_inv : (a * b)⁻¹ = a⁻¹ * b⁻¹ := by simp @[to_additive] theorem inv_div' : (a / b)⁻¹ = a⁻¹ / b⁻¹ := by simp @[to_additive] theorem div_eq_inv_mul : a / b = b⁻¹ * a := by simp @[to_additive] theorem inv_mul_eq_div : a⁻¹ * b = b / a := by simp @[to_additive] theorem inv_mul' : (a * b)⁻¹ = a⁻¹ / b := by simp @[to_additive] theorem inv_div_inv : a⁻¹ / b⁻¹ = b / a := by simp @[to_additive] theorem inv_inv_div_inv : (a⁻¹ / b⁻¹)⁻¹ = a / b := by simp @[to_additive] theorem one_div_mul_one_div : 1 / a * (1 / b) = 1 / (a * b) := by simp @[to_additive] theorem div_right_comm : a / b / c = a / c / b := by simp @[to_additive, field_simps] theorem div_div : a / b / c = a / (b * c) := by simp @[to_additive] theorem div_mul : a / b * c = a / (b / c) := by simp @[to_additive] theorem mul_div_left_comm : a * (b / c) = b * (a / c) := by simp @[to_additive] theorem mul_div_right_comm : a * b / c = a / c * b := by simp @[to_additive] theorem div_mul_eq_div_div : a / (b * c) = a / b / c := by simp @[to_additive, field_simps] theorem div_mul_eq_mul_div : a / b * c = a * c / b := by simp @[to_additive] theorem one_div_mul_eq_div : 1 / a * b = b / a := by simp @[to_additive] theorem mul_comm_div : a / b * c = a * (c / b) := by simp @[to_additive] theorem div_mul_comm : a / b * c = c / b * a := by simp @[to_additive] theorem div_mul_eq_div_mul_one_div : a / (b * c) = a / b * (1 / c) := by simp @[to_additive] theorem div_div_div_eq : a / b / (c / d) = a * d / (b * c) := by simp @[to_additive] theorem div_div_div_comm : a / b / (c / d) = a / c / (b / d) := by simp @[to_additive] theorem div_mul_div_comm : a / b * (c / d) = a * c / (b * d) := by simp @[to_additive] theorem mul_div_mul_comm : a * b / (c * d) = a / c * (b / d) := by simp @[to_additive zsmul_add] lemma mul_zpow : ∀ n : ℤ, (a * b) ^ n = a ^ n * b ^ n | (n : ℕ) => by simp_rw [zpow_natCast, mul_pow] | .negSucc n => by simp_rw [zpow_negSucc, ← inv_pow, mul_inv, mul_pow] @[to_additive (attr := simp) nsmul_sub] lemma div_pow (a b : α) (n : ℕ) : (a / b) ^ n = a ^ n / b ^ n := by simp only [div_eq_mul_inv, mul_pow, inv_pow] @[to_additive (attr := simp) zsmul_sub] lemma div_zpow (a b : α) (n : ℤ) : (a / b) ^ n = a ^ n / b ^ n := by simp only [div_eq_mul_inv, mul_zpow, inv_zpow] end DivisionCommMonoid section Group variable [Group G] {a b c d : G} {n : ℤ} @[to_additive (attr := simp)] theorem div_eq_inv_self : a / b = b⁻¹ ↔ a = 1 := by rw [div_eq_mul_inv, mul_left_eq_self] @[to_additive] theorem mul_left_surjective (a : G) : Surjective (a * ·) := fun x ↦ ⟨a⁻¹ * x, mul_inv_cancel_left a x⟩ @[to_additive] theorem mul_right_surjective (a : G) : Function.Surjective fun x ↦ x * a := fun x ↦ ⟨x * a⁻¹, inv_mul_cancel_right x a⟩ @[to_additive] theorem eq_mul_inv_of_mul_eq (h : a * c = b) : a = b * c⁻¹ := by simp [h.symm] @[to_additive] theorem eq_inv_mul_of_mul_eq (h : b * a = c) : a = b⁻¹ * c := by simp [h.symm] @[to_additive] theorem inv_mul_eq_of_eq_mul (h : b = a * c) : a⁻¹ * b = c := by simp [h] @[to_additive] theorem mul_inv_eq_of_eq_mul (h : a = c * b) : a * b⁻¹ = c := by simp [h] @[to_additive] theorem eq_mul_of_mul_inv_eq (h : a * c⁻¹ = b) : a = b * c := by simp [h.symm] @[to_additive] theorem eq_mul_of_inv_mul_eq (h : b⁻¹ * a = c) : a = b * c := by simp [h.symm, mul_inv_cancel_left] @[to_additive] theorem mul_eq_of_eq_inv_mul (h : b = a⁻¹ * c) : a * b = c := by rw [h, mul_inv_cancel_left] @[to_additive] theorem mul_eq_of_eq_mul_inv (h : a = c * b⁻¹) : a * b = c := by simp [h] @[to_additive] theorem mul_eq_one_iff_eq_inv : a * b = 1 ↔ a = b⁻¹ := ⟨eq_inv_of_mul_eq_one_left, fun h ↦ by rw [h, mul_left_inv]⟩ @[to_additive] theorem mul_eq_one_iff_inv_eq : a * b = 1 ↔ a⁻¹ = b := by rw [mul_eq_one_iff_eq_inv, inv_eq_iff_eq_inv] @[to_additive] theorem eq_inv_iff_mul_eq_one : a = b⁻¹ ↔ a * b = 1 := mul_eq_one_iff_eq_inv.symm @[to_additive] theorem inv_eq_iff_mul_eq_one : a⁻¹ = b ↔ a * b = 1 := mul_eq_one_iff_inv_eq.symm @[to_additive] theorem eq_mul_inv_iff_mul_eq : a = b * c⁻¹ ↔ a * c = b := ⟨fun h ↦ by rw [h, inv_mul_cancel_right], fun h ↦ by rw [← h, mul_inv_cancel_right]⟩ @[to_additive] theorem eq_inv_mul_iff_mul_eq : a = b⁻¹ * c ↔ b * a = c := ⟨fun h ↦ by rw [h, mul_inv_cancel_left], fun h ↦ by rw [← h, inv_mul_cancel_left]⟩ @[to_additive] theorem inv_mul_eq_iff_eq_mul : a⁻¹ * b = c ↔ b = a * c := ⟨fun h ↦ by rw [← h, mul_inv_cancel_left], fun h ↦ by rw [h, inv_mul_cancel_left]⟩ @[to_additive] theorem mul_inv_eq_iff_eq_mul : a * b⁻¹ = c ↔ a = c * b := ⟨fun h ↦ by rw [← h, inv_mul_cancel_right], fun h ↦ by rw [h, mul_inv_cancel_right]⟩ @[to_additive] theorem mul_inv_eq_one : a * b⁻¹ = 1 ↔ a = b := by rw [mul_eq_one_iff_eq_inv, inv_inv] @[to_additive] theorem inv_mul_eq_one : a⁻¹ * b = 1 ↔ a = b := by rw [mul_eq_one_iff_eq_inv, inv_inj] @[to_additive (attr := simp)] theorem conj_eq_one_iff : a * b * a⁻¹ = 1 ↔ b = 1 := by rw [mul_inv_eq_one, mul_right_eq_self] @[to_additive] theorem div_left_injective : Function.Injective fun a ↦ a / b := by -- FIXME this could be by `simpa`, but it fails. This is probably a bug in `simpa`. simp only [div_eq_mul_inv] exact fun a a' h ↦ mul_left_injective b⁻¹ h @[to_additive] theorem div_right_injective : Function.Injective fun a ↦ b / a := by -- FIXME see above simp only [div_eq_mul_inv] exact fun a a' h ↦ inv_injective (mul_right_injective b h) @[to_additive (attr := simp)] theorem div_mul_cancel (a b : G) : a / b * b = a := by rw [div_eq_mul_inv, inv_mul_cancel_right a b] @[to_additive (attr := simp) sub_self] theorem div_self' (a : G) : a / a = 1 := by rw [div_eq_mul_inv, mul_right_inv a] @[to_additive (attr := simp)] theorem mul_div_cancel_right (a b : G) : a * b / b = a := by rw [div_eq_mul_inv, mul_inv_cancel_right a b] @[to_additive (attr := simp)] lemma div_mul_cancel_right (a b : G) : a / (b * a) = b⁻¹ := by rw [← inv_div, mul_div_cancel_right] @[to_additive (attr := simp)] theorem mul_div_mul_right_eq_div (a b c : G) : a * c / (b * c) = a / b := by rw [div_mul_eq_div_div_swap]; simp only [mul_left_inj, eq_self_iff_true, mul_div_cancel_right] @[to_additive eq_sub_of_add_eq] theorem eq_div_of_mul_eq' (h : a * c = b) : a = b / c := by simp [← h] @[to_additive sub_eq_of_eq_add] theorem div_eq_of_eq_mul'' (h : a = c * b) : a / b = c := by simp [h] @[to_additive] theorem eq_mul_of_div_eq (h : a / c = b) : a = b * c := by simp [← h] @[to_additive] theorem mul_eq_of_eq_div (h : a = c / b) : a * b = c := by simp [h] @[to_additive (attr := simp)] theorem div_right_inj : a / b = a / c ↔ b = c := div_right_injective.eq_iff @[to_additive (attr := simp)] theorem div_left_inj : b / a = c / a ↔ b = c := by rw [div_eq_mul_inv, div_eq_mul_inv] exact mul_left_inj _ @[to_additive (attr := simp) sub_add_sub_cancel] theorem div_mul_div_cancel' (a b c : G) : a / b * (b / c) = a / c := by rw [← mul_div_assoc, div_mul_cancel] @[to_additive (attr := simp) sub_sub_sub_cancel_right] theorem div_div_div_cancel_right' (a b c : G) : a / c / (b / c) = a / b := by rw [← inv_div c b, div_inv_eq_mul, div_mul_div_cancel'] @[to_additive] theorem div_eq_one : a / b = 1 ↔ a = b := ⟨eq_of_div_eq_one, fun h ↦ by rw [h, div_self']⟩ alias ⟨_, div_eq_one_of_eq⟩ := div_eq_one alias ⟨_, sub_eq_zero_of_eq⟩ := sub_eq_zero @[to_additive] theorem div_ne_one : a / b ≠ 1 ↔ a ≠ b := not_congr div_eq_one @[to_additive (attr := simp)] theorem div_eq_self : a / b = a ↔ b = 1 := by rw [div_eq_mul_inv, mul_right_eq_self, inv_eq_one] @[to_additive eq_sub_iff_add_eq] theorem eq_div_iff_mul_eq' : a = b / c ↔ a * c = b := by rw [div_eq_mul_inv, eq_mul_inv_iff_mul_eq] @[to_additive] theorem div_eq_iff_eq_mul : a / b = c ↔ a = c * b := by rw [div_eq_mul_inv, mul_inv_eq_iff_eq_mul] @[to_additive] theorem eq_iff_eq_of_div_eq_div (H : a / b = c / d) : a = b ↔ c = d := by rw [← div_eq_one, H, div_eq_one] @[to_additive] theorem leftInverse_div_mul_left (c : G) : Function.LeftInverse (fun x ↦ x / c) fun x ↦ x * c := fun x ↦ mul_div_cancel_right x c @[to_additive] theorem leftInverse_mul_left_div (c : G) : Function.LeftInverse (fun x ↦ x * c) fun x ↦ x / c := fun x ↦ div_mul_cancel x c @[to_additive] theorem leftInverse_mul_right_inv_mul (c : G) : Function.LeftInverse (fun x ↦ c * x) fun x ↦ c⁻¹ * x := fun x ↦ mul_inv_cancel_left c x @[to_additive] theorem leftInverse_inv_mul_mul_right (c : G) : Function.LeftInverse (fun x ↦ c⁻¹ * x) fun x ↦ c * x := fun x ↦ inv_mul_cancel_left c x @[to_additive (attr := simp) natAbs_nsmul_eq_zero] lemma pow_natAbs_eq_one : a ^ n.natAbs = 1 ↔ a ^ n = 1 := by cases n <;> simp set_option linter.existingAttributeWarning false in @[to_additive, deprecated pow_natAbs_eq_one (since := "2024-02-14")] lemma exists_pow_eq_one_of_zpow_eq_one (hn : n ≠ 0) (h : a ^ n = 1) : ∃ n : ℕ, 0 < n ∧ a ^ n = 1 := ⟨_, Int.natAbs_pos.2 hn, pow_natAbs_eq_one.2 h⟩ attribute [deprecated natAbs_nsmul_eq_zero (since := "2024-02-14")] exists_nsmul_eq_zero_of_zsmul_eq_zero @[to_additive sub_nsmul] lemma pow_sub (a : G) {m n : ℕ} (h : n ≤ m) : a ^ (m - n) = a ^ m * (a ^ n)⁻¹ := eq_mul_inv_of_mul_eq <| by rw [← pow_add, Nat.sub_add_cancel h] @[to_additive sub_nsmul_neg] theorem inv_pow_sub (a : G) {m n : ℕ} (h : n ≤ m) : a⁻¹ ^ (m - n) = (a ^ m)⁻¹ * a ^ n := by rw [pow_sub a⁻¹ h, inv_pow, inv_pow, inv_inv] @[to_additive add_one_zsmul] lemma zpow_add_one (a : G) : ∀ n : ℤ, a ^ (n + 1) = a ^ n * a | (n : ℕ) => by simp only [← Int.ofNat_succ, zpow_natCast, pow_succ] | .negSucc 0 => by simp [Int.negSucc_eq', Int.add_left_neg] | .negSucc (n + 1) => by rw [zpow_negSucc, pow_succ', mul_inv_rev, inv_mul_cancel_right] rw [Int.negSucc_eq, Int.neg_add, Int.neg_add_cancel_right] exact zpow_negSucc _ _ @[to_additive sub_one_zsmul] lemma zpow_sub_one (a : G) (n : ℤ) : a ^ (n - 1) = a ^ n * a⁻¹ := calc a ^ (n - 1) = a ^ (n - 1) * a * a⁻¹ := (mul_inv_cancel_right _ _).symm _ = a ^ n * a⁻¹ := by rw [← zpow_add_one, Int.sub_add_cancel] @[to_additive add_zsmul] lemma zpow_add (a : G) (m n : ℤ) : a ^ (m + n) = a ^ m * a ^ n := by induction n using Int.induction_on with | hz => simp | hp n ihn => simp only [← Int.add_assoc, zpow_add_one, ihn, mul_assoc] | hn n ihn => rw [zpow_sub_one, ← mul_assoc, ← ihn, ← zpow_sub_one, Int.add_sub_assoc] @[to_additive one_add_zsmul] lemma zpow_one_add (a : G) (n : ℤ) : a ^ (1 + n) = a * a ^ n := by rw [zpow_add, zpow_one] @[to_additive add_zsmul_self] lemma mul_self_zpow (a : G) (n : ℤ) : a * a ^ n = a ^ (n + 1) := by rw [Int.add_comm, zpow_add, zpow_one] @[to_additive add_self_zsmul] lemma mul_zpow_self (a : G) (n : ℤ) : a ^ n * a = a ^ (n + 1) := (zpow_add_one ..).symm @[to_additive sub_zsmul] lemma zpow_sub (a : G) (m n : ℤ) : a ^ (m - n) = a ^ m * (a ^ n)⁻¹ := by rw [Int.sub_eq_add_neg, zpow_add, zpow_neg] @[to_additive] lemma zpow_mul_comm (a : G) (m n : ℤ) : a ^ m * a ^ n = a ^ n * a ^ m := by rw [← zpow_add, Int.add_comm, zpow_add] theorem zpow_eq_zpow_emod {x : G} (m : ℤ) {n : ℤ} (h : x ^ n = 1) : x ^ m = x ^ (m % n) := calc x ^ m = x ^ (m % n + n * (m / n)) := by rw [Int.emod_add_ediv] _ = x ^ (m % n) := by simp [zpow_add, zpow_mul, h] theorem zpow_eq_zpow_emod' {x : G} (m : ℤ) {n : ℕ} (h : x ^ n = 1) : x ^ m = x ^ (m % (n : ℤ)) := zpow_eq_zpow_emod m (by simpa) /-- To show a property of all powers of `g` it suffices to show it is closed under multiplication by `g` and `g⁻¹` on the left. For subgroups generated by more than one element, see `Subgroup.closure_induction_left`. -/ @[to_additive "To show a property of all multiples of `g` it suffices to show it is closed under addition by `g` and `-g` on the left. For additive subgroups generated by more than one element, see `AddSubgroup.closure_induction_left`."] lemma zpow_induction_left {g : G} {P : G → Prop} (h_one : P (1 : G)) (h_mul : ∀ a, P a → P (g * a)) (h_inv : ∀ a, P a → P (g⁻¹ * a)) (n : ℤ) : P (g ^ n) := by induction' n using Int.induction_on with n ih n ih · rwa [zpow_zero] · rw [Int.add_comm, zpow_add, zpow_one] exact h_mul _ ih · rw [Int.sub_eq_add_neg, Int.add_comm, zpow_add, zpow_neg_one] exact h_inv _ ih /-- To show a property of all powers of `g` it suffices to show it is closed under multiplication by `g` and `g⁻¹` on the right. For subgroups generated by more than one element, see `Subgroup.closure_induction_right`. -/ @[to_additive "To show a property of all multiples of `g` it suffices to show it is closed under addition by `g` and `-g` on the right. For additive subgroups generated by more than one element, see `AddSubgroup.closure_induction_right`."] lemma zpow_induction_right {g : G} {P : G → Prop} (h_one : P (1 : G)) (h_mul : ∀ a, P a → P (a * g)) (h_inv : ∀ a, P a → P (a * g⁻¹)) (n : ℤ) : P (g ^ n) := by induction' n using Int.induction_on with n ih n ih · rwa [zpow_zero] · rw [zpow_add_one] exact h_mul _ ih · rw [zpow_sub_one] exact h_inv _ ih end Group section CommGroup variable [CommGroup G] {a b c d : G} attribute [local simp] mul_assoc mul_comm mul_left_comm div_eq_mul_inv @[to_additive] theorem div_eq_of_eq_mul' {a b c : G} (h : a = b * c) : a / b = c := by rw [h, div_eq_mul_inv, mul_comm, inv_mul_cancel_left] @[to_additive (attr := simp)] theorem mul_div_mul_left_eq_div (a b c : G) : c * a / (c * b) = a / b := by rw [div_eq_mul_inv, mul_inv_rev, mul_comm b⁻¹ c⁻¹, mul_comm c a, mul_assoc, ← mul_assoc c, mul_right_inv, one_mul, div_eq_mul_inv] @[to_additive eq_sub_of_add_eq'] theorem eq_div_of_mul_eq'' (h : c * a = b) : a = b / c := by simp [h.symm] @[to_additive] theorem eq_mul_of_div_eq' (h : a / b = c) : a = b * c := by simp [h.symm] @[to_additive] theorem mul_eq_of_eq_div' (h : b = c / a) : a * b = c := by rw [h, div_eq_mul_inv, mul_comm c, mul_inv_cancel_left] @[to_additive sub_sub_self] theorem div_div_self' (a b : G) : a / (a / b) = b := by simp @[to_additive] theorem div_eq_div_mul_div (a b c : G) : a / b = c / b * (a / c) := by simp [mul_left_comm c] @[to_additive (attr := simp)] theorem div_div_cancel (a b : G) : a / (a / b) = b := div_div_self' a b @[to_additive (attr := simp)] theorem div_div_cancel_left (a b : G) : a / b / a = b⁻¹ := by simp @[to_additive eq_sub_iff_add_eq'] theorem eq_div_iff_mul_eq'' : a = b / c ↔ c * a = b := by rw [eq_div_iff_mul_eq', mul_comm] @[to_additive] theorem div_eq_iff_eq_mul' : a / b = c ↔ a = b * c := by rw [div_eq_iff_eq_mul, mul_comm] @[to_additive (attr := simp)] theorem mul_div_cancel_left (a b : G) : a * b / a = b := by rw [div_eq_inv_mul, inv_mul_cancel_left] @[to_additive (attr := simp)] theorem mul_div_cancel (a b : G) : a * (b / a) = b := by rw [← mul_div_assoc, mul_div_cancel_left] @[to_additive (attr := simp)] theorem div_mul_cancel_left (a b : G) : a / (a * b) = b⁻¹ := by rw [← inv_div, mul_div_cancel_left] -- This lemma is in the `simp` set under the name `mul_inv_cancel_comm_assoc`, -- along with the additive version `add_neg_cancel_comm_assoc`, -- defined in `Algebra.Group.Commute` @[to_additive] theorem mul_mul_inv_cancel'_right (a b : G) : a * (b * a⁻¹) = b := by rw [← div_eq_mul_inv, mul_div_cancel a b] @[to_additive (attr := simp)] theorem mul_mul_div_cancel (a b c : G) : a * c * (b / c) = a * b := by rw [mul_assoc, mul_div_cancel] @[to_additive (attr := simp)] theorem div_mul_mul_cancel (a b c : G) : a / c * (b * c) = a * b := by rw [mul_left_comm, div_mul_cancel, mul_comm] @[to_additive (attr := simp) sub_add_sub_cancel'] theorem div_mul_div_cancel'' (a b c : G) : a / b * (c / a) = c / b := by rw [mul_comm]; apply div_mul_div_cancel' @[to_additive (attr := simp)] theorem mul_div_div_cancel (a b c : G) : a * b / (a / c) = b * c := by rw [← div_mul, mul_div_cancel_left] @[to_additive (attr := simp)] theorem div_div_div_cancel_left (a b c : G) : c / a / (c / b) = b / a := by rw [← inv_div b c, div_inv_eq_mul, mul_comm, div_mul_div_cancel'] @[to_additive] theorem div_eq_div_iff_mul_eq_mul : a / b = c / d ↔ a * d = c * b := by rw [div_eq_iff_eq_mul, div_mul_eq_mul_div, eq_comm, div_eq_iff_eq_mul'] simp only [mul_comm, eq_comm] @[to_additive] theorem div_eq_div_iff_div_eq_div : a / b = c / d ↔ a / c = b / d := by rw [div_eq_iff_eq_mul, div_mul_eq_mul_div, div_eq_iff_eq_mul', mul_div_assoc] end CommGroup section multiplicative variable [Monoid β] (p r : α → α → Prop) [IsTotal α r] (f : α → α → β) @[to_additive additive_of_symmetric_of_isTotal] lemma multiplicative_of_symmetric_of_isTotal (hsymm : Symmetric p) (hf_swap : ∀ {a b}, p a b → f a b * f b a = 1) (hmul : ∀ {a b c}, r a b → r b c → p a b → p b c → p a c → f a c = f a b * f b c) {a b c : α} (pab : p a b) (pbc : p b c) (pac : p a c) : f a c = f a b * f b c := by have hmul' : ∀ {b c}, r b c → p a b → p b c → p a c → f a c = f a b * f b c := by intros b c rbc pab pbc pac obtain rab | rba := total_of r a b · exact hmul rab rbc pab pbc pac rw [← one_mul (f a c), ← hf_swap pab, mul_assoc] obtain rac | rca := total_of r a c · rw [hmul rba rac (hsymm pab) pac pbc] · rw [hmul rbc rca pbc (hsymm pac) (hsymm pab), mul_assoc, hf_swap (hsymm pac), mul_one] obtain rbc | rcb := total_of r b c · exact hmul' rbc pab pbc pac · rw [hmul' rcb pac (hsymm pbc) pab, mul_assoc, hf_swap (hsymm pbc), mul_one] /-- If a binary function from a type equipped with a total relation `r` to a monoid is anti-symmetric (i.e. satisfies `f a b * f b a = 1`), in order to show it is multiplicative (i.e. satisfies `f a c = f a b * f b c`), we may assume `r a b` and `r b c` are satisfied. We allow restricting to a subset specified by a predicate `p`. -/ @[to_additive additive_of_isTotal "If a binary function from a type equipped with a total relation `r` to an additive monoid is anti-symmetric (i.e. satisfies `f a b + f b a = 0`), in order to show it is additive (i.e. satisfies `f a c = f a b + f b c`), we may assume `r a b` and `r b c` are satisfied. We allow restricting to a subset specified by a predicate `p`."] theorem multiplicative_of_isTotal (p : α → Prop) (hswap : ∀ {a b}, p a → p b → f a b * f b a = 1) (hmul : ∀ {a b c}, r a b → r b c → p a → p b → p c → f a c = f a b * f b c) {a b c : α} (pa : p a) (pb : p b) (pc : p c) : f a c = f a b * f b c := by apply multiplicative_of_symmetric_of_isTotal (fun a b => p a ∧ p b) r f fun _ _ => And.symm · simp_rw [and_imp]; exact @hswap · exact fun rab rbc pab _pbc pac => hmul rab rbc pab.1 pab.2 pac.2 exacts [⟨pa, pb⟩, ⟨pb, pc⟩, ⟨pa, pc⟩] end multiplicative @[deprecated (since := "2024-03-20")] alias div_mul_cancel' := div_mul_cancel @[deprecated (since := "2024-03-20")] alias mul_div_cancel'' := mul_div_cancel_right -- The name `add_sub_cancel` was reused -- @[deprecated (since := "2024-03-20")] alias add_sub_cancel := add_sub_cancel_right @[deprecated (since := "2024-03-20")] alias div_mul_cancel''' := div_mul_cancel_right @[deprecated (since := "2024-03-20")] alias sub_add_cancel'' := sub_add_cancel_right @[deprecated (since := "2024-03-20")] alias mul_div_cancel''' := mul_div_cancel_left @[deprecated (since := "2024-03-20")] alias add_sub_cancel' := add_sub_cancel_left @[deprecated (since := "2024-03-20")] alias mul_div_cancel'_right := mul_div_cancel @[deprecated (since := "2024-03-20")] alias add_sub_cancel'_right := add_sub_cancel @[deprecated (since := "2024-03-20")] alias div_mul_cancel'' := div_mul_cancel_left @[deprecated (since := "2024-03-20")] alias sub_add_cancel' := sub_add_cancel_left
Algebra\Group\Center.lean
/- Copyright (c) 2021 Eric Wieser. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Eric Wieser, Jireh Loreaux -/ import Mathlib.Algebra.Group.Commute.Units import Mathlib.Algebra.Group.Invertible.Basic import Mathlib.Data.Set.Basic import Mathlib.Logic.Basic /-! # Centers of magmas and semigroups ## Main definitions * `Set.center`: the center of a magma * `Set.addCenter`: the center of an additive magma * `Set.centralizer`: the centralizer of a subset of a magma * `Set.addCentralizer`: the centralizer of a subset of an additive magma ## See also See `Mathlib.GroupTheory.Subsemigroup.Center` for the definition of the center as a subsemigroup: * `Subsemigroup.center`: the center of a semigroup * `AddSubsemigroup.center`: the center of an additive semigroup We provide `Submonoid.center`, `AddSubmonoid.center`, `Subgroup.center`, `AddSubgroup.center`, `Subsemiring.center`, and `Subring.center` in other files. See `Mathlib.GroupTheory.Subsemigroup.Centralizer` for the definition of the centralizer as a subsemigroup: * `Subsemigroup.centralizer`: the centralizer of a subset of a semigroup * `AddSubsemigroup.centralizer`: the centralizer of a subset of an additive semigroup We provide `Monoid.centralizer`, `AddMonoid.centralizer`, `Subgroup.centralizer`, and `AddSubgroup.centralizer` in other files. -/ assert_not_exists Finset assert_not_exists MonoidWithZero assert_not_exists Subsemigroup variable {M : Type*} {S T : Set M} /-- Conditions for an element to be additively central -/ structure IsAddCentral [Add M] (z : M) : Prop where /-- addition commutes -/ comm (a : M) : z + a = a + z /-- associative property for left addition -/ left_assoc (b c : M) : z + (b + c) = (z + b) + c /-- middle associative addition property -/ mid_assoc (a c : M) : (a + z) + c = a + (z + c) /-- associative property for right addition -/ right_assoc (a b : M) : (a + b) + z = a + (b + z) /-- Conditions for an element to be multiplicatively central -/ @[to_additive] structure IsMulCentral [Mul M] (z : M) : Prop where /-- multiplication commutes -/ comm (a : M) : z * a = a * z /-- associative property for left multiplication -/ left_assoc (b c : M) : z * (b * c) = (z * b) * c /-- middle associative multiplication property -/ mid_assoc (a c : M) : (a * z) * c = a * (z * c) /-- associative property for right multiplication -/ right_assoc (a b : M) : (a * b) * z = a * (b * z) attribute [mk_iff] IsMulCentral IsAddCentral attribute [to_additive existing] isMulCentral_iff namespace IsMulCentral variable {a b c : M} [Mul M] -- cf. `Commute.left_comm` @[to_additive] protected theorem left_comm (h : IsMulCentral a) (b c) : a * (b * c) = b * (a * c) := by simp only [h.comm, h.right_assoc] -- cf. `Commute.right_comm` @[to_additive] protected theorem right_comm (h : IsMulCentral c) (a b) : a * b * c = a * c * b := by simp only [h.right_assoc, h.mid_assoc, h.comm] end IsMulCentral namespace Set /-! ### Center -/ section Mul variable [Mul M] variable (M) in /-- The center of a magma. -/ @[to_additive addCenter " The center of an additive magma. "] def center : Set M := { z | IsMulCentral z } variable (S) in /-- The centralizer of a subset of a magma. -/ @[to_additive addCentralizer " The centralizer of a subset of an additive magma. "] def centralizer : Set M := {c | ∀ m ∈ S, m * c = c * m} -- Porting note: The `to_additive` version used to be `mem_addCenter` without the iff @[to_additive mem_addCenter_iff] theorem mem_center_iff {z : M} : z ∈ center M ↔ IsMulCentral z := Iff.rfl @[to_additive mem_addCentralizer] lemma mem_centralizer_iff {c : M} : c ∈ centralizer S ↔ ∀ m ∈ S, m * c = c * m := Iff.rfl @[to_additive (attr := simp) add_mem_addCenter] theorem mul_mem_center {z₁ z₂ : M} (hz₁ : z₁ ∈ Set.center M) (hz₂ : z₂ ∈ Set.center M) : z₁ * z₂ ∈ Set.center M where comm a := calc z₁ * z₂ * a = z₂ * z₁ * a := by rw [hz₁.comm] _ = z₂ * (z₁ * a) := by rw [hz₁.mid_assoc z₂] _ = (a * z₁) * z₂ := by rw [hz₁.comm, hz₂.comm] _ = a * (z₁ * z₂) := by rw [hz₂.right_assoc a z₁] left_assoc (b c : M) := calc z₁ * z₂ * (b * c) = z₁ * (z₂ * (b * c)) := by rw [hz₂.mid_assoc] _ = z₁ * ((z₂ * b) * c) := by rw [hz₂.left_assoc] _ = (z₁ * (z₂ * b)) * c := by rw [hz₁.left_assoc] _ = z₁ * z₂ * b * c := by rw [hz₂.mid_assoc] mid_assoc (a c : M) := calc a * (z₁ * z₂) * c = ((a * z₁) * z₂) * c := by rw [hz₁.mid_assoc] _ = (a * z₁) * (z₂ * c) := by rw [hz₂.mid_assoc] _ = a * (z₁ * (z₂ * c)) := by rw [hz₁.mid_assoc] _ = a * (z₁ * z₂ * c) := by rw [hz₂.mid_assoc] right_assoc (a b : M) := calc a * b * (z₁ * z₂) = ((a * b) * z₁) * z₂ := by rw [hz₂.right_assoc] _ = (a * (b * z₁)) * z₂ := by rw [hz₁.right_assoc] _ = a * ((b * z₁) * z₂) := by rw [hz₂.right_assoc] _ = a * (b * (z₁ * z₂)) := by rw [hz₁.mid_assoc] @[to_additive addCenter_subset_addCentralizer] lemma center_subset_centralizer (S : Set M) : Set.center M ⊆ S.centralizer := fun _ hx m _ ↦ (hx.comm m).symm @[to_additive (attr := gcongr) addCentralizer_subset] lemma centralizer_subset (h : S ⊆ T) : centralizer T ⊆ centralizer S := fun _ ht s hs ↦ ht s (h hs) @[to_additive subset_addCentralizer_addCentralizer] lemma subset_centralizer_centralizer : S ⊆ S.centralizer.centralizer := by intro x hx simp only [Set.mem_centralizer_iff] exact fun y hy => (hy x hx).symm @[to_additive (attr := simp) addCentralizer_addCentralizer_addCentralizer] lemma centralizer_centralizer_centralizer (S : Set M) : S.centralizer.centralizer.centralizer = S.centralizer := by refine Set.Subset.antisymm ?_ Set.subset_centralizer_centralizer intro x hx rw [Set.mem_centralizer_iff] intro y hy rw [Set.mem_centralizer_iff] at hx exact hx y <| Set.subset_centralizer_centralizer hy @[to_additive decidableMemAddCentralizer] instance decidableMemCentralizer [∀ a : M, Decidable <| ∀ b ∈ S, b * a = a * b] : DecidablePred (· ∈ centralizer S) := fun _ ↦ decidable_of_iff' _ mem_centralizer_iff end Mul section Semigroup variable [Semigroup M] {a b : M} @[to_additive] theorem _root_.Semigroup.mem_center_iff {z : M} : z ∈ Set.center M ↔ ∀ g, g * z = z * g := ⟨fun a g ↦ by rw [IsMulCentral.comm a g], fun h ↦ ⟨fun _ ↦ (Commute.eq (h _)).symm, fun _ _ ↦ (mul_assoc z _ _).symm, fun _ _ ↦ mul_assoc _ z _, fun _ _ ↦ mul_assoc _ _ z⟩ ⟩ @[to_additive (attr := simp) add_mem_addCentralizer] lemma mul_mem_centralizer (ha : a ∈ centralizer S) (hb : b ∈ centralizer S) : a * b ∈ centralizer S := fun g hg ↦ by rw [mul_assoc, ← hb g hg, ← mul_assoc, ha g hg, mul_assoc] @[to_additive (attr := simp) addCentralizer_eq_top_iff_subset] theorem centralizer_eq_top_iff_subset : centralizer S = Set.univ ↔ S ⊆ center M := eq_top_iff.trans <| ⟨ fun h _ hx ↦ Semigroup.mem_center_iff.mpr fun _ ↦ by rw [h trivial _ hx], fun h _ _ _ hm ↦ (h hm).comm _⟩ variable (M) in @[to_additive (attr := simp) addCentralizer_univ] lemma centralizer_univ : centralizer univ = center M := Subset.antisymm (fun _ ha ↦ Semigroup.mem_center_iff.mpr fun b ↦ ha b (Set.mem_univ b)) fun _ ha b _ ↦ (ha.comm b).symm -- TODO Add `instance : Decidable (IsMulCentral a)` for `instance decidableMemCenter [Mul M]` @[to_additive decidableMemAddCenter] instance decidableMemCenter [∀ a : M, Decidable <| ∀ b : M, b * a = a * b] : DecidablePred (· ∈ center M) := fun _ => decidable_of_iff' _ (Semigroup.mem_center_iff) end Semigroup section CommSemigroup variable [CommSemigroup M] variable (M) @[to_additive (attr := simp) addCenter_eq_univ] theorem center_eq_univ : center M = univ := (Subset.antisymm (subset_univ _)) fun _ _ => Semigroup.mem_center_iff.mpr (fun _ => mul_comm _ _) @[to_additive (attr := simp) addCentralizer_eq_univ] lemma centralizer_eq_univ : centralizer S = univ := eq_univ_of_forall fun _ _ _ ↦ mul_comm _ _ end CommSemigroup section MulOneClass variable [MulOneClass M] @[to_additive (attr := simp) zero_mem_addCenter] theorem one_mem_center : (1 : M) ∈ Set.center M where comm _ := by rw [one_mul, mul_one] left_assoc _ _ := by rw [one_mul, one_mul] mid_assoc _ _ := by rw [mul_one, one_mul] right_assoc _ _ := by rw [mul_one, mul_one] @[to_additive (attr := simp) zero_mem_addCentralizer] lemma one_mem_centralizer : (1 : M) ∈ centralizer S := by simp [mem_centralizer_iff] end MulOneClass section Monoid variable [Monoid M] @[to_additive subset_addCenter_add_units] theorem subset_center_units : ((↑) : Mˣ → M) ⁻¹' center M ⊆ Set.center Mˣ := fun _ ha => by rw [_root_.Semigroup.mem_center_iff] intro _ rw [← Units.eq_iff, Units.val_mul, Units.val_mul, ha.comm] @[to_additive (attr := simp)] theorem units_inv_mem_center {a : Mˣ} (ha : ↑a ∈ Set.center M) : ↑a⁻¹ ∈ Set.center M := by rw [Semigroup.mem_center_iff] at * exact (Commute.units_inv_right <| ha ·) @[simp] theorem invOf_mem_center {a : M} [Invertible a] (ha : a ∈ Set.center M) : ⅟a ∈ Set.center M := by rw [Semigroup.mem_center_iff] at * exact (Commute.invOf_right <| ha ·) end Monoid section DivisionMonoid variable [DivisionMonoid M] {a b : M} @[to_additive (attr := simp) neg_mem_addCenter] theorem inv_mem_center (ha : a ∈ Set.center M) : a⁻¹ ∈ Set.center M := by rw [_root_.Semigroup.mem_center_iff] intro _ rw [← inv_inj, mul_inv_rev, inv_inv, ha.comm, mul_inv_rev, inv_inv] @[to_additive (attr := simp) sub_mem_addCenter] theorem div_mem_center (ha : a ∈ Set.center M) (hb : b ∈ Set.center M) : a / b ∈ Set.center M := by rw [div_eq_mul_inv] exact mul_mem_center ha (inv_mem_center hb) end DivisionMonoid section Group variable [Group M] {a b : M} @[to_additive (attr := simp) neg_mem_addCentralizer] lemma inv_mem_centralizer (ha : a ∈ centralizer S) : a⁻¹ ∈ centralizer S := fun g hg ↦ by rw [mul_inv_eq_iff_eq_mul, mul_assoc, eq_inv_mul_iff_mul_eq, ha g hg] @[to_additive (attr := simp) sub_mem_addCentralizer] lemma div_mem_centralizer (ha : a ∈ centralizer S) (hb : b ∈ centralizer S) : a / b ∈ centralizer S := by simpa only [div_eq_mul_inv] using mul_mem_centralizer ha (inv_mem_centralizer hb) end Group end Set
Algebra\Group\Commutator.lean
/- Copyright (c) 2022 Thomas Browning. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Thomas Browning -/ import Mathlib.Algebra.Group.Defs import Mathlib.Data.Bracket /-! # The bracket on a group given by commutator. -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered /-- The commutator of two elements `g₁` and `g₂`. -/ instance commutatorElement {G : Type*} [Group G] : Bracket G G := ⟨fun g₁ g₂ ↦ g₁ * g₂ * g₁⁻¹ * g₂⁻¹⟩ theorem commutatorElement_def {G : Type*} [Group G] (g₁ g₂ : G) : ⁅g₁, g₂⁆ = g₁ * g₂ * g₁⁻¹ * g₂⁻¹ := rfl
Algebra\Group\Conj.lean
/- Copyright (c) 2018 Patrick Massot. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Patrick Massot, Chris Hughes, Michael Howes -/ import Mathlib.Algebra.Group.Aut import Mathlib.Algebra.Group.Semiconj.Units /-! # Conjugacy of group elements See also `MulAut.conj` and `Quandle.conj`. -/ -- TODO: After #13027, -- assert_not_exists MonoidWithZero assert_not_exists Multiset universe u v variable {α : Type u} {β : Type v} section Monoid variable [Monoid α] [Monoid β] /-- We say that `a` is conjugate to `b` if for some unit `c` we have `c * a * c⁻¹ = b`. -/ def IsConj (a b : α) := ∃ c : αˣ, SemiconjBy (↑c) a b @[refl] theorem IsConj.refl (a : α) : IsConj a a := ⟨1, SemiconjBy.one_left a⟩ @[symm] theorem IsConj.symm {a b : α} : IsConj a b → IsConj b a | ⟨c, hc⟩ => ⟨c⁻¹, hc.units_inv_symm_left⟩ theorem isConj_comm {g h : α} : IsConj g h ↔ IsConj h g := ⟨IsConj.symm, IsConj.symm⟩ @[trans] theorem IsConj.trans {a b c : α} : IsConj a b → IsConj b c → IsConj a c | ⟨c₁, hc₁⟩, ⟨c₂, hc₂⟩ => ⟨c₂ * c₁, hc₂.mul_left hc₁⟩ @[simp] theorem isConj_iff_eq {α : Type*} [CommMonoid α] {a b : α} : IsConj a b ↔ a = b := ⟨fun ⟨c, hc⟩ => by rw [SemiconjBy, mul_comm, ← Units.mul_inv_eq_iff_eq_mul, mul_assoc, c.mul_inv, mul_one] at hc exact hc, fun h => by rw [h]⟩ protected theorem MonoidHom.map_isConj (f : α →* β) {a b : α} : IsConj a b → IsConj (f a) (f b) | ⟨c, hc⟩ => ⟨Units.map f c, by rw [Units.coe_map, SemiconjBy, ← f.map_mul, hc.eq, f.map_mul]⟩ end Monoid section CancelMonoid variable [CancelMonoid α] -- These lemmas hold for `RightCancelMonoid` with the current proofs, but for the sake of -- not duplicating code (these lemmas also hold for `LeftCancelMonoids`) we leave these -- not generalised. @[simp] theorem isConj_one_right {a : α} : IsConj 1 a ↔ a = 1 := ⟨fun ⟨c, hc⟩ => mul_right_cancel (hc.symm.trans ((mul_one _).trans (one_mul _).symm)), fun h => by rw [h]⟩ @[simp] theorem isConj_one_left {a : α} : IsConj a 1 ↔ a = 1 := calc IsConj a 1 ↔ IsConj 1 a := ⟨IsConj.symm, IsConj.symm⟩ _ ↔ a = 1 := isConj_one_right end CancelMonoid section Group variable [Group α] @[simp] theorem isConj_iff {a b : α} : IsConj a b ↔ ∃ c : α, c * a * c⁻¹ = b := ⟨fun ⟨c, hc⟩ => ⟨c, mul_inv_eq_iff_eq_mul.2 hc⟩, fun ⟨c, hc⟩ => ⟨⟨c, c⁻¹, mul_inv_self c, inv_mul_self c⟩, mul_inv_eq_iff_eq_mul.1 hc⟩⟩ -- Porting note: not in simp NF. -- @[simp] theorem conj_inv {a b : α} : (b * a * b⁻¹)⁻¹ = b * a⁻¹ * b⁻¹ := ((MulAut.conj b).map_inv a).symm @[simp] theorem conj_mul {a b c : α} : b * a * b⁻¹ * (b * c * b⁻¹) = b * (a * c) * b⁻¹ := ((MulAut.conj b).map_mul a c).symm @[simp] theorem conj_pow {i : ℕ} {a b : α} : (a * b * a⁻¹) ^ i = a * b ^ i * a⁻¹ := by induction' i with i hi · simp · simp [pow_succ, hi] @[simp] theorem conj_zpow {i : ℤ} {a b : α} : (a * b * a⁻¹) ^ i = a * b ^ i * a⁻¹ := by induction' i · change (a * b * a⁻¹) ^ (_ : ℤ) = a * b ^ (_ : ℤ) * a⁻¹ simp [zpow_natCast] · simp only [zpow_negSucc, conj_pow, mul_inv_rev, inv_inv] rw [mul_assoc] -- Porting note: Added `change`, `zpow_natCast`, and `rw`. theorem conj_injective {x : α} : Function.Injective fun g : α => x * g * x⁻¹ := (MulAut.conj x).injective end Group namespace IsConj /- This small quotient API is largely copied from the API of `Associates`; where possible, try to keep them in sync -/ /-- The setoid of the relation `IsConj` iff there is a unit `u` such that `u * x = y * u` -/ protected def setoid (α : Type*) [Monoid α] : Setoid α where r := IsConj iseqv := ⟨IsConj.refl, IsConj.symm, IsConj.trans⟩ end IsConj attribute [local instance] IsConj.setoid /-- The quotient type of conjugacy classes of a group. -/ def ConjClasses (α : Type*) [Monoid α] : Type _ := Quotient (IsConj.setoid α) namespace ConjClasses section Monoid variable [Monoid α] [Monoid β] /-- The canonical quotient map from a monoid `α` into the `ConjClasses` of `α` -/ protected def mk {α : Type*} [Monoid α] (a : α) : ConjClasses α := ⟦a⟧ instance : Inhabited (ConjClasses α) := ⟨⟦1⟧⟩ theorem mk_eq_mk_iff_isConj {a b : α} : ConjClasses.mk a = ConjClasses.mk b ↔ IsConj a b := Iff.intro Quotient.exact Quot.sound theorem quotient_mk_eq_mk (a : α) : ⟦a⟧ = ConjClasses.mk a := rfl theorem quot_mk_eq_mk (a : α) : Quot.mk Setoid.r a = ConjClasses.mk a := rfl theorem forall_isConj {p : ConjClasses α → Prop} : (∀ a, p a) ↔ ∀ a, p (ConjClasses.mk a) := Iff.intro (fun h _ => h _) fun h a => Quotient.inductionOn a h theorem mk_surjective : Function.Surjective (@ConjClasses.mk α _) := forall_isConj.2 fun a => ⟨a, rfl⟩ instance : One (ConjClasses α) := ⟨⟦1⟧⟩ theorem one_eq_mk_one : (1 : ConjClasses α) = ConjClasses.mk 1 := rfl theorem exists_rep (a : ConjClasses α) : ∃ a0 : α, ConjClasses.mk a0 = a := Quot.exists_rep a /-- A `MonoidHom` maps conjugacy classes of one group to conjugacy classes of another. -/ def map (f : α →* β) : ConjClasses α → ConjClasses β := Quotient.lift (ConjClasses.mk ∘ f) fun _ _ ab => mk_eq_mk_iff_isConj.2 (f.map_isConj ab) theorem map_surjective {f : α →* β} (hf : Function.Surjective f) : Function.Surjective (ConjClasses.map f) := by intro b obtain ⟨b, rfl⟩ := ConjClasses.mk_surjective b obtain ⟨a, rfl⟩ := hf b exact ⟨ConjClasses.mk a, rfl⟩ -- Porting note: This has not been adapted to mathlib4, is it still accurate? library_note "slow-failing instance priority"/-- Certain instances trigger further searches when they are considered as candidate instances; these instances should be assigned a priority lower than the default of 1000 (for example, 900). The conditions for this rule are as follows: * a class `C` has instances `instT : C T` and `instT' : C T'` * types `T` and `T'` are both specializations of another type `S` * the parameters supplied to `S` to produce `T` are not (fully) determined by `instT`, instead they have to be found by instance search If those conditions hold, the instance `instT` should be assigned lower priority. For example, suppose the search for an instance of `DecidableEq (Multiset α)` tries the candidate instance `Con.quotient.decidableEq (c : Con M) : decidableEq c.quotient`. Since `Multiset` and `Con.quotient` are both quotient types, unification will check that the relations `List.perm` and `c.toSetoid.r` unify. However, `c.toSetoid` depends on a `Mul M` instance, so this unification triggers a search for `Mul (List α)`; this will traverse all subclasses of `Mul` before failing. On the other hand, the search for an instance of `DecidableEq (Con.quotient c)` for `c : Con M` can quickly reject the candidate instance `Multiset.decidableEq` because the type of `List.perm : List ?m_1 → List ?m_1 → Prop` does not unify with `M → M → Prop`. Therefore, we should assign `Con.quotient.decidableEq` a lower priority because it fails slowly. (In terms of the rules above, `C := DecidableEq`, `T := Con.quotient`, `instT := Con.quotient.decidableEq`, `T' := Multiset`, `instT' := Multiset.decidableEq`, and `S := Quot`.) If the type involved is a free variable (rather than an instantiation of some type `S`), the instance priority should be even lower, see Note [lower instance priority]. -/ -- see Note [slow-failing instance priority] instance (priority := 900) [DecidableRel (IsConj : α → α → Prop)] : DecidableEq (ConjClasses α) := inferInstanceAs <| DecidableEq <| Quotient (IsConj.setoid α) end Monoid section CommMonoid variable [CommMonoid α] theorem mk_injective : Function.Injective (@ConjClasses.mk α _) := fun _ _ => (mk_eq_mk_iff_isConj.trans isConj_iff_eq).1 theorem mk_bijective : Function.Bijective (@ConjClasses.mk α _) := ⟨mk_injective, mk_surjective⟩ /-- The bijection between a `CommGroup` and its `ConjClasses`. -/ def mkEquiv : α ≃ ConjClasses α := ⟨ConjClasses.mk, Quotient.lift id fun (a : α) b => isConj_iff_eq.1, Quotient.lift_mk _ _, by rw [Function.RightInverse, Function.LeftInverse, forall_isConj] intro x rw [← quotient_mk_eq_mk, ← quotient_mk_eq_mk, Quotient.lift_mk, id]⟩ end CommMonoid end ConjClasses section Monoid variable [Monoid α] /-- Given an element `a`, `conjugatesOf a` is the set of conjugates. -/ def conjugatesOf (a : α) : Set α := { b | IsConj a b } theorem mem_conjugatesOf_self {a : α} : a ∈ conjugatesOf a := IsConj.refl _ theorem IsConj.conjugatesOf_eq {a b : α} (ab : IsConj a b) : conjugatesOf a = conjugatesOf b := Set.ext fun _ => ⟨fun ag => ab.symm.trans ag, fun bg => ab.trans bg⟩ theorem isConj_iff_conjugatesOf_eq {a b : α} : IsConj a b ↔ conjugatesOf a = conjugatesOf b := ⟨IsConj.conjugatesOf_eq, fun h => by have ha := @mem_conjugatesOf_self _ _ b -- Porting note: added `@`. rwa [← h] at ha⟩ end Monoid namespace ConjClasses variable [Monoid α] attribute [local instance] IsConj.setoid /-- Given a conjugacy class `a`, `carrier a` is the set it represents. -/ def carrier : ConjClasses α → Set α := Quotient.lift conjugatesOf fun (_ : α) _ ab => IsConj.conjugatesOf_eq ab theorem mem_carrier_mk {a : α} : a ∈ carrier (ConjClasses.mk a) := IsConj.refl _ theorem mem_carrier_iff_mk_eq {a : α} {b : ConjClasses α} : a ∈ carrier b ↔ ConjClasses.mk a = b := by revert b rw [forall_isConj] intro b rw [carrier, eq_comm, mk_eq_mk_iff_isConj, ← quotient_mk_eq_mk, Quotient.lift_mk] rfl theorem carrier_eq_preimage_mk {a : ConjClasses α} : a.carrier = ConjClasses.mk ⁻¹' {a} := Set.ext fun _ => mem_carrier_iff_mk_eq end ConjClasses
Algebra\Group\ConjFinite.lean
/- Copyright (c) 2022 Eric Rodriguez. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Eric Rodriguez -/ import Mathlib.Algebra.Group.Conj import Mathlib.Data.Finite.Basic import Mathlib.Data.Fintype.Units /-! # Conjugacy of elements of finite groups -/ -- TODO: After #13027, -- assert_not_exists MonoidWithZero variable {α : Type*} [Monoid α] attribute [local instance] IsConj.setoid instance [Fintype α] [DecidableRel (IsConj : α → α → Prop)] : Fintype (ConjClasses α) := Quotient.fintype (IsConj.setoid α) instance [Finite α] : Finite (ConjClasses α) := Quotient.finite _ instance [DecidableEq α] [Fintype α] : DecidableRel (IsConj : α → α → Prop) := fun a b => inferInstanceAs (Decidable (∃ c : αˣ, c.1 * a = b * c.1)) instance conjugatesOf.fintype [Fintype α] [DecidableRel (IsConj : α → α → Prop)] {a : α} : Fintype (conjugatesOf a) := @Subtype.fintype _ _ (‹DecidableRel IsConj› a) _ namespace ConjClasses variable [Fintype α] [DecidableRel (IsConj : α → α → Prop)] instance {x : ConjClasses α} : Fintype (carrier x) := Quotient.recOnSubsingleton x fun _ => conjugatesOf.fintype end ConjClasses
Algebra\Group\Defs.lean
/- Copyright (c) 2014 Jeremy Avigad. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Jeremy Avigad, Leonardo de Moura, Simon Hudon, Mario Carneiro -/ import Mathlib.Data.Int.Notation import Mathlib.Algebra.Group.ZeroOne import Mathlib.Tactic.Lemma import Mathlib.Tactic.TypeStar import Mathlib.Tactic.Simps.Basic import Mathlib.Tactic.ToAdditive import Mathlib.Util.AssertExists /-! # Typeclasses for (semi)groups and monoids In this file we define typeclasses for algebraic structures with one binary operation. The classes are named `(Add)?(Comm)?(Semigroup|Monoid|Group)`, where `Add` means that the class uses additive notation and `Comm` means that the class assumes that the binary operation is commutative. The file does not contain any lemmas except for * axioms of typeclasses restated in the root namespace; * lemmas required for instances. For basic lemmas about these classes see `Algebra.Group.Basic`. We also introduce notation classes `SMul` and `VAdd` for multiplicative and additive actions and register the following instances: - `Pow M ℕ`, for monoids `M`, and `Pow G ℤ` for groups `G`; - `SMul ℕ M` for additive monoids `M`, and `SMul ℤ G` for additive groups `G`. `SMul` is typically, but not exclusively, used for scalar multiplication-like operators. See the module `Algebra.AddTorsor` for a motivating example for the name `VAdd` (vector addition)`. ## Notation - `+`, `-`, `*`, `/`, `^` : the usual arithmetic operations; the underlying functions are `Add.add`, `Neg.neg`/`Sub.sub`, `Mul.mul`, `Div.div`, and `HPow.hPow`. - `a • b` is used as notation for `HSMul.hSMul a b`. - `a +ᵥ b` is used as notation for `HVAdd.hVAdd a b`. -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered universe u v w open Function /-- The notation typeclass for heterogeneous additive actions. This enables the notation `a +ᵥ b : γ` where `a : α`, `b : β`. -/ class HVAdd (α : Type u) (β : Type v) (γ : outParam (Type w)) where /-- `a +ᵥ b` computes the sum of `a` and `b`. The meaning of this notation is type-dependent. -/ hVAdd : α → β → γ /-- The notation typeclass for heterogeneous scalar multiplication. This enables the notation `a • b : γ` where `a : α`, `b : β`. It is assumed to represent a left action in some sense. The notation `a • b` is augmented with a macro (below) to have it elaborate as a left action. Only the `b` argument participates in the elaboration algorithm: the algorithm uses the type of `b` when calculating the type of the surrounding arithmetic expression and it tries to insert coercions into `b` to get some `b'` such that `a • b'` has the same type as `b'`. See the module documentation near the macro for more details. -/ class HSMul (α : Type u) (β : Type v) (γ : outParam (Type w)) where /-- `a • b` computes the product of `a` and `b`. The meaning of this notation is type-dependent, but it is intended to be used for left actions. -/ hSMul : α → β → γ attribute [notation_class smul Simps.copySecond] HSMul attribute [notation_class nsmul Simps.nsmulArgs] HSMul attribute [notation_class zsmul Simps.zsmulArgs] HSMul /-- Type class for the `+ᵥ` notation. -/ class VAdd (G : Type u) (P : Type v) where /-- `a +ᵥ b` computes the sum of `a` and `b`. The meaning of this notation is type-dependent, but it is intended to be used for left actions. -/ vadd : G → P → P /-- Type class for the `-ᵥ` notation. -/ class VSub (G : outParam Type*) (P : Type*) where /-- `a -ᵥ b` computes the difference of `a` and `b`. The meaning of this notation is type-dependent, but it is intended to be used for additive torsors. -/ vsub : P → P → G /-- Typeclass for types with a scalar multiplication operation, denoted `•` (`\bu`) -/ @[to_additive (attr := ext)] class SMul (M : Type u) (α : Type v) where /-- `a • b` computes the product of `a` and `b`. The meaning of this notation is type-dependent, but it is intended to be used for left actions. -/ smul : M → α → α @[inherit_doc] infixl:65 " +ᵥ " => HVAdd.hVAdd @[inherit_doc] infixl:65 " -ᵥ " => VSub.vsub @[inherit_doc] infixr:73 " • " => HSMul.hSMul /-! We have a macro to make `x • y` notation participate in the expression tree elaborator, like other arithmetic expressions such as `+`, `*`, `/`, `^`, `=`, inequalities, etc. The macro is using the `leftact%` elaborator introduced in [this RFC](https://github.com/leanprover/lean4/issues/2854). As a concrete example of the effect of this macro, consider ```lean variable [Ring R] [AddCommMonoid M] [Module R M] (r : R) (N : Submodule R M) (m : M) (n : N) #check m + r • n ``` Without the macro, the expression would elaborate as `m + ↑(r • n : ↑N) : M`. With the macro, the expression elaborates as `m + r • (↑n : M) : M`. To get the first interpretation, one can write `m + (r • n :)`. Here is a quick review of the expression tree elaborator: 1. It builds up an expression tree of all the immediately accessible operations that are marked with `binop%`, `unop%`, `leftact%`, `rightact%`, `binrel%`, etc. 2. It elaborates every leaf term of this tree (without an expected type, so as if it were temporarily wrapped in `(... :)`). 3. Using the types of each elaborated leaf, it computes a supremum type they can all be coerced to, if such a supremum exists. 4. It inserts coercions around leaf terms wherever needed. The hypothesis is that individual expression trees tend to be calculations with respect to a single algebraic structure. Note(kmill): If we were to remove `HSMul` and switch to using `SMul` directly, then the expression tree elaborator would not be able to insert coercions within the right operand; they would likely appear as `↑(x • y)` rather than `x • ↑y`, unlike other arithmetic operations. -/ @[inherit_doc HSMul.hSMul] macro_rules | `($x • $y) => `(leftact% HSMul.hSMul $x $y) attribute [to_additive existing] Mul Div HMul instHMul HDiv instHDiv HSMul attribute [to_additive (reorder := 1 2) SMul] Pow attribute [to_additive (reorder := 1 2)] HPow attribute [to_additive existing (reorder := 1 2, 5 6) hSMul] HPow.hPow attribute [to_additive existing (reorder := 1 2, 4 5) smul] Pow.pow @[to_additive (attr := default_instance)] instance instHSMul {α β} [SMul α β] : HSMul α β β where hSMul := SMul.smul @[to_additive] theorem SMul.smul_eq_hSMul {α β} [SMul α β] : (SMul.smul : α → β → β) = HSMul.hSMul := rfl attribute [to_additive existing (reorder := 1 2)] instHPow variable {G : Type*} /-- Class of types that have an inversion operation. -/ @[to_additive, notation_class] class Inv (α : Type u) where /-- Invert an element of α. -/ inv : α → α @[inherit_doc] postfix:max "⁻¹" => Inv.inv section Mul variable [Mul G] /-- `leftMul g` denotes left multiplication by `g` -/ @[to_additive "`leftAdd g` denotes left addition by `g`"] def leftMul : G → G → G := fun g : G ↦ fun x : G ↦ g * x /-- `rightMul g` denotes right multiplication by `g` -/ @[to_additive "`rightAdd g` denotes right addition by `g`"] def rightMul : G → G → G := fun g : G ↦ fun x : G ↦ x * g /-- A mixin for left cancellative multiplication. -/ class IsLeftCancelMul (G : Type u) [Mul G] : Prop where /-- Multiplication is left cancellative. -/ protected mul_left_cancel : ∀ a b c : G, a * b = a * c → b = c /-- A mixin for right cancellative multiplication. -/ class IsRightCancelMul (G : Type u) [Mul G] : Prop where /-- Multiplication is right cancellative. -/ protected mul_right_cancel : ∀ a b c : G, a * b = c * b → a = c /-- A mixin for cancellative multiplication. -/ class IsCancelMul (G : Type u) [Mul G] extends IsLeftCancelMul G, IsRightCancelMul G : Prop /-- A mixin for left cancellative addition. -/ class IsLeftCancelAdd (G : Type u) [Add G] : Prop where /-- Addition is left cancellative. -/ protected add_left_cancel : ∀ a b c : G, a + b = a + c → b = c attribute [to_additive IsLeftCancelAdd] IsLeftCancelMul /-- A mixin for right cancellative addition. -/ class IsRightCancelAdd (G : Type u) [Add G] : Prop where /-- Addition is right cancellative. -/ protected add_right_cancel : ∀ a b c : G, a + b = c + b → a = c attribute [to_additive IsRightCancelAdd] IsRightCancelMul /-- A mixin for cancellative addition. -/ class IsCancelAdd (G : Type u) [Add G] extends IsLeftCancelAdd G, IsRightCancelAdd G : Prop attribute [to_additive IsCancelAdd] IsCancelMul section IsLeftCancelMul variable [IsLeftCancelMul G] {a b c : G} @[to_additive] theorem mul_left_cancel : a * b = a * c → b = c := IsLeftCancelMul.mul_left_cancel a b c @[to_additive] theorem mul_left_cancel_iff : a * b = a * c ↔ b = c := ⟨mul_left_cancel, congrArg _⟩ end IsLeftCancelMul section IsRightCancelMul variable [IsRightCancelMul G] {a b c : G} @[to_additive] theorem mul_right_cancel : a * b = c * b → a = c := IsRightCancelMul.mul_right_cancel a b c @[to_additive] theorem mul_right_cancel_iff : b * a = c * a ↔ b = c := ⟨mul_right_cancel, congrArg (· * a)⟩ end IsRightCancelMul end Mul /-- A semigroup is a type with an associative `(*)`. -/ @[ext] class Semigroup (G : Type u) extends Mul G where /-- Multiplication is associative -/ protected mul_assoc : ∀ a b c : G, a * b * c = a * (b * c) /-- An additive semigroup is a type with an associative `(+)`. -/ @[ext] class AddSemigroup (G : Type u) extends Add G where /-- Addition is associative -/ protected add_assoc : ∀ a b c : G, a + b + c = a + (b + c) attribute [to_additive] Semigroup section Semigroup variable [Semigroup G] @[to_additive] theorem mul_assoc : ∀ a b c : G, a * b * c = a * (b * c) := Semigroup.mul_assoc end Semigroup /-- A commutative additive magma is a type with an addition which commutes. -/ @[ext] class AddCommMagma (G : Type u) extends Add G where /-- Addition is commutative in an commutative additive magma. -/ protected add_comm : ∀ a b : G, a + b = b + a /-- A commutative multiplicative magma is a type with a multiplication which commutes. -/ @[ext] class CommMagma (G : Type u) extends Mul G where /-- Multiplication is commutative in a commutative multiplicative magma. -/ protected mul_comm : ∀ a b : G, a * b = b * a attribute [to_additive] CommMagma /-- A commutative semigroup is a type with an associative commutative `(*)`. -/ @[ext] class CommSemigroup (G : Type u) extends Semigroup G, CommMagma G where /-- A commutative additive semigroup is a type with an associative commutative `(+)`. -/ @[ext] class AddCommSemigroup (G : Type u) extends AddSemigroup G, AddCommMagma G where attribute [to_additive] CommSemigroup attribute [to_additive existing] CommSemigroup.toCommMagma section CommMagma variable [CommMagma G] @[to_additive] theorem mul_comm : ∀ a b : G, a * b = b * a := CommMagma.mul_comm /-- Any `CommMagma G` that satisfies `IsRightCancelMul G` also satisfies `IsLeftCancelMul G`. -/ @[to_additive AddCommMagma.IsRightCancelAdd.toIsLeftCancelAdd "Any `AddCommMagma G` that satisfies `IsRightCancelAdd G` also satisfies `IsLeftCancelAdd G`."] lemma CommMagma.IsRightCancelMul.toIsLeftCancelMul (G : Type u) [CommMagma G] [IsRightCancelMul G] : IsLeftCancelMul G := ⟨fun _ _ _ h => mul_right_cancel <| (mul_comm _ _).trans (h.trans (mul_comm _ _))⟩ /-- Any `CommMagma G` that satisfies `IsLeftCancelMul G` also satisfies `IsRightCancelMul G`. -/ @[to_additive AddCommMagma.IsLeftCancelAdd.toIsRightCancelAdd "Any `AddCommMagma G` that satisfies `IsLeftCancelAdd G` also satisfies `IsRightCancelAdd G`."] lemma CommMagma.IsLeftCancelMul.toIsRightCancelMul (G : Type u) [CommMagma G] [IsLeftCancelMul G] : IsRightCancelMul G := ⟨fun _ _ _ h => mul_left_cancel <| (mul_comm _ _).trans (h.trans (mul_comm _ _))⟩ /-- Any `CommMagma G` that satisfies `IsLeftCancelMul G` also satisfies `IsCancelMul G`. -/ @[to_additive AddCommMagma.IsLeftCancelAdd.toIsCancelAdd "Any `AddCommMagma G` that satisfies `IsLeftCancelAdd G` also satisfies `IsCancelAdd G`."] lemma CommMagma.IsLeftCancelMul.toIsCancelMul (G : Type u) [CommMagma G] [IsLeftCancelMul G] : IsCancelMul G := { CommMagma.IsLeftCancelMul.toIsRightCancelMul G with } /-- Any `CommMagma G` that satisfies `IsRightCancelMul G` also satisfies `IsCancelMul G`. -/ @[to_additive AddCommMagma.IsRightCancelAdd.toIsCancelAdd "Any `AddCommMagma G` that satisfies `IsRightCancelAdd G` also satisfies `IsCancelAdd G`."] lemma CommMagma.IsRightCancelMul.toIsCancelMul (G : Type u) [CommMagma G] [IsRightCancelMul G] : IsCancelMul G := { CommMagma.IsRightCancelMul.toIsLeftCancelMul G with } end CommMagma /-- A `LeftCancelSemigroup` is a semigroup such that `a * b = a * c` implies `b = c`. -/ @[ext] class LeftCancelSemigroup (G : Type u) extends Semigroup G where protected mul_left_cancel : ∀ a b c : G, a * b = a * c → b = c library_note "lower cancel priority" /-- We lower the priority of inheriting from cancellative structures. This attemts to avoid expensive checks involving bundling and unbundling with the `IsDomain` class. since `IsDomain` already depends on `Semiring`, we can synthesize that one first. Zulip discussion: https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Why.20is.20.60simpNF.60.20complaining.20here.3F -/ attribute [instance 75] LeftCancelSemigroup.toSemigroup -- See note [lower cancel priority] /-- An `AddLeftCancelSemigroup` is an additive semigroup such that `a + b = a + c` implies `b = c`. -/ @[ext] class AddLeftCancelSemigroup (G : Type u) extends AddSemigroup G where protected add_left_cancel : ∀ a b c : G, a + b = a + c → b = c attribute [instance 75] AddLeftCancelSemigroup.toAddSemigroup -- See note [lower cancel priority] attribute [to_additive] LeftCancelSemigroup /-- Any `LeftCancelSemigroup` satisfies `IsLeftCancelMul`. -/ @[to_additive AddLeftCancelSemigroup.toIsLeftCancelAdd "Any `AddLeftCancelSemigroup` satisfies `IsLeftCancelAdd`."] instance (priority := 100) LeftCancelSemigroup.toIsLeftCancelMul (G : Type u) [LeftCancelSemigroup G] : IsLeftCancelMul G := { mul_left_cancel := LeftCancelSemigroup.mul_left_cancel } /-- A `RightCancelSemigroup` is a semigroup such that `a * b = c * b` implies `a = c`. -/ @[ext] class RightCancelSemigroup (G : Type u) extends Semigroup G where protected mul_right_cancel : ∀ a b c : G, a * b = c * b → a = c attribute [instance 75] RightCancelSemigroup.toSemigroup -- See note [lower cancel priority] /-- An `AddRightCancelSemigroup` is an additive semigroup such that `a + b = c + b` implies `a = c`. -/ @[ext] class AddRightCancelSemigroup (G : Type u) extends AddSemigroup G where protected add_right_cancel : ∀ a b c : G, a + b = c + b → a = c attribute [instance 75] AddRightCancelSemigroup.toAddSemigroup -- See note [lower cancel priority] attribute [to_additive] RightCancelSemigroup /-- Any `RightCancelSemigroup` satisfies `IsRightCancelMul`. -/ @[to_additive AddRightCancelSemigroup.toIsRightCancelAdd "Any `AddRightCancelSemigroup` satisfies `IsRightCancelAdd`."] instance (priority := 100) RightCancelSemigroup.toIsRightCancelMul (G : Type u) [RightCancelSemigroup G] : IsRightCancelMul G := { mul_right_cancel := RightCancelSemigroup.mul_right_cancel } /-- Typeclass for expressing that a type `M` with multiplication and a one satisfies `1 * a = a` and `a * 1 = a` for all `a : M`. -/ class MulOneClass (M : Type u) extends One M, Mul M where /-- One is a left neutral element for multiplication -/ protected one_mul : ∀ a : M, 1 * a = a /-- One is a right neutral element for multiplication -/ protected mul_one : ∀ a : M, a * 1 = a /-- Typeclass for expressing that a type `M` with addition and a zero satisfies `0 + a = a` and `a + 0 = a` for all `a : M`. -/ class AddZeroClass (M : Type u) extends Zero M, Add M where /-- Zero is a left neutral element for addition -/ protected zero_add : ∀ a : M, 0 + a = a /-- Zero is a right neutral element for addition -/ protected add_zero : ∀ a : M, a + 0 = a attribute [to_additive] MulOneClass @[to_additive (attr := ext)] theorem MulOneClass.ext {M : Type u} : ∀ ⦃m₁ m₂ : MulOneClass M⦄, m₁.mul = m₂.mul → m₁ = m₂ := by rintro @⟨⟨one₁⟩, ⟨mul₁⟩, one_mul₁, mul_one₁⟩ @⟨⟨one₂⟩, ⟨mul₂⟩, one_mul₂, mul_one₂⟩ ⟨rfl⟩ -- FIXME (See https://github.com/leanprover/lean4/issues/1711) -- congr suffices one₁ = one₂ by cases this; rfl exact (one_mul₂ one₁).symm.trans (mul_one₁ one₂) section MulOneClass variable {M : Type u} [MulOneClass M] @[to_additive (attr := simp)] theorem one_mul : ∀ a : M, 1 * a = a := MulOneClass.one_mul @[to_additive (attr := simp)] theorem mul_one : ∀ a : M, a * 1 = a := MulOneClass.mul_one end MulOneClass section variable {M : Type u} /-- The fundamental power operation in a monoid. `npowRec n a = a*a*...*a` n times. Use instead `a ^ n`, which has better definitional behavior. -/ def npowRec [One M] [Mul M] : ℕ → M → M | 0, _ => 1 | n + 1, a => npowRec n a * a /-- The fundamental scalar multiplication in an additive monoid. `nsmulRec n a = a+a+...+a` n times. Use instead `n • a`, which has better definitional behavior. -/ def nsmulRec [Zero M] [Add M] : ℕ → M → M | 0, _ => 0 | n + 1, a => nsmulRec n a + a attribute [to_additive existing] npowRec end library_note "forgetful inheritance"/-- Suppose that one can put two mathematical structures on a type, a rich one `R` and a poor one `P`, and that one can deduce the poor structure from the rich structure through a map `F` (called a forgetful functor) (think `R = MetricSpace` and `P = TopologicalSpace`). A possible implementation would be to have a type class `rich` containing a field `R`, a type class `poor` containing a field `P`, and an instance from `rich` to `poor`. However, this creates diamond problems, and a better approach is to let `rich` extend `poor` and have a field saying that `F R = P`. To illustrate this, consider the pair `MetricSpace` / `TopologicalSpace`. Consider the topology on a product of two metric spaces. With the first approach, it could be obtained by going first from each metric space to its topology, and then taking the product topology. But it could also be obtained by considering the product metric space (with its sup distance) and then the topology coming from this distance. These would be the same topology, but not definitionally, which means that from the point of view of Lean's kernel, there would be two different `TopologicalSpace` instances on the product. This is not compatible with the way instances are designed and used: there should be at most one instance of a kind on each type. This approach has created an instance diamond that does not commute definitionally. The second approach solves this issue. Now, a metric space contains both a distance, a topology, and a proof that the topology coincides with the one coming from the distance. When one defines the product of two metric spaces, one uses the sup distance and the product topology, and one has to give the proof that the sup distance induces the product topology. Following both sides of the instance diamond then gives rise (definitionally) to the product topology on the product space. Another approach would be to have the rich type class take the poor type class as an instance parameter. It would solve the diamond problem, but it would lead to a blow up of the number of type classes one would need to declare to work with complicated classes, say a real inner product space, and would create exponential complexity when working with products of such complicated spaces, that are avoided by bundling things carefully as above. Note that this description of this specific case of the product of metric spaces is oversimplified compared to mathlib, as there is an intermediate typeclass between `MetricSpace` and `TopologicalSpace` called `UniformSpace`. The above scheme is used at both levels, embedding a topology in the uniform space structure, and a uniform structure in the metric space structure. Note also that, when `P` is a proposition, there is no such issue as any two proofs of `P` are definitionally equivalent in Lean. To avoid boilerplate, there are some designs that can automatically fill the poor fields when creating a rich structure if one doesn't want to do something special about them. For instance, in the definition of metric spaces, default tactics fill the uniform space fields if they are not given explicitly. One can also have a helper function creating the rich structure from a structure with fewer fields, where the helper function fills the remaining fields. See for instance `UniformSpace.ofCore` or `RealInnerProduct.ofCore`. For more details on this question, called the forgetful inheritance pattern, see [Competing inheritance paths in dependent type theory: a case study in functional analysis](https://hal.inria.fr/hal-02463336). -/ /-! ### Design note on `AddMonoid` and `Monoid` An `AddMonoid` has a natural `ℕ`-action, defined by `n • a = a + ... + a`, that we want to declare as an instance as it makes it possible to use the language of linear algebra. However, there are often other natural `ℕ`-actions. For instance, for any semiring `R`, the space of polynomials `Polynomial R` has a natural `R`-action defined by multiplication on the coefficients. This means that `Polynomial ℕ` would have two natural `ℕ`-actions, which are equal but not defeq. The same goes for linear maps, tensor products, and so on (and even for `ℕ` itself). To solve this issue, we embed an `ℕ`-action in the definition of an `AddMonoid` (which is by default equal to the naive action `a + ... + a`, but can be adjusted when needed), and declare a `SMul ℕ α` instance using this action. See Note [forgetful inheritance] for more explanations on this pattern. For example, when we define `Polynomial R`, then we declare the `ℕ`-action to be by multiplication on each coefficient (using the `ℕ`-action on `R` that comes from the fact that `R` is an `AddMonoid`). In this way, the two natural `SMul ℕ (Polynomial ℕ)` instances are defeq. The tactic `to_additive` transfers definitions and results from multiplicative monoids to additive monoids. To work, it has to map fields to fields. This means that we should also add corresponding fields to the multiplicative structure `Monoid`, which could solve defeq problems for powers if needed. These problems do not come up in practice, so most of the time we will not need to adjust the `npow` field when defining multiplicative objects. -/ /-- An `AddMonoid` is an `AddSemigroup` with an element `0` such that `0 + a = a + 0 = a`. -/ class AddMonoid (M : Type u) extends AddSemigroup M, AddZeroClass M where /-- Multiplication by a natural number. Set this to `nsmulRec` unless `Module` diamonds are possible. -/ protected nsmul : ℕ → M → M /-- Multiplication by `(0 : ℕ)` gives `0`. -/ protected nsmul_zero : ∀ x, nsmul 0 x = 0 := by intros; rfl /-- Multiplication by `(n + 1 : ℕ)` behaves as expected. -/ protected nsmul_succ : ∀ (n : ℕ) (x), nsmul (n + 1) x = nsmul n x + x := by intros; rfl attribute [instance 150] AddSemigroup.toAdd attribute [instance 50] AddZeroClass.toAdd /-- A `Monoid` is a `Semigroup` with an element `1` such that `1 * a = a * 1 = a`. -/ @[to_additive] class Monoid (M : Type u) extends Semigroup M, MulOneClass M where /-- Raising to the power of a natural number. -/ protected npow : ℕ → M → M := npowRec /-- Raising to the power `(0 : ℕ)` gives `1`. -/ protected npow_zero : ∀ x, npow 0 x = 1 := by intros; rfl /-- Raising to the power `(n + 1 : ℕ)` behaves as expected. -/ protected npow_succ : ∀ (n : ℕ) (x), npow (n + 1) x = npow n x * x := by intros; rfl -- Bug #660 attribute [to_additive existing] Monoid.toMulOneClass @[default_instance high] instance Monoid.toNatPow {M : Type*} [Monoid M] : Pow M ℕ := ⟨fun x n ↦ Monoid.npow n x⟩ instance AddMonoid.toNatSMul {M : Type*} [AddMonoid M] : SMul ℕ M := ⟨AddMonoid.nsmul⟩ attribute [to_additive existing toNatSMul] Monoid.toNatPow section Monoid variable {M : Type*} [Monoid M] {a b c : M} {m n : ℕ} @[to_additive (attr := simp) nsmul_eq_smul] theorem npow_eq_pow (n : ℕ) (x : M) : Monoid.npow n x = x ^ n := rfl @[to_additive] lemma left_inv_eq_right_inv (hba : b * a = 1) (hac : a * c = 1) : b = c := by rw [← one_mul c, ← hba, mul_assoc, hac, mul_one b] -- the attributes are intentionally out of order. `zero_smul` proves `zero_nsmul`. @[to_additive zero_nsmul, simp] theorem pow_zero (a : M) : a ^ 0 = 1 := Monoid.npow_zero _ @[to_additive succ_nsmul] theorem pow_succ (a : M) (n : ℕ) : a ^ (n + 1) = a ^ n * a := Monoid.npow_succ n a @[to_additive (attr := simp) one_nsmul] lemma pow_one (a : M) : a ^ 1 = a := by rw [pow_succ, pow_zero, one_mul] @[to_additive succ_nsmul'] lemma pow_succ' (a : M) : ∀ n, a ^ (n + 1) = a * a ^ n | 0 => by simp | n + 1 => by rw [pow_succ _ n, pow_succ, pow_succ', mul_assoc] @[to_additive] lemma pow_mul_comm' (a : M) (n : ℕ) : a ^ n * a = a * a ^ n := by rw [← pow_succ, pow_succ'] /-- Note that most of the lemmas about powers of two refer to it as `sq`. -/ @[to_additive two_nsmul] lemma pow_two (a : M) : a ^ 2 = a * a := by rw [pow_succ, pow_one] -- TODO: Should `alias` automatically transfer `to_additive` statements? @[to_additive existing two_nsmul] alias sq := pow_two @[to_additive three'_nsmul] lemma pow_three' (a : M) : a ^ 3 = a * a * a := by rw [pow_succ, pow_two] @[to_additive three_nsmul] lemma pow_three (a : M) : a ^ 3 = a * (a * a) := by rw [pow_succ', pow_two] -- the attributes are intentionally out of order. @[to_additive nsmul_zero, simp] lemma one_pow : ∀ n, (1 : M) ^ n = 1 | 0 => pow_zero _ | n + 1 => by rw [pow_succ, one_pow, one_mul] @[to_additive add_nsmul] lemma pow_add (a : M) (m : ℕ) : ∀ n, a ^ (m + n) = a ^ m * a ^ n | 0 => by rw [Nat.add_zero, pow_zero, mul_one] | n + 1 => by rw [pow_succ, ← mul_assoc, ← pow_add, ← pow_succ, Nat.add_assoc] @[to_additive] lemma pow_mul_comm (a : M) (m n : ℕ) : a ^ m * a ^ n = a ^ n * a ^ m := by rw [← pow_add, ← pow_add, Nat.add_comm] @[to_additive mul_nsmul] lemma pow_mul (a : M) (m : ℕ) : ∀ n, a ^ (m * n) = (a ^ m) ^ n | 0 => by rw [Nat.mul_zero, pow_zero, pow_zero] | n + 1 => by rw [Nat.mul_succ, pow_add, pow_succ, pow_mul] @[to_additive mul_nsmul'] lemma pow_mul' (a : M) (m n : ℕ) : a ^ (m * n) = (a ^ n) ^ m := by rw [Nat.mul_comm, pow_mul] @[to_additive nsmul_left_comm] lemma pow_right_comm (a : M) (m n : ℕ) : (a ^ m) ^ n = (a ^ n) ^ m := by rw [← pow_mul, Nat.mul_comm, pow_mul] end Monoid /-- An additive commutative monoid is an additive monoid with commutative `(+)`. -/ class AddCommMonoid (M : Type u) extends AddMonoid M, AddCommSemigroup M /-- A commutative monoid is a monoid with commutative `(*)`. -/ @[to_additive] class CommMonoid (M : Type u) extends Monoid M, CommSemigroup M attribute [to_additive existing] CommMonoid.toCommSemigroup section LeftCancelMonoid /-- An additive monoid in which addition is left-cancellative. Main examples are `ℕ` and groups. This is the right typeclass for many sum lemmas, as having a zero is useful to define the sum over the empty set, so `AddLeftCancelSemigroup` is not enough. -/ class AddLeftCancelMonoid (M : Type u) extends AddLeftCancelSemigroup M, AddMonoid M attribute [instance 75] AddLeftCancelMonoid.toAddMonoid -- See note [lower cancel priority] /-- A monoid in which multiplication is left-cancellative. -/ @[to_additive] class LeftCancelMonoid (M : Type u) extends LeftCancelSemigroup M, Monoid M attribute [instance 75] LeftCancelMonoid.toMonoid -- See note [lower cancel priority] attribute [to_additive existing] LeftCancelMonoid.toMonoid end LeftCancelMonoid section RightCancelMonoid /-- An additive monoid in which addition is right-cancellative. Main examples are `ℕ` and groups. This is the right typeclass for many sum lemmas, as having a zero is useful to define the sum over the empty set, so `AddRightCancelSemigroup` is not enough. -/ class AddRightCancelMonoid (M : Type u) extends AddRightCancelSemigroup M, AddMonoid M attribute [instance 75] AddRightCancelMonoid.toAddMonoid -- See note [lower cancel priority] /-- A monoid in which multiplication is right-cancellative. -/ @[to_additive] class RightCancelMonoid (M : Type u) extends RightCancelSemigroup M, Monoid M attribute [instance 75] RightCancelMonoid.toMonoid -- See note [lower cancel priority] attribute [to_additive existing] RightCancelMonoid.toMonoid end RightCancelMonoid section CancelMonoid /-- An additive monoid in which addition is cancellative on both sides. Main examples are `ℕ` and groups. This is the right typeclass for many sum lemmas, as having a zero is useful to define the sum over the empty set, so `AddRightCancelMonoid` is not enough. -/ class AddCancelMonoid (M : Type u) extends AddLeftCancelMonoid M, AddRightCancelMonoid M /-- A monoid in which multiplication is cancellative. -/ @[to_additive] class CancelMonoid (M : Type u) extends LeftCancelMonoid M, RightCancelMonoid M attribute [to_additive existing] CancelMonoid.toRightCancelMonoid /-- Commutative version of `AddCancelMonoid`. -/ class AddCancelCommMonoid (M : Type u) extends AddLeftCancelMonoid M, AddCommMonoid M attribute [instance 75] AddCancelCommMonoid.toAddCommMonoid -- See note [lower cancel priority] /-- Commutative version of `CancelMonoid`. -/ @[to_additive] class CancelCommMonoid (M : Type u) extends LeftCancelMonoid M, CommMonoid M attribute [instance 75] CancelCommMonoid.toCommMonoid -- See note [lower cancel priority] attribute [to_additive existing] CancelCommMonoid.toCommMonoid -- see Note [lower instance priority] @[to_additive] instance (priority := 100) CancelCommMonoid.toCancelMonoid (M : Type u) [CancelCommMonoid M] : CancelMonoid M := { CommMagma.IsLeftCancelMul.toIsRightCancelMul M with } /-- Any `CancelMonoid G` satisfies `IsCancelMul G`. -/ @[to_additive toIsCancelAdd "Any `AddCancelMonoid G` satisfies `IsCancelAdd G`."] instance (priority := 100) CancelMonoid.toIsCancelMul (M : Type u) [CancelMonoid M] : IsCancelMul M := { mul_left_cancel := LeftCancelSemigroup.mul_left_cancel mul_right_cancel := RightCancelSemigroup.mul_right_cancel } end CancelMonoid /-- The fundamental power operation in a group. `zpowRec n a = a*a*...*a` n times, for integer `n`. Use instead `a ^ n`, which has better definitional behavior. -/ def zpowRec [One G] [Mul G] [Inv G] (npow : ℕ → G → G := npowRec) : ℤ → G → G | Int.ofNat n, a => npow n a | Int.negSucc n, a => (npow n.succ a)⁻¹ /-- The fundamental scalar multiplication in an additive group. `zpowRec n a = a+a+...+a` n times, for integer `n`. Use instead `n • a`, which has better definitional behavior. -/ def zsmulRec [Zero G] [Add G] [Neg G] (nsmul : ℕ → G → G := nsmulRec) : ℤ → G → G | Int.ofNat n, a => nsmul n a | Int.negSucc n, a => -nsmul n.succ a attribute [to_additive existing] zpowRec section InvolutiveInv /-- Auxiliary typeclass for types with an involutive `Neg`. -/ class InvolutiveNeg (A : Type*) extends Neg A where protected neg_neg : ∀ x : A, - -x = x /-- Auxiliary typeclass for types with an involutive `Inv`. -/ @[to_additive] class InvolutiveInv (G : Type*) extends Inv G where protected inv_inv : ∀ x : G, x⁻¹⁻¹ = x variable [InvolutiveInv G] @[to_additive (attr := simp)] theorem inv_inv (a : G) : a⁻¹⁻¹ = a := InvolutiveInv.inv_inv _ end InvolutiveInv /-! ### Design note on `DivInvMonoid`/`SubNegMonoid` and `DivisionMonoid`/`SubtractionMonoid` Those two pairs of made-up classes fulfill slightly different roles. `DivInvMonoid`/`SubNegMonoid` provides the minimum amount of information to define the `ℤ` action (`zpow` or `zsmul`). Further, it provides a `div` field, matching the forgetful inheritance pattern. This is useful to shorten extension clauses of stronger structures (`Group`, `GroupWithZero`, `DivisionRing`, `Field`) and for a few structures with a rather weak pseudo-inverse (`Matrix`). `DivisionMonoid`/`SubtractionMonoid` is targeted at structures with stronger pseudo-inverses. It is an ad hoc collection of axioms that are mainly respected by three things: * Groups * Groups with zero * The pointwise monoids `Set α`, `Finset α`, `Filter α` It acts as a middle ground for structures with an inversion operator that plays well with multiplication, except for the fact that it might not be a true inverse (`a / a ≠ 1` in general). The axioms are pretty arbitrary (many other combinations are equivalent to it), but they are independent: * Without `DivisionMonoid.div_eq_mul_inv`, you can define `/` arbitrarily. * Without `DivisionMonoid.inv_inv`, you can consider `WithTop Unit` with `a⁻¹ = ⊤` for all `a`. * Without `DivisionMonoid.mul_inv_rev`, you can consider `WithTop α` with `a⁻¹ = a` for all `a` where `α` non commutative. * Without `DivisionMonoid.inv_eq_of_mul`, you can consider any `CommMonoid` with `a⁻¹ = a` for all `a`. As a consequence, a few natural structures do not fit in this framework. For example, `ENNReal` respects everything except for the fact that `(0 * ∞)⁻¹ = 0⁻¹ = ∞` while `∞⁻¹ * 0⁻¹ = 0 * ∞ = 0`. -/ /-- In a class equipped with instances of both `Monoid` and `Inv`, this definition records what the default definition for `Div` would be: `a * b⁻¹`. This is later provided as the default value for the `Div` instance in `DivInvMonoid`. We keep it as a separate definition rather than inlining it in `DivInvMonoid` so that the `Div` field of individual `DivInvMonoid`s constructed using that default value will not be unfolded at `.instance` transparency. -/ def DivInvMonoid.div' {G : Type u} [Monoid G] [Inv G] (a b : G) : G := a * b⁻¹ /-- A `DivInvMonoid` is a `Monoid` with operations `/` and `⁻¹` satisfying `div_eq_mul_inv : ∀ a b, a / b = a * b⁻¹`. This deduplicates the name `div_eq_mul_inv`. The default for `div` is such that `a / b = a * b⁻¹` holds by definition. Adding `div` as a field rather than defining `a / b := a * b⁻¹` allows us to avoid certain classes of unification failures, for example: Let `Foo X` be a type with a `∀ X, Div (Foo X)` instance but no `∀ X, Inv (Foo X)`, e.g. when `Foo X` is a `EuclideanDomain`. Suppose we also have an instance `∀ X [Cromulent X], GroupWithZero (Foo X)`. Then the `(/)` coming from `GroupWithZero.div` cannot be definitionally equal to the `(/)` coming from `Foo.Div`. In the same way, adding a `zpow` field makes it possible to avoid definitional failures in diamonds. See the definition of `Monoid` and Note [forgetful inheritance] for more explanations on this. -/ class DivInvMonoid (G : Type u) extends Monoid G, Inv G, Div G where protected div := DivInvMonoid.div' /-- `a / b := a * b⁻¹` -/ protected div_eq_mul_inv : ∀ a b : G, a / b = a * b⁻¹ := by intros; rfl /-- The power operation: `a ^ n = a * ··· * a`; `a ^ (-n) = a⁻¹ * ··· a⁻¹` (`n` times) -/ protected zpow : ℤ → G → G := zpowRec npowRec /-- `a ^ 0 = 1` -/ protected zpow_zero' : ∀ a : G, zpow 0 a = 1 := by intros; rfl /-- `a ^ (n + 1) = a ^ n * a` -/ protected zpow_succ' (n : ℕ) (a : G) : zpow (Int.ofNat n.succ) a = zpow (Int.ofNat n) a * a := by intros; rfl /-- `a ^ -(n + 1) = (a ^ (n + 1))⁻¹` -/ protected zpow_neg' (n : ℕ) (a : G) : zpow (Int.negSucc n) a = (zpow n.succ a)⁻¹ := by intros; rfl /-- In a class equipped with instances of both `AddMonoid` and `Neg`, this definition records what the default definition for `Sub` would be: `a + -b`. This is later provided as the default value for the `Sub` instance in `SubNegMonoid`. We keep it as a separate definition rather than inlining it in `SubNegMonoid` so that the `Sub` field of individual `SubNegMonoid`s constructed using that default value will not be unfolded at `.instance` transparency. -/ def SubNegMonoid.sub' {G : Type u} [AddMonoid G] [Neg G] (a b : G) : G := a + -b attribute [to_additive existing SubNegMonoid.sub'] DivInvMonoid.div' /-- A `SubNegMonoid` is an `AddMonoid` with unary `-` and binary `-` operations satisfying `sub_eq_add_neg : ∀ a b, a - b = a + -b`. The default for `sub` is such that `a - b = a + -b` holds by definition. Adding `sub` as a field rather than defining `a - b := a + -b` allows us to avoid certain classes of unification failures, for example: Let `foo X` be a type with a `∀ X, Sub (Foo X)` instance but no `∀ X, Neg (Foo X)`. Suppose we also have an instance `∀ X [Cromulent X], AddGroup (Foo X)`. Then the `(-)` coming from `AddGroup.sub` cannot be definitionally equal to the `(-)` coming from `Foo.Sub`. In the same way, adding a `zsmul` field makes it possible to avoid definitional failures in diamonds. See the definition of `AddMonoid` and Note [forgetful inheritance] for more explanations on this. -/ class SubNegMonoid (G : Type u) extends AddMonoid G, Neg G, Sub G where protected sub := SubNegMonoid.sub' protected sub_eq_add_neg : ∀ a b : G, a - b = a + -b := by intros; rfl /-- Multiplication by an integer. Set this to `zsmulRec` unless `Module` diamonds are possible. -/ protected zsmul : ℤ → G → G protected zsmul_zero' : ∀ a : G, zsmul 0 a = 0 := by intros; rfl protected zsmul_succ' (n : ℕ) (a : G) : zsmul (Int.ofNat n.succ) a = zsmul (Int.ofNat n) a + a := by intros; rfl protected zsmul_neg' (n : ℕ) (a : G) : zsmul (Int.negSucc n) a = -zsmul n.succ a := by intros; rfl attribute [to_additive SubNegMonoid] DivInvMonoid instance DivInvMonoid.Pow {M} [DivInvMonoid M] : Pow M ℤ := ⟨fun x n ↦ DivInvMonoid.zpow n x⟩ instance SubNegMonoid.SMulInt {M} [SubNegMonoid M] : SMul ℤ M := ⟨SubNegMonoid.zsmul⟩ attribute [to_additive existing SubNegMonoid.SMulInt] DivInvMonoid.Pow section DivInvMonoid variable [DivInvMonoid G] {a b : G} @[to_additive (attr := simp) zsmul_eq_smul] theorem zpow_eq_pow (n : ℤ) (x : G) : DivInvMonoid.zpow n x = x ^ n := rfl @[to_additive (attr := simp) zero_zsmul] theorem zpow_zero (a : G) : a ^ (0 : ℤ) = 1 := DivInvMonoid.zpow_zero' a @[to_additive (attr := simp, norm_cast) natCast_zsmul] theorem zpow_natCast (a : G) : ∀ n : ℕ, a ^ (n : ℤ) = a ^ n | 0 => (zpow_zero _).trans (pow_zero _).symm | n + 1 => calc a ^ (↑(n + 1) : ℤ) = a ^ (n : ℤ) * a := DivInvMonoid.zpow_succ' _ _ _ = a ^ n * a := congrArg (· * a) (zpow_natCast a n) _ = a ^ (n + 1) := (pow_succ _ _).symm @[deprecated (since := "2024-03-20")] alias zpow_coe_nat := zpow_natCast @[deprecated (since := "2024-03-20")] alias coe_nat_zsmul := natCast_zsmul -- See note [no_index around OfNat.ofNat] @[to_additive ofNat_zsmul] lemma zpow_ofNat (a : G) (n : ℕ) : a ^ (no_index (OfNat.ofNat n) : ℤ) = a ^ OfNat.ofNat n := zpow_natCast .. theorem zpow_negSucc (a : G) (n : ℕ) : a ^ (Int.negSucc n) = (a ^ (n + 1))⁻¹ := by rw [← zpow_natCast] exact DivInvMonoid.zpow_neg' n a theorem negSucc_zsmul {G} [SubNegMonoid G] (a : G) (n : ℕ) : Int.negSucc n • a = -((n + 1) • a) := by rw [← natCast_zsmul] exact SubNegMonoid.zsmul_neg' n a attribute [to_additive existing (attr := simp) negSucc_zsmul] zpow_negSucc /-- Dividing by an element is the same as multiplying by its inverse. This is a duplicate of `DivInvMonoid.div_eq_mul_inv` ensuring that the types unfold better. -/ @[to_additive "Subtracting an element is the same as adding by its negative. This is a duplicate of `SubNegMonoid.sub_eq_mul_neg` ensuring that the types unfold better."] theorem div_eq_mul_inv (a b : G) : a / b = a * b⁻¹ := DivInvMonoid.div_eq_mul_inv _ _ alias division_def := div_eq_mul_inv @[to_additive (attr := simp) one_zsmul] lemma zpow_one (a : G) : a ^ (1 : ℤ) = a := by rw [zpow_ofNat, pow_one] @[to_additive two_zsmul] lemma zpow_two (a : G) : a ^ (2 : ℤ) = a * a := by rw [zpow_ofNat, pow_two] @[to_additive neg_one_zsmul] lemma zpow_neg_one (x : G) : x ^ (-1 : ℤ) = x⁻¹ := (zpow_negSucc x 0).trans <| congr_arg Inv.inv (pow_one x) @[to_additive] lemma zpow_neg_coe_of_pos (a : G) : ∀ {n : ℕ}, 0 < n → a ^ (-(n : ℤ)) = (a ^ n)⁻¹ | _ + 1, _ => zpow_negSucc _ _ end DivInvMonoid section InvOneClass /-- Typeclass for expressing that `-0 = 0`. -/ class NegZeroClass (G : Type*) extends Zero G, Neg G where protected neg_zero : -(0 : G) = 0 /-- A `SubNegMonoid` where `-0 = 0`. -/ class SubNegZeroMonoid (G : Type*) extends SubNegMonoid G, NegZeroClass G /-- Typeclass for expressing that `1⁻¹ = 1`. -/ @[to_additive] class InvOneClass (G : Type*) extends One G, Inv G where protected inv_one : (1 : G)⁻¹ = 1 /-- A `DivInvMonoid` where `1⁻¹ = 1`. -/ @[to_additive SubNegZeroMonoid] class DivInvOneMonoid (G : Type*) extends DivInvMonoid G, InvOneClass G -- FIXME: `to_additive` is not operating on the second parent. (#660) attribute [to_additive existing] DivInvOneMonoid.toInvOneClass variable [InvOneClass G] @[to_additive (attr := simp)] theorem inv_one : (1 : G)⁻¹ = 1 := InvOneClass.inv_one end InvOneClass /-- A `SubtractionMonoid` is a `SubNegMonoid` with involutive negation and such that `-(a + b) = -b + -a` and `a + b = 0 → -a = b`. -/ class SubtractionMonoid (G : Type u) extends SubNegMonoid G, InvolutiveNeg G where protected neg_add_rev (a b : G) : -(a + b) = -b + -a /-- Despite the asymmetry of `neg_eq_of_add`, the symmetric version is true thanks to the involutivity of negation. -/ protected neg_eq_of_add (a b : G) : a + b = 0 → -a = b /-- A `DivisionMonoid` is a `DivInvMonoid` with involutive inversion and such that `(a * b)⁻¹ = b⁻¹ * a⁻¹` and `a * b = 1 → a⁻¹ = b`. This is the immediate common ancestor of `Group` and `GroupWithZero`. -/ @[to_additive SubtractionMonoid] class DivisionMonoid (G : Type u) extends DivInvMonoid G, InvolutiveInv G where protected mul_inv_rev (a b : G) : (a * b)⁻¹ = b⁻¹ * a⁻¹ /-- Despite the asymmetry of `inv_eq_of_mul`, the symmetric version is true thanks to the involutivity of inversion. -/ protected inv_eq_of_mul (a b : G) : a * b = 1 → a⁻¹ = b attribute [to_additive existing] DivisionMonoid.toInvolutiveInv section DivisionMonoid variable [DivisionMonoid G] {a b : G} @[to_additive (attr := simp) neg_add_rev] theorem mul_inv_rev (a b : G) : (a * b)⁻¹ = b⁻¹ * a⁻¹ := DivisionMonoid.mul_inv_rev _ _ @[to_additive] theorem inv_eq_of_mul_eq_one_right : a * b = 1 → a⁻¹ = b := DivisionMonoid.inv_eq_of_mul _ _ @[to_additive] theorem inv_eq_of_mul_eq_one_left (h : a * b = 1) : b⁻¹ = a := by rw [← inv_eq_of_mul_eq_one_right h, inv_inv] @[to_additive] theorem eq_inv_of_mul_eq_one_left (h : a * b = 1) : a = b⁻¹ := (inv_eq_of_mul_eq_one_left h).symm end DivisionMonoid /-- Commutative `SubtractionMonoid`. -/ class SubtractionCommMonoid (G : Type u) extends SubtractionMonoid G, AddCommMonoid G /-- Commutative `DivisionMonoid`. This is the immediate common ancestor of `CommGroup` and `CommGroupWithZero`. -/ @[to_additive SubtractionCommMonoid] class DivisionCommMonoid (G : Type u) extends DivisionMonoid G, CommMonoid G attribute [to_additive existing] DivisionCommMonoid.toCommMonoid /-- A `Group` is a `Monoid` with an operation `⁻¹` satisfying `a⁻¹ * a = 1`. There is also a division operation `/` such that `a / b = a * b⁻¹`, with a default so that `a / b = a * b⁻¹` holds by definition. Use `Group.ofLeftAxioms` or `Group.ofRightAxioms` to define a group structure on a type with the minumum proof obligations. -/ class Group (G : Type u) extends DivInvMonoid G where protected mul_left_inv : ∀ a : G, a⁻¹ * a = 1 /-- An `AddGroup` is an `AddMonoid` with a unary `-` satisfying `-a + a = 0`. There is also a binary operation `-` such that `a - b = a + -b`, with a default so that `a - b = a + -b` holds by definition. Use `AddGroup.ofLeftAxioms` or `AddGroup.ofRightAxioms` to define an additive group structure on a type with the minumum proof obligations. -/ class AddGroup (A : Type u) extends SubNegMonoid A where protected add_left_neg : ∀ a : A, -a + a = 0 attribute [to_additive] Group section Group variable [Group G] {a b c : G} @[to_additive (attr := simp)] theorem mul_left_inv : ∀ a : G, a⁻¹ * a = 1 := Group.mul_left_inv @[to_additive] theorem inv_mul_self (a : G) : a⁻¹ * a = 1 := mul_left_inv a @[to_additive] private theorem inv_eq_of_mul (h : a * b = 1) : a⁻¹ = b := left_inv_eq_right_inv (inv_mul_self a) h @[to_additive (attr := simp)] theorem mul_right_inv (a : G) : a * a⁻¹ = 1 := by rw [← mul_left_inv a⁻¹, inv_eq_of_mul (mul_left_inv a)] @[to_additive] theorem mul_inv_self (a : G) : a * a⁻¹ = 1 := mul_right_inv a @[to_additive (attr := simp)] theorem inv_mul_cancel_left (a b : G) : a⁻¹ * (a * b) = b := by rw [← mul_assoc, mul_left_inv, one_mul] @[to_additive (attr := simp)] theorem mul_inv_cancel_left (a b : G) : a * (a⁻¹ * b) = b := by rw [← mul_assoc, mul_right_inv, one_mul] @[to_additive (attr := simp)] theorem mul_inv_cancel_right (a b : G) : a * b * b⁻¹ = a := by rw [mul_assoc, mul_right_inv, mul_one] @[to_additive (attr := simp)] theorem inv_mul_cancel_right (a b : G) : a * b⁻¹ * b = a := by rw [mul_assoc, mul_left_inv, mul_one] @[to_additive AddGroup.toSubtractionMonoid] instance (priority := 100) Group.toDivisionMonoid : DivisionMonoid G := { inv_inv := fun a ↦ inv_eq_of_mul (mul_left_inv a) mul_inv_rev := fun a b ↦ inv_eq_of_mul <| by rw [mul_assoc, mul_inv_cancel_left, mul_right_inv] inv_eq_of_mul := fun _ _ ↦ inv_eq_of_mul } -- see Note [lower instance priority] @[to_additive] instance (priority := 100) Group.toCancelMonoid : CancelMonoid G := { ‹Group G› with mul_right_cancel := fun a b c h ↦ by rw [← mul_inv_cancel_right a b, h, mul_inv_cancel_right] mul_left_cancel := fun a b c h ↦ by rw [← inv_mul_cancel_left a b, h, inv_mul_cancel_left] } end Group /-- An additive commutative group is an additive group with commutative `(+)`. -/ class AddCommGroup (G : Type u) extends AddGroup G, AddCommMonoid G /-- A commutative group is a group with commutative `(*)`. -/ @[to_additive] class CommGroup (G : Type u) extends Group G, CommMonoid G attribute [to_additive existing] CommGroup.toCommMonoid section CommGroup variable [CommGroup G] -- see Note [lower instance priority] @[to_additive] instance (priority := 100) CommGroup.toCancelCommMonoid : CancelCommMonoid G := { ‹CommGroup G›, Group.toCancelMonoid with } -- see Note [lower instance priority] @[to_additive] instance (priority := 100) CommGroup.toDivisionCommMonoid : DivisionCommMonoid G := { ‹CommGroup G›, Group.toDivisionMonoid with } @[to_additive (attr := simp)] lemma inv_mul_cancel_comm (a b : G) : a⁻¹ * b * a = b := by rw [mul_comm, mul_inv_cancel_left] @[to_additive (attr := simp)] lemma mul_inv_cancel_comm (a b : G) : a * b * a⁻¹ = b := by rw [mul_comm, inv_mul_cancel_left] @[to_additive (attr := simp)] lemma inv_mul_cancel_comm_assoc (a b : G) : a⁻¹ * (b * a) = b := by rw [mul_comm, mul_inv_cancel_right] @[to_additive (attr := simp)] lemma mul_inv_cancel_comm_assoc (a b : G) : a * (b * a⁻¹) = b := by rw [mul_comm, inv_mul_cancel_right] end CommGroup /-! We initialize all projections for `@[simps]` here, so that we don't have to do it in later files. Note: the lemmas generated for the `npow`/`zpow` projections will *not* apply to `x ^ y`, since the argument order of these projections doesn't match the argument order of `^`. The `nsmul`/`zsmul` lemmas will be correct. -/ initialize_simps_projections Semigroup initialize_simps_projections AddSemigroup initialize_simps_projections CommSemigroup initialize_simps_projections AddCommSemigroup initialize_simps_projections LeftCancelSemigroup initialize_simps_projections AddLeftCancelSemigroup initialize_simps_projections RightCancelSemigroup initialize_simps_projections AddRightCancelSemigroup initialize_simps_projections Monoid initialize_simps_projections AddMonoid initialize_simps_projections CommMonoid initialize_simps_projections AddCommMonoid initialize_simps_projections LeftCancelMonoid initialize_simps_projections AddLeftCancelMonoid initialize_simps_projections RightCancelMonoid initialize_simps_projections AddRightCancelMonoid initialize_simps_projections CancelMonoid initialize_simps_projections AddCancelMonoid initialize_simps_projections CancelCommMonoid initialize_simps_projections AddCancelCommMonoid initialize_simps_projections DivInvMonoid initialize_simps_projections SubNegMonoid initialize_simps_projections DivInvOneMonoid initialize_simps_projections SubNegZeroMonoid initialize_simps_projections DivisionMonoid initialize_simps_projections SubtractionMonoid initialize_simps_projections DivisionCommMonoid initialize_simps_projections SubtractionCommMonoid initialize_simps_projections Group initialize_simps_projections AddGroup initialize_simps_projections CommGroup initialize_simps_projections AddCommGroup assert_not_exists Function.Injective assert_not_exists IsCommutative
Algebra\Group\Embedding.lean
/- Copyright (c) 2021 Damiano Testa. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Damiano Testa -/ import Mathlib.Algebra.Group.Basic import Mathlib.Logic.Embedding.Basic /-! # The embedding of a cancellative semigroup into itself by multiplication by a fixed element. -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered variable {G : Type*} section LeftOrRightCancelSemigroup /-- If left-multiplication by any element is cancellative, left-multiplication by `g` is an embedding. -/ @[to_additive (attr := simps) "If left-addition by any element is cancellative, left-addition by `g` is an embedding."] def mulLeftEmbedding [Mul G] [IsLeftCancelMul G] (g : G) : G ↪ G where toFun h := g * h inj' := mul_right_injective g /-- If right-multiplication by any element is cancellative, right-multiplication by `g` is an embedding. -/ @[to_additive (attr := simps) "If right-addition by any element is cancellative, right-addition by `g` is an embedding."] def mulRightEmbedding [Mul G] [IsRightCancelMul G] (g : G) : G ↪ G where toFun h := h * g inj' := mul_left_injective g @[to_additive] theorem mulLeftEmbedding_eq_mulRightEmbedding [CommSemigroup G] [IsCancelMul G] (g : G) : mulLeftEmbedding g = mulRightEmbedding g := by ext exact mul_comm _ _ end LeftOrRightCancelSemigroup
Algebra\Group\Even.lean
/- Copyright (c) 2022 Damiano Testa. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Damiano Testa -/ import Mathlib.Algebra.Group.Opposite import Mathlib.Algebra.Group.TypeTags /-! # Squares and even elements This file defines square and even elements in a monoid. ## Main declarations * `IsSquare a` means that there is some `r` such that `a = r * r` * `Even a` means that there is some `r` such that `a = r + r` ## TODO * Try to generalize `IsSquare/Even` lemmas further. For example, there are still a few lemmas in `Algebra.Ring.Parity` whose `Semiring` assumptions I (DT) am not convinced are necessary. * The "old" definition of `Even a` asked for the existence of an element `c` such that `a = 2 * c`. For this reason, several fixes introduce an extra `two_mul` or `← two_mul`. It might be the case that by making a careful choice of `simp` lemma, this can be avoided. ## See also `Mathlib.Algebra.Ring.Parity` for the definition of odd elements. -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered open MulOpposite variable {F α β R : Type*} section Mul variable [Mul α] /-- An element `a` of a type `α` with multiplication satisfies `IsSquare a` if `a = r * r`, for some `r : α`. -/ @[to_additive "An element `a` of a type `α` with addition satisfies `Even a` if `a = r + r`, for some `r : α`."] def IsSquare (a : α) : Prop := ∃ r, a = r * r @[to_additive (attr := simp)] lemma isSquare_mul_self (m : α) : IsSquare (m * m) := ⟨m, rfl⟩ @[to_additive] lemma isSquare_op_iff {a : α} : IsSquare (op a) ↔ IsSquare a := ⟨fun ⟨c, hc⟩ ↦ ⟨unop c, congr_arg unop hc⟩, fun ⟨c, hc⟩ ↦ ⟨op c, congr_arg op hc⟩⟩ @[to_additive] lemma isSquare_unop_iff {a : αᵐᵒᵖ} : IsSquare (unop a) ↔ IsSquare a := isSquare_op_iff.symm @[to_additive] instance [DecidablePred (IsSquare : α → Prop)] : DecidablePred (IsSquare : αᵐᵒᵖ → Prop) := fun _ ↦ decidable_of_iff _ isSquare_unop_iff @[simp] lemma even_ofMul_iff {a : α} : Even (Additive.ofMul a) ↔ IsSquare a := Iff.rfl @[simp] lemma isSquare_toMul_iff {a : Additive α} : IsSquare (Additive.toMul a) ↔ Even a := Iff.rfl instance Additive.instDecidablePredEven [DecidablePred (IsSquare : α → Prop)] : DecidablePred (Even : Additive α → Prop) := fun _ ↦ decidable_of_iff _ isSquare_toMul_iff end Mul section Add variable [Add α] @[simp] lemma isSquare_ofAdd_iff {a : α} : IsSquare (Multiplicative.ofAdd a) ↔ Even a := Iff.rfl @[simp] lemma even_toAdd_iff {a : Multiplicative α} : Even (Multiplicative.toAdd a) ↔ IsSquare a := Iff.rfl instance Multiplicative.instDecidablePredIsSquare [DecidablePred (Even : α → Prop)] : DecidablePred (IsSquare : Multiplicative α → Prop) := fun _ ↦ decidable_of_iff _ even_toAdd_iff end Add @[to_additive (attr := simp)] lemma isSquare_one [MulOneClass α] : IsSquare (1 : α) := ⟨1, (mul_one _).symm⟩ @[to_additive] lemma IsSquare.map [MulOneClass α] [MulOneClass β] [FunLike F α β] [MonoidHomClass F α β] {m : α} (f : F) : IsSquare m → IsSquare (f m) := by rintro ⟨m, rfl⟩ exact ⟨f m, by simp⟩ section Monoid variable [Monoid α] {n : ℕ} {a : α} @[to_additive even_iff_exists_two_nsmul] lemma isSquare_iff_exists_sq (m : α) : IsSquare m ↔ ∃ c, m = c ^ 2 := by simp [IsSquare, pow_two] alias ⟨IsSquare.exists_sq, isSquare_of_exists_sq⟩ := isSquare_iff_exists_sq attribute [to_additive Even.exists_two_nsmul "Alias of the forwards direction of `even_iff_exists_two_nsmul`."] IsSquare.exists_sq @[to_additive] lemma IsSquare.pow (n : ℕ) : IsSquare a → IsSquare (a ^ n) := by rintro ⟨a, rfl⟩; exact ⟨a ^ n, (Commute.refl _).mul_pow _⟩ @[to_additive Even.nsmul'] lemma Even.isSquare_pow : Even n → ∀ a : α, IsSquare (a ^ n) := by rintro ⟨n, rfl⟩ a; exact ⟨a ^ n, pow_add _ _ _⟩ @[to_additive even_two_nsmul] lemma IsSquare_sq (a : α) : IsSquare (a ^ 2) := ⟨a, pow_two _⟩ end Monoid @[to_additive] lemma IsSquare.mul [CommSemigroup α] {a b : α} : IsSquare a → IsSquare b → IsSquare (a * b) := by rintro ⟨a, rfl⟩ ⟨b, rfl⟩; exact ⟨a * b, mul_mul_mul_comm _ _ _ _⟩ section DivisionMonoid variable [DivisionMonoid α] {a : α} @[to_additive (attr := simp)] lemma isSquare_inv : IsSquare a⁻¹ ↔ IsSquare a := by constructor <;> intro h · rw [← isSquare_op_iff, ← inv_inv a] exact h.map (MulEquiv.inv' α) · exact (isSquare_op_iff.mpr h).map (MulEquiv.inv' α).symm alias ⟨_, IsSquare.inv⟩ := isSquare_inv attribute [to_additive] IsSquare.inv @[to_additive] lemma IsSquare.zpow (n : ℤ) : IsSquare a → IsSquare (a ^ n) := by rintro ⟨a, rfl⟩; exact ⟨a ^ n, (Commute.refl _).mul_zpow _⟩ end DivisionMonoid @[to_additive] lemma IsSquare.div [DivisionCommMonoid α] {a b : α} (ha : IsSquare a) (hb : IsSquare b) : IsSquare (a / b) := by rw [div_eq_mul_inv]; exact ha.mul hb.inv @[to_additive (attr := simp) Even.zsmul'] lemma Even.isSquare_zpow [Group α] {n : ℤ} : Even n → ∀ a : α, IsSquare (a ^ n) := by rintro ⟨n, rfl⟩ a; exact ⟨a ^ n, zpow_add _ _ _⟩
Algebra\Group\Ext.lean
/- Copyright (c) 2021 Bryan Gin-ge Chen. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Bryan Gin-ge Chen, Yury Kudryashov -/ import Mathlib.Algebra.Group.Hom.Defs /-! # Extensionality lemmas for monoid and group structures In this file we prove extensionality lemmas for `Monoid` and higher algebraic structures with one binary operation. Extensionality lemmas for structures that are lower in the hierarchy can be found in `Algebra.Group.Defs`. ## Implementation details To get equality of `npow` etc, we define a monoid homomorphism between two monoid structures on the same type, then apply lemmas like `MonoidHom.map_div`, `MonoidHom.map_pow` etc. To refer to the `*` operator of a particular instance `i`, we use `(letI := i; HMul.hMul : M → M → M)` instead of `i.mul` (which elaborates to `Mul.mul`), as the former uses `HMul.hMul` which is the canonical spelling. ## Tags monoid, group, extensionality -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered open Function universe u @[to_additive (attr := ext)] theorem Monoid.ext {M : Type u} ⦃m₁ m₂ : Monoid M⦄ (h_mul : (letI := m₁; HMul.hMul : M → M → M) = (letI := m₂; HMul.hMul : M → M → M)) : m₁ = m₂ := by have : m₁.toMulOneClass = m₂.toMulOneClass := MulOneClass.ext h_mul have h₁ : m₁.one = m₂.one := congr_arg (·.one) this let f : @MonoidHom M M m₁.toMulOneClass m₂.toMulOneClass := @MonoidHom.mk _ _ (_) _ (@OneHom.mk _ _ (_) _ id h₁) (fun x y => congr_fun (congr_fun h_mul x) y) have : m₁.npow = m₂.npow := by ext n x exact @MonoidHom.map_pow M M m₁ m₂ f x n rcases m₁ with @⟨@⟨⟨_⟩⟩, ⟨_⟩⟩ rcases m₂ with @⟨@⟨⟨_⟩⟩, ⟨_⟩⟩ congr @[to_additive] theorem CommMonoid.toMonoid_injective {M : Type u} : Function.Injective (@CommMonoid.toMonoid M) := by rintro ⟨⟩ ⟨⟩ h congr @[to_additive (attr := ext)] theorem CommMonoid.ext {M : Type*} ⦃m₁ m₂ : CommMonoid M⦄ (h_mul : (letI := m₁; HMul.hMul : M → M → M) = (letI := m₂; HMul.hMul : M → M → M)) : m₁ = m₂ := CommMonoid.toMonoid_injective <| Monoid.ext h_mul @[to_additive] theorem LeftCancelMonoid.toMonoid_injective {M : Type u} : Function.Injective (@LeftCancelMonoid.toMonoid M) := by rintro @⟨@⟨⟩⟩ @⟨@⟨⟩⟩ h congr <;> injection h @[to_additive (attr := ext)] theorem LeftCancelMonoid.ext {M : Type u} ⦃m₁ m₂ : LeftCancelMonoid M⦄ (h_mul : (letI := m₁; HMul.hMul : M → M → M) = (letI := m₂; HMul.hMul : M → M → M)) : m₁ = m₂ := LeftCancelMonoid.toMonoid_injective <| Monoid.ext h_mul @[to_additive] theorem RightCancelMonoid.toMonoid_injective {M : Type u} : Function.Injective (@RightCancelMonoid.toMonoid M) := by rintro @⟨@⟨⟩⟩ @⟨@⟨⟩⟩ h congr <;> injection h @[to_additive (attr := ext)] theorem RightCancelMonoid.ext {M : Type u} ⦃m₁ m₂ : RightCancelMonoid M⦄ (h_mul : (letI := m₁; HMul.hMul : M → M → M) = (letI := m₂; HMul.hMul : M → M → M)) : m₁ = m₂ := RightCancelMonoid.toMonoid_injective <| Monoid.ext h_mul @[to_additive] theorem CancelMonoid.toLeftCancelMonoid_injective {M : Type u} : Function.Injective (@CancelMonoid.toLeftCancelMonoid M) := by rintro ⟨⟩ ⟨⟩ h congr @[to_additive (attr := ext)] theorem CancelMonoid.ext {M : Type*} ⦃m₁ m₂ : CancelMonoid M⦄ (h_mul : (letI := m₁; HMul.hMul : M → M → M) = (letI := m₂; HMul.hMul : M → M → M)) : m₁ = m₂ := CancelMonoid.toLeftCancelMonoid_injective <| LeftCancelMonoid.ext h_mul @[to_additive] theorem CancelCommMonoid.toCommMonoid_injective {M : Type u} : Function.Injective (@CancelCommMonoid.toCommMonoid M) := by rintro @⟨@⟨@⟨⟩⟩⟩ @⟨@⟨@⟨⟩⟩⟩ h congr <;> { injection h with h' injection h' } @[to_additive (attr := ext)] theorem CancelCommMonoid.ext {M : Type*} ⦃m₁ m₂ : CancelCommMonoid M⦄ (h_mul : (letI := m₁; HMul.hMul : M → M → M) = (letI := m₂; HMul.hMul : M → M → M)) : m₁ = m₂ := CancelCommMonoid.toCommMonoid_injective <| CommMonoid.ext h_mul @[to_additive (attr := ext)] theorem DivInvMonoid.ext {M : Type*} ⦃m₁ m₂ : DivInvMonoid M⦄ (h_mul : (letI := m₁; HMul.hMul : M → M → M) = (letI := m₂; HMul.hMul : M → M → M)) (h_inv : (letI := m₁; Inv.inv : M → M) = (letI := m₂; Inv.inv : M → M)) : m₁ = m₂ := by have h_mon := Monoid.ext h_mul have h₁ : m₁.one = m₂.one := congr_arg (·.one) h_mon let f : @MonoidHom M M m₁.toMulOneClass m₂.toMulOneClass := @MonoidHom.mk _ _ (_) _ (@OneHom.mk _ _ (_) _ id h₁) (fun x y => congr_fun (congr_fun h_mul x) y) have : m₁.npow = m₂.npow := congr_arg (·.npow) h_mon have : m₁.zpow = m₂.zpow := by ext m x exact @MonoidHom.map_zpow' M M m₁ m₂ f (congr_fun h_inv) x m have : m₁.div = m₂.div := by ext a b exact @map_div' _ _ (F := @MonoidHom _ _ (_) _) _ (id _) _ (@MonoidHom.instMonoidHomClass _ _ (_) _) f (congr_fun h_inv) a b rcases m₁ with @⟨_, ⟨_⟩, ⟨_⟩⟩ rcases m₂ with @⟨_, ⟨_⟩, ⟨_⟩⟩ congr @[to_additive] lemma Group.toDivInvMonoid_injective {G : Type*} : Injective (@Group.toDivInvMonoid G) := by rintro ⟨⟩ ⟨⟩ ⟨⟩; rfl @[to_additive (attr := ext)] theorem Group.ext {G : Type*} ⦃g₁ g₂ : Group G⦄ (h_mul : g₁.mul = g₂.mul) : g₁ = g₂ := by have h₁ : g₁.one = g₂.one := congr_arg (·.one) (Monoid.ext h_mul) let f : @MonoidHom G G g₁.toMulOneClass g₂.toMulOneClass := @MonoidHom.mk _ _ (_) _ (@OneHom.mk _ _ (_) _ id h₁) (fun x y => congr_fun (congr_fun h_mul x) y) exact Group.toDivInvMonoid_injective (DivInvMonoid.ext h_mul (funext <| @MonoidHom.map_inv G G g₁ g₂.toDivisionMonoid f)) @[to_additive] lemma CommGroup.toGroup_injective {G : Type*} : Injective (@CommGroup.toGroup G) := by rintro ⟨⟩ ⟨⟩ ⟨⟩; rfl @[to_additive (attr := ext)] theorem CommGroup.ext {G : Type*} ⦃g₁ g₂ : CommGroup G⦄ (h_mul : g₁.mul = g₂.mul) : g₁ = g₂ := CommGroup.toGroup_injective <| Group.ext h_mul
Algebra\Group\FiniteSupport.lean
/- Copyright (c) 2021 Oliver Nash. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Oliver Nash -/ import Mathlib.Algebra.Group.Support import Mathlib.Data.Set.Finite /-! # Finiteness of support -/ namespace Function variable {α β γ : Type*} [One γ] @[to_additive (attr := simp)] lemma mulSupport_along_fiber_finite_of_finite (f : α × β → γ) (a : α) (h : (mulSupport f).Finite) : (mulSupport fun b ↦ f (a, b)).Finite := (h.image Prod.snd).subset (mulSupport_along_fiber_subset f a) end Function
Algebra\Group\Indicator.lean
/- Copyright (c) 2020 Zhouhang Zhou. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Zhouhang Zhou -/ import Mathlib.Algebra.Group.Pi.Lemmas import Mathlib.Algebra.Group.Support /-! # Indicator function - `Set.indicator (s : Set α) (f : α → β) (a : α)` is `f a` if `a ∈ s` and is `0` otherwise. - `Set.mulIndicator (s : Set α) (f : α → β) (a : α)` is `f a` if `a ∈ s` and is `1` otherwise. ## Implementation note In mathematics, an indicator function or a characteristic function is a function used to indicate membership of an element in a set `s`, having the value `1` for all elements of `s` and the value `0` otherwise. But since it is usually used to restrict a function to a certain set `s`, we let the indicator function take the value `f x` for some function `f`, instead of `1`. If the usual indicator function is needed, just set `f` to be the constant function `fun _ ↦ 1`. The indicator function is implemented non-computably, to avoid having to pass around `Decidable` arguments. This is in contrast with the design of `Pi.single` or `Set.piecewise`. ## Tags indicator, characteristic -/ assert_not_exists MonoidWithZero open Function variable {α β ι M N : Type*} namespace Set section One variable [One M] [One N] {s t : Set α} {f g : α → M} {a : α} /-- `Set.mulIndicator s f a` is `f a` if `a ∈ s`, `1` otherwise. -/ @[to_additive "`Set.indicator s f a` is `f a` if `a ∈ s`, `0` otherwise."] noncomputable def mulIndicator (s : Set α) (f : α → M) (x : α) : M := haveI := Classical.decPred (· ∈ s) if x ∈ s then f x else 1 @[to_additive (attr := simp)] theorem piecewise_eq_mulIndicator [DecidablePred (· ∈ s)] : s.piecewise f 1 = s.mulIndicator f := funext fun _ => @if_congr _ _ _ _ (id _) _ _ _ _ Iff.rfl rfl rfl -- Porting note: needed unfold for mulIndicator @[to_additive] theorem mulIndicator_apply (s : Set α) (f : α → M) (a : α) [Decidable (a ∈ s)] : mulIndicator s f a = if a ∈ s then f a else 1 := by unfold mulIndicator congr @[to_additive (attr := simp)] theorem mulIndicator_of_mem (h : a ∈ s) (f : α → M) : mulIndicator s f a = f a := if_pos h @[to_additive (attr := simp)] theorem mulIndicator_of_not_mem (h : a ∉ s) (f : α → M) : mulIndicator s f a = 1 := if_neg h @[to_additive] theorem mulIndicator_eq_one_or_self (s : Set α) (f : α → M) (a : α) : mulIndicator s f a = 1 ∨ mulIndicator s f a = f a := by by_cases h : a ∈ s · exact Or.inr (mulIndicator_of_mem h f) · exact Or.inl (mulIndicator_of_not_mem h f) @[to_additive (attr := simp)] theorem mulIndicator_apply_eq_self : s.mulIndicator f a = f a ↔ a ∉ s → f a = 1 := letI := Classical.dec (a ∈ s) ite_eq_left_iff.trans (by rw [@eq_comm _ (f a)]) @[to_additive (attr := simp)] theorem mulIndicator_eq_self : s.mulIndicator f = f ↔ mulSupport f ⊆ s := by simp only [funext_iff, subset_def, mem_mulSupport, mulIndicator_apply_eq_self, not_imp_comm] @[to_additive] theorem mulIndicator_eq_self_of_superset (h1 : s.mulIndicator f = f) (h2 : s ⊆ t) : t.mulIndicator f = f := by rw [mulIndicator_eq_self] at h1 ⊢ exact Subset.trans h1 h2 @[to_additive (attr := simp)] theorem mulIndicator_apply_eq_one : mulIndicator s f a = 1 ↔ a ∈ s → f a = 1 := letI := Classical.dec (a ∈ s) ite_eq_right_iff @[to_additive (attr := simp)] theorem mulIndicator_eq_one : (mulIndicator s f = fun x => 1) ↔ Disjoint (mulSupport f) s := by simp only [funext_iff, mulIndicator_apply_eq_one, Set.disjoint_left, mem_mulSupport, not_imp_not] @[to_additive (attr := simp)] theorem mulIndicator_eq_one' : mulIndicator s f = 1 ↔ Disjoint (mulSupport f) s := mulIndicator_eq_one @[to_additive] theorem mulIndicator_apply_ne_one {a : α} : s.mulIndicator f a ≠ 1 ↔ a ∈ s ∩ mulSupport f := by simp only [Ne, mulIndicator_apply_eq_one, Classical.not_imp, mem_inter_iff, mem_mulSupport] @[to_additive (attr := simp)] theorem mulSupport_mulIndicator : Function.mulSupport (s.mulIndicator f) = s ∩ Function.mulSupport f := ext fun x => by simp [Function.mem_mulSupport, mulIndicator_apply_eq_one] /-- If a multiplicative indicator function is not equal to `1` at a point, then that point is in the set. -/ @[to_additive "If an additive indicator function is not equal to `0` at a point, then that point is in the set."] theorem mem_of_mulIndicator_ne_one (h : mulIndicator s f a ≠ 1) : a ∈ s := not_imp_comm.1 (fun hn => mulIndicator_of_not_mem hn f) h @[to_additive] theorem eqOn_mulIndicator : EqOn (mulIndicator s f) f s := fun _ hx => mulIndicator_of_mem hx f @[to_additive] theorem mulSupport_mulIndicator_subset : mulSupport (s.mulIndicator f) ⊆ s := fun _ hx => hx.imp_symm fun h => mulIndicator_of_not_mem h f @[to_additive (attr := simp)] theorem mulIndicator_mulSupport : mulIndicator (mulSupport f) f = f := mulIndicator_eq_self.2 Subset.rfl @[to_additive (attr := simp)] theorem mulIndicator_range_comp {ι : Sort*} (f : ι → α) (g : α → M) : mulIndicator (range f) g ∘ f = g ∘ f := letI := Classical.decPred (· ∈ range f) piecewise_range_comp _ _ _ @[to_additive] theorem mulIndicator_congr (h : EqOn f g s) : mulIndicator s f = mulIndicator s g := funext fun x => by simp only [mulIndicator] split_ifs with h_1 · exact h h_1 rfl @[to_additive (attr := simp)] theorem mulIndicator_univ (f : α → M) : mulIndicator (univ : Set α) f = f := mulIndicator_eq_self.2 <| subset_univ _ @[to_additive (attr := simp)] theorem mulIndicator_empty (f : α → M) : mulIndicator (∅ : Set α) f = fun _ => 1 := mulIndicator_eq_one.2 <| disjoint_empty _ @[to_additive] theorem mulIndicator_empty' (f : α → M) : mulIndicator (∅ : Set α) f = 1 := mulIndicator_empty f variable (M) @[to_additive (attr := simp)] theorem mulIndicator_one (s : Set α) : (mulIndicator s fun _ => (1 : M)) = fun _ => (1 : M) := mulIndicator_eq_one.2 <| by simp only [mulSupport_one, empty_disjoint] @[to_additive (attr := simp)] theorem mulIndicator_one' {s : Set α} : s.mulIndicator (1 : α → M) = 1 := mulIndicator_one M s variable {M} @[to_additive] theorem mulIndicator_mulIndicator (s t : Set α) (f : α → M) : mulIndicator s (mulIndicator t f) = mulIndicator (s ∩ t) f := funext fun x => by simp only [mulIndicator] split_ifs <;> simp_all (config := { contextual := true }) @[to_additive (attr := simp)] theorem mulIndicator_inter_mulSupport (s : Set α) (f : α → M) : mulIndicator (s ∩ mulSupport f) f = mulIndicator s f := by rw [← mulIndicator_mulIndicator, mulIndicator_mulSupport] @[to_additive] theorem comp_mulIndicator (h : M → β) (f : α → M) {s : Set α} {x : α} [DecidablePred (· ∈ s)] : h (s.mulIndicator f x) = s.piecewise (h ∘ f) (const α (h 1)) x := by letI := Classical.decPred (· ∈ s) convert s.apply_piecewise f (const α 1) (fun _ => h) (x := x) using 2 @[to_additive] theorem mulIndicator_comp_right {s : Set α} (f : β → α) {g : α → M} {x : β} : mulIndicator (f ⁻¹' s) (g ∘ f) x = mulIndicator s g (f x) := by simp only [mulIndicator, Function.comp] split_ifs with h h' h'' <;> first | rfl | contradiction @[to_additive] theorem mulIndicator_image {s : Set α} {f : β → M} {g : α → β} (hg : Injective g) {x : α} : mulIndicator (g '' s) f (g x) = mulIndicator s (f ∘ g) x := by rw [← mulIndicator_comp_right, preimage_image_eq _ hg] @[to_additive] theorem mulIndicator_comp_of_one {g : M → N} (hg : g 1 = 1) : mulIndicator s (g ∘ f) = g ∘ mulIndicator s f := by funext simp only [mulIndicator] split_ifs <;> simp [*] @[to_additive] theorem comp_mulIndicator_const (c : M) (f : M → N) (hf : f 1 = 1) : (fun x => f (s.mulIndicator (fun _ => c) x)) = s.mulIndicator fun _ => f c := (mulIndicator_comp_of_one hf).symm @[to_additive] theorem mulIndicator_preimage (s : Set α) (f : α → M) (B : Set M) : mulIndicator s f ⁻¹' B = s.ite (f ⁻¹' B) (1 ⁻¹' B) := letI := Classical.decPred (· ∈ s) piecewise_preimage s f 1 B @[to_additive] theorem mulIndicator_one_preimage (s : Set M) : t.mulIndicator 1 ⁻¹' s ∈ ({Set.univ, ∅} : Set (Set α)) := by classical rw [mulIndicator_one', preimage_one] split_ifs <;> simp @[to_additive] theorem mulIndicator_const_preimage_eq_union (U : Set α) (s : Set M) (a : M) [Decidable (a ∈ s)] [Decidable ((1 : M) ∈ s)] : (U.mulIndicator fun _ => a) ⁻¹' s = (if a ∈ s then U else ∅) ∪ if (1 : M) ∈ s then Uᶜ else ∅ := by rw [mulIndicator_preimage, preimage_one, preimage_const] split_ifs <;> simp [← compl_eq_univ_diff] @[to_additive] theorem mulIndicator_const_preimage (U : Set α) (s : Set M) (a : M) : (U.mulIndicator fun _ => a) ⁻¹' s ∈ ({Set.univ, U, Uᶜ, ∅} : Set (Set α)) := by classical rw [mulIndicator_const_preimage_eq_union] split_ifs <;> simp theorem indicator_one_preimage [Zero M] (U : Set α) (s : Set M) : U.indicator 1 ⁻¹' s ∈ ({Set.univ, U, Uᶜ, ∅} : Set (Set α)) := indicator_const_preimage _ _ 1 @[to_additive] theorem mulIndicator_preimage_of_not_mem (s : Set α) (f : α → M) {t : Set M} (ht : (1 : M) ∉ t) : mulIndicator s f ⁻¹' t = f ⁻¹' t ∩ s := by simp [mulIndicator_preimage, Pi.one_def, Set.preimage_const_of_not_mem ht] @[to_additive] theorem mem_range_mulIndicator {r : M} {s : Set α} {f : α → M} : r ∈ range (mulIndicator s f) ↔ r = 1 ∧ s ≠ univ ∨ r ∈ f '' s := by simp [mulIndicator, ite_eq_iff, exists_or, eq_univ_iff_forall, and_comm, or_comm, @eq_comm _ r 1] @[to_additive] theorem mulIndicator_rel_mulIndicator {r : M → M → Prop} (h1 : r 1 1) (ha : a ∈ s → r (f a) (g a)) : r (mulIndicator s f a) (mulIndicator s g a) := by simp only [mulIndicator] split_ifs with has exacts [ha has, h1] end One section Monoid variable [MulOneClass M] {s t : Set α} {f g : α → M} {a : α} @[to_additive] theorem mulIndicator_union_mul_inter_apply (f : α → M) (s t : Set α) (a : α) : mulIndicator (s ∪ t) f a * mulIndicator (s ∩ t) f a = mulIndicator s f a * mulIndicator t f a := by by_cases hs : a ∈ s <;> by_cases ht : a ∈ t <;> simp [*] @[to_additive] theorem mulIndicator_union_mul_inter (f : α → M) (s t : Set α) : mulIndicator (s ∪ t) f * mulIndicator (s ∩ t) f = mulIndicator s f * mulIndicator t f := funext <| mulIndicator_union_mul_inter_apply f s t @[to_additive] theorem mulIndicator_union_of_not_mem_inter (h : a ∉ s ∩ t) (f : α → M) : mulIndicator (s ∪ t) f a = mulIndicator s f a * mulIndicator t f a := by rw [← mulIndicator_union_mul_inter_apply f s t, mulIndicator_of_not_mem h, mul_one] @[to_additive] theorem mulIndicator_union_of_disjoint (h : Disjoint s t) (f : α → M) : mulIndicator (s ∪ t) f = fun a => mulIndicator s f a * mulIndicator t f a := funext fun _ => mulIndicator_union_of_not_mem_inter (fun ha => h.le_bot ha) _ open scoped symmDiff in @[to_additive] theorem mulIndicator_symmDiff (s t : Set α) (f : α → M) : mulIndicator (s ∆ t) f = mulIndicator (s \ t) f * mulIndicator (t \ s) f := mulIndicator_union_of_disjoint (disjoint_sdiff_self_right.mono_left sdiff_le) _ @[to_additive] theorem mulIndicator_mul (s : Set α) (f g : α → M) : (mulIndicator s fun a => f a * g a) = fun a => mulIndicator s f a * mulIndicator s g a := by funext simp only [mulIndicator] split_ifs · rfl rw [mul_one] @[to_additive] theorem mulIndicator_mul' (s : Set α) (f g : α → M) : mulIndicator s (f * g) = mulIndicator s f * mulIndicator s g := mulIndicator_mul s f g @[to_additive (attr := simp)] theorem mulIndicator_compl_mul_self_apply (s : Set α) (f : α → M) (a : α) : mulIndicator sᶜ f a * mulIndicator s f a = f a := by_cases (fun ha : a ∈ s => by simp [ha]) fun ha => by simp [ha] @[to_additive (attr := simp)] theorem mulIndicator_compl_mul_self (s : Set α) (f : α → M) : mulIndicator sᶜ f * mulIndicator s f = f := funext <| mulIndicator_compl_mul_self_apply s f @[to_additive (attr := simp)] theorem mulIndicator_self_mul_compl_apply (s : Set α) (f : α → M) (a : α) : mulIndicator s f a * mulIndicator sᶜ f a = f a := by_cases (fun ha : a ∈ s => by simp [ha]) fun ha => by simp [ha] @[to_additive (attr := simp)] theorem mulIndicator_self_mul_compl (s : Set α) (f : α → M) : mulIndicator s f * mulIndicator sᶜ f = f := funext <| mulIndicator_self_mul_compl_apply s f @[to_additive] theorem mulIndicator_mul_eq_left {f g : α → M} (h : Disjoint (mulSupport f) (mulSupport g)) : (mulSupport f).mulIndicator (f * g) = f := by refine (mulIndicator_congr fun x hx => ?_).trans mulIndicator_mulSupport have : g x = 1 := nmem_mulSupport.1 (disjoint_left.1 h hx) rw [Pi.mul_apply, this, mul_one] @[to_additive] theorem mulIndicator_mul_eq_right {f g : α → M} (h : Disjoint (mulSupport f) (mulSupport g)) : (mulSupport g).mulIndicator (f * g) = g := by refine (mulIndicator_congr fun x hx => ?_).trans mulIndicator_mulSupport have : f x = 1 := nmem_mulSupport.1 (disjoint_right.1 h hx) rw [Pi.mul_apply, this, one_mul] @[to_additive] theorem mulIndicator_mul_compl_eq_piecewise [DecidablePred (· ∈ s)] (f g : α → M) : s.mulIndicator f * sᶜ.mulIndicator g = s.piecewise f g := by ext x by_cases h : x ∈ s · rw [piecewise_eq_of_mem _ _ _ h, Pi.mul_apply, Set.mulIndicator_of_mem h, Set.mulIndicator_of_not_mem (Set.not_mem_compl_iff.2 h), mul_one] · rw [piecewise_eq_of_not_mem _ _ _ h, Pi.mul_apply, Set.mulIndicator_of_not_mem h, Set.mulIndicator_of_mem (Set.mem_compl h), one_mul] /-- `Set.mulIndicator` as a `monoidHom`. -/ @[to_additive "`Set.indicator` as an `addMonoidHom`."] noncomputable def mulIndicatorHom {α} (M) [MulOneClass M] (s : Set α) : (α → M) →* α → M where toFun := mulIndicator s map_one' := mulIndicator_one M s map_mul' := mulIndicator_mul s end Monoid section Group variable {G : Type*} [Group G] {s t : Set α} {f g : α → G} {a : α} @[to_additive] theorem mulIndicator_inv' (s : Set α) (f : α → G) : mulIndicator s f⁻¹ = (mulIndicator s f)⁻¹ := (mulIndicatorHom G s).map_inv f @[to_additive] theorem mulIndicator_inv (s : Set α) (f : α → G) : (mulIndicator s fun a => (f a)⁻¹) = fun a => (mulIndicator s f a)⁻¹ := mulIndicator_inv' s f @[to_additive] theorem mulIndicator_div (s : Set α) (f g : α → G) : (mulIndicator s fun a => f a / g a) = fun a => mulIndicator s f a / mulIndicator s g a := (mulIndicatorHom G s).map_div f g @[to_additive] theorem mulIndicator_div' (s : Set α) (f g : α → G) : mulIndicator s (f / g) = mulIndicator s f / mulIndicator s g := mulIndicator_div s f g @[to_additive indicator_compl'] theorem mulIndicator_compl (s : Set α) (f : α → G) : mulIndicator sᶜ f = f * (mulIndicator s f)⁻¹ := eq_mul_inv_of_mul_eq <| s.mulIndicator_compl_mul_self f @[to_additive indicator_compl] theorem mulIndicator_compl' (s : Set α) (f : α → G) : mulIndicator sᶜ f = f / mulIndicator s f := by rw [div_eq_mul_inv, mulIndicator_compl] @[to_additive indicator_diff'] theorem mulIndicator_diff (h : s ⊆ t) (f : α → G) : mulIndicator (t \ s) f = mulIndicator t f * (mulIndicator s f)⁻¹ := eq_mul_inv_of_mul_eq <| by rw [Pi.mul_def, ← mulIndicator_union_of_disjoint, diff_union_self, union_eq_self_of_subset_right h] exact disjoint_sdiff_self_left @[to_additive indicator_diff] theorem mulIndicator_diff' (h : s ⊆ t) (f : α → G) : mulIndicator (t \ s) f = mulIndicator t f / mulIndicator s f := by rw [mulIndicator_diff h, div_eq_mul_inv] open scoped symmDiff in @[to_additive] theorem apply_mulIndicator_symmDiff {g : G → β} (hg : ∀ x, g x⁻¹ = g x) (s t : Set α) (f : α → G) (x : α) : g (mulIndicator (s ∆ t) f x) = g (mulIndicator s f x / mulIndicator t f x) := by by_cases hs : x ∈ s <;> by_cases ht : x ∈ t <;> simp [mem_symmDiff, *] end Group end Set @[to_additive] theorem MonoidHom.map_mulIndicator {M N : Type*} [MulOneClass M] [MulOneClass N] (f : M →* N) (s : Set α) (g : α → M) (x : α) : f (s.mulIndicator g x) = s.mulIndicator (f ∘ g) x := by simp [Set.mulIndicator_comp_of_one]
Algebra\Group\InjSurj.lean
/- Copyright (c) 2020 Johan Commelin. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Johan Commelin -/ import Mathlib.Algebra.Group.Defs import Mathlib.Logic.Function.Basic import Mathlib.Data.Int.Cast.Basic import Mathlib.Tactic.Spread /-! # Lifting algebraic data classes along injective/surjective maps This file provides definitions that are meant to deal with situations such as the following: Suppose that `G` is a group, and `H` is a type endowed with `One H`, `Mul H`, and `Inv H`. Suppose furthermore, that `f : G → H` is a surjective map that respects the multiplication, and the unit elements. Then `H` satisfies the group axioms. The relevant definition in this case is `Function.Surjective.group`. Dually, there is also `Function.Injective.group`. And there are versions for (additive) (commutative) semigroups/monoids. ## Implementation note The `nsmul` and `zsmul` assumptions on any tranfer definition for an algebraic structure involving both addition and multiplication (eg `AddMonoidWithOne`) is `∀ n x, f (n • x) = n • f x`, which is what we would expect. However, we cannot do the same for transfer definitions built using `to_additive` (eg `AddMonoid`) as we want the multiplicative versions to be `∀ x n, f (x ^ n) = f x ^ n`. As a result, we must use `Function.swap` when using additivised transfer definitions in non-additivised ones. -/ namespace Function /-! ### Injective -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered namespace Injective variable {M₁ : Type*} {M₂ : Type*} [Mul M₁] /-- A type endowed with `*` is a semigroup, if it admits an injective map that preserves `*` to a semigroup. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `+` is an additive semigroup, if it admits an injective map that preserves `+` to an additive semigroup."] protected def semigroup [Semigroup M₂] (f : M₁ → M₂) (hf : Injective f) (mul : ∀ x y, f (x * y) = f x * f y) : Semigroup M₁ := { ‹Mul M₁› with mul_assoc := fun x y z => hf <| by erw [mul, mul, mul, mul, mul_assoc] } /-- A type endowed with `*` is a commutative magma, if it admits a surjective map that preserves `*` from a commutative magma. -/ @[to_additive (attr := reducible) -- See note [reducible non-instances] "A type endowed with `+` is an additive commutative semigroup, if it admits a surjective map that preserves `+` from an additive commutative semigroup."] protected def commMagma [CommMagma M₂] (f : M₁ → M₂) (hf : Injective f) (mul : ∀ x y, f (x * y) = f x * f y) : CommMagma M₁ where mul_comm x y := hf <| by rw [mul, mul, mul_comm] /-- A type endowed with `*` is a commutative semigroup, if it admits an injective map that preserves `*` to a commutative semigroup. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `+` is an additive commutative semigroup,if it admits an injective map that preserves `+` to an additive commutative semigroup."] protected def commSemigroup [CommSemigroup M₂] (f : M₁ → M₂) (hf : Injective f) (mul : ∀ x y, f (x * y) = f x * f y) : CommSemigroup M₁ where toSemigroup := hf.semigroup f mul __ := hf.commMagma f mul /-- A type endowed with `*` is a left cancel semigroup, if it admits an injective map that preserves `*` to a left cancel semigroup. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `+` is an additive left cancel semigroup, if it admits an injective map that preserves `+` to an additive left cancel semigroup."] protected def leftCancelSemigroup [LeftCancelSemigroup M₂] (f : M₁ → M₂) (hf : Injective f) (mul : ∀ x y, f (x * y) = f x * f y) : LeftCancelSemigroup M₁ := { hf.semigroup f mul with mul_left_cancel := fun x y z H => hf <| (mul_right_inj (f x)).1 <| by erw [← mul, ← mul, H] } /-- A type endowed with `*` is a right cancel semigroup, if it admits an injective map that preserves `*` to a right cancel semigroup. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `+` is an additive right cancel semigroup, if it admits an injective map that preserves `+` to an additive right cancel semigroup."] protected def rightCancelSemigroup [RightCancelSemigroup M₂] (f : M₁ → M₂) (hf : Injective f) (mul : ∀ x y, f (x * y) = f x * f y) : RightCancelSemigroup M₁ := { hf.semigroup f mul with mul_right_cancel := fun x y z H => hf <| (mul_left_inj (f y)).1 <| by erw [← mul, ← mul, H] } variable [One M₁] /-- A type endowed with `1` and `*` is a `MulOneClass`, if it admits an injective map that preserves `1` and `*` to a `MulOneClass`. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `0` and `+` is an `AddZeroClass`, if it admits an injective map that preserves `0` and `+` to an `AddZeroClass`."] protected def mulOneClass [MulOneClass M₂] (f : M₁ → M₂) (hf : Injective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) : MulOneClass M₁ := { ‹One M₁›, ‹Mul M₁› with one_mul := fun x => hf <| by erw [mul, one, one_mul], mul_one := fun x => hf <| by erw [mul, one, mul_one] } variable [Pow M₁ ℕ] /-- A type endowed with `1` and `*` is a monoid, if it admits an injective map that preserves `1` and `*` to a monoid. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `0` and `+` is an additive monoid, if it admits an injective map that preserves `0` and `+` to an additive monoid. See note [reducible non-instances]."] protected def monoid [Monoid M₂] (f : M₁ → M₂) (hf : Injective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) : Monoid M₁ := { hf.mulOneClass f one mul, hf.semigroup f mul with npow := fun n x => x ^ n, npow_zero := fun x => hf <| by erw [npow, one, pow_zero], npow_succ := fun n x => hf <| by erw [npow, pow_succ, mul, npow] } /-- A type endowed with `0`, `1` and `+` is an additive monoid with one, if it admits an injective map that preserves `0`, `1` and `+` to an additive monoid with one. See note [reducible non-instances]. -/ protected abbrev addMonoidWithOne {M₁} [Zero M₁] [One M₁] [Add M₁] [SMul ℕ M₁] [NatCast M₁] [AddMonoidWithOne M₂] (f : M₁ → M₂) (hf : Injective f) (zero : f 0 = 0) (one : f 1 = 1) (add : ∀ x y, f (x + y) = f x + f y) (nsmul : ∀ (n : ℕ) (x), f (n • x) = n • f x) (natCast : ∀ n : ℕ, f n = n) : AddMonoidWithOne M₁ := { hf.addMonoid f zero add (swap nsmul) with natCast := Nat.cast, natCast_zero := hf (by erw [natCast, Nat.cast_zero, zero]), natCast_succ := fun n => hf (by erw [natCast, Nat.cast_succ, add, one, natCast]), one := 1 } /-- A type endowed with `1` and `*` is a left cancel monoid, if it admits an injective map that preserves `1` and `*` to a left cancel monoid. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `0` and `+` is an additive left cancel monoid, if it admits an injective map that preserves `0` and `+` to an additive left cancel monoid."] protected def leftCancelMonoid [LeftCancelMonoid M₂] (f : M₁ → M₂) (hf : Injective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) : LeftCancelMonoid M₁ := { hf.leftCancelSemigroup f mul, hf.monoid f one mul npow with } /-- A type endowed with `1` and `*` is a right cancel monoid, if it admits an injective map that preserves `1` and `*` to a right cancel monoid. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `0` and `+` is an additive left cancel monoid,if it admits an injective map that preserves `0` and `+` to an additive left cancel monoid."] protected def rightCancelMonoid [RightCancelMonoid M₂] (f : M₁ → M₂) (hf : Injective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) : RightCancelMonoid M₁ := { hf.rightCancelSemigroup f mul, hf.monoid f one mul npow with } /-- A type endowed with `1` and `*` is a cancel monoid, if it admits an injective map that preserves `1` and `*` to a cancel monoid. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `0` and `+` is an additive left cancel monoid,if it admits an injective map that preserves `0` and `+` to an additive left cancel monoid."] protected def cancelMonoid [CancelMonoid M₂] (f : M₁ → M₂) (hf : Injective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) : CancelMonoid M₁ := { hf.leftCancelMonoid f one mul npow, hf.rightCancelMonoid f one mul npow with } /-- A type endowed with `1` and `*` is a commutative monoid, if it admits an injective map that preserves `1` and `*` to a commutative monoid. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `0` and `+` is an additive commutative monoid, if it admits an injective map that preserves `0` and `+` to an additive commutative monoid."] protected def commMonoid [CommMonoid M₂] (f : M₁ → M₂) (hf : Injective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) : CommMonoid M₁ := { hf.monoid f one mul npow, hf.commSemigroup f mul with } /-- A type endowed with `0`, `1` and `+` is an additive commutative monoid with one, if it admits an injective map that preserves `0`, `1` and `+` to an additive commutative monoid with one. See note [reducible non-instances]. -/ protected abbrev addCommMonoidWithOne {M₁} [Zero M₁] [One M₁] [Add M₁] [SMul ℕ M₁] [NatCast M₁] [AddCommMonoidWithOne M₂] (f : M₁ → M₂) (hf : Injective f) (zero : f 0 = 0) (one : f 1 = 1) (add : ∀ x y, f (x + y) = f x + f y) (nsmul : ∀ (n : ℕ) (x), f (n • x) = n • f x) (natCast : ∀ n : ℕ, f n = n) : AddCommMonoidWithOne M₁ where __ := hf.addMonoidWithOne f zero one add nsmul natCast __ := hf.addCommMonoid _ zero add (swap nsmul) /-- A type endowed with `1` and `*` is a cancel commutative monoid, if it admits an injective map that preserves `1` and `*` to a cancel commutative monoid. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `0` and `+` is an additive cancel commutative monoid, if it admits an injective map that preserves `0` and `+` to an additive cancel commutative monoid."] protected def cancelCommMonoid [CancelCommMonoid M₂] (f : M₁ → M₂) (hf : Injective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) : CancelCommMonoid M₁ := { hf.leftCancelSemigroup f mul, hf.commMonoid f one mul npow with } /-- A type has an involutive inversion if it admits a surjective map that preserves `⁻¹` to a type which has an involutive inversion. See note [reducible non-instances] -/ @[to_additive (attr := reducible) "A type has an involutive negation if it admits a surjective map that preserves `-` to a type which has an involutive negation."] protected def involutiveInv {M₁ : Type*} [Inv M₁] [InvolutiveInv M₂] (f : M₁ → M₂) (hf : Injective f) (inv : ∀ x, f x⁻¹ = (f x)⁻¹) : InvolutiveInv M₁ where inv := Inv.inv inv_inv x := hf <| by rw [inv, inv, inv_inv] variable [Inv M₁] /-- A type endowed with `1` and `⁻¹` is a `InvOneClass`, if it admits an injective map that preserves `1` and `⁻¹` to a `InvOneClass`. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `0` and unary `-` is an `NegZeroClass`, if it admits an injective map that preserves `0` and unary `-` to an `NegZeroClass`."] protected def invOneClass [InvOneClass M₂] (f : M₁ → M₂) (hf : Injective f) (one : f 1 = 1) (inv : ∀ x, f (x⁻¹) = (f x)⁻¹) : InvOneClass M₁ := { ‹One M₁›, ‹Inv M₁› with inv_one := hf <| by erw [inv, one, inv_one] } variable [Div M₁] [Pow M₁ ℤ] /-- A type endowed with `1`, `*`, `⁻¹`, and `/` is a `DivInvMonoid` if it admits an injective map that preserves `1`, `*`, `⁻¹`, and `/` to a `DivInvMonoid`. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) subNegMonoid "A type endowed with `0`, `+`, unary `-`, and binary `-` is a `SubNegMonoid` if it admits an injective map that preserves `0`, `+`, unary `-`, and binary `-` to a `SubNegMonoid`. This version takes custom `nsmul` and `zsmul` as `[SMul ℕ M₁]` and `[SMul ℤ M₁]` arguments."] protected def divInvMonoid [DivInvMonoid M₂] (f : M₁ → M₂) (hf : Injective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) (inv : ∀ x, f x⁻¹ = (f x)⁻¹) (div : ∀ x y, f (x / y) = f x / f y) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) (zpow : ∀ (x) (n : ℤ), f (x ^ n) = f x ^ n) : DivInvMonoid M₁ := { hf.monoid f one mul npow, ‹Inv M₁›, ‹Div M₁› with zpow := fun n x => x ^ n, zpow_zero' := fun x => hf <| by erw [zpow, zpow_zero, one], zpow_succ' := fun n x => hf <| by erw [zpow, mul, zpow_natCast, pow_succ, zpow, zpow_natCast], zpow_neg' := fun n x => hf <| by erw [zpow, zpow_negSucc, inv, zpow, zpow_natCast], div_eq_mul_inv := fun x y => hf <| by erw [div, mul, inv, div_eq_mul_inv] } /-- A type endowed with `1`, `*`, `⁻¹`, and `/` is a `DivInvOneMonoid` if it admits an injective map that preserves `1`, `*`, `⁻¹`, and `/` to a `DivInvOneMonoid`. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) subNegZeroMonoid "A type endowed with `0`, `+`, unary `-`, and binary `-` is a `SubNegZeroMonoid` if it admits an injective map that preserves `0`, `+`, unary `-`, and binary `-` to a `SubNegZeroMonoid`. This version takes custom `nsmul` and `zsmul` as `[SMul ℕ M₁]` and `[SMul ℤ M₁]` arguments."] protected def divInvOneMonoid [DivInvOneMonoid M₂] (f : M₁ → M₂) (hf : Injective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) (inv : ∀ x, f x⁻¹ = (f x)⁻¹) (div : ∀ x y, f (x / y) = f x / f y) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) (zpow : ∀ (x) (n : ℤ), f (x ^ n) = f x ^ n) : DivInvOneMonoid M₁ := { hf.divInvMonoid f one mul inv div npow zpow, hf.invOneClass f one inv with } /-- A type endowed with `1`, `*`, `⁻¹`, and `/` is a `DivisionMonoid` if it admits an injective map that preserves `1`, `*`, `⁻¹`, and `/` to a `DivisionMonoid`. See note [reducible non-instances] -/ @[to_additive (attr := reducible) subtractionMonoid "A type endowed with `0`, `+`, unary `-`, and binary `-` is a `SubtractionMonoid` if it admits an injective map that preserves `0`, `+`, unary `-`, and binary `-` to a `SubtractionMonoid`. This version takes custom `nsmul` and `zsmul` as `[SMul ℕ M₁]` and `[SMul ℤ M₁]` arguments."] protected def divisionMonoid [DivisionMonoid M₂] (f : M₁ → M₂) (hf : Injective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) (inv : ∀ x, f x⁻¹ = (f x)⁻¹) (div : ∀ x y, f (x / y) = f x / f y) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) (zpow : ∀ (x) (n : ℤ), f (x ^ n) = f x ^ n) : DivisionMonoid M₁ := { hf.divInvMonoid f one mul inv div npow zpow, hf.involutiveInv f inv with mul_inv_rev := fun x y => hf <| by erw [inv, mul, mul_inv_rev, mul, inv, inv], inv_eq_of_mul := fun x y h => hf <| by erw [inv, inv_eq_of_mul_eq_one_right (by erw [← mul, h, one])] } /-- A type endowed with `1`, `*`, `⁻¹`, and `/` is a `DivisionCommMonoid` if it admits an injective map that preserves `1`, `*`, `⁻¹`, and `/` to a `DivisionCommMonoid`. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) subtractionCommMonoid "A type endowed with `0`, `+`, unary `-`, and binary `-` is a `SubtractionCommMonoid` if it admits an injective map that preserves `0`, `+`, unary `-`, and binary `-` to a `SubtractionCommMonoid`. This version takes custom `nsmul` and `zsmul` as `[SMul ℕ M₁]` and `[SMul ℤ M₁]` arguments."] protected def divisionCommMonoid [DivisionCommMonoid M₂] (f : M₁ → M₂) (hf : Injective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) (inv : ∀ x, f x⁻¹ = (f x)⁻¹) (div : ∀ x y, f (x / y) = f x / f y) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) (zpow : ∀ (x) (n : ℤ), f (x ^ n) = f x ^ n) : DivisionCommMonoid M₁ := { hf.divisionMonoid f one mul inv div npow zpow, hf.commSemigroup f mul with } /-- A type endowed with `1`, `*` and `⁻¹` is a group, if it admits an injective map that preserves `1`, `*` and `⁻¹` to a group. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `0` and `+` is an additive group, if it admits an injective map that preserves `0` and `+` to an additive group."] protected def group [Group M₂] (f : M₁ → M₂) (hf : Injective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) (inv : ∀ x, f x⁻¹ = (f x)⁻¹) (div : ∀ x y, f (x / y) = f x / f y) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) (zpow : ∀ (x) (n : ℤ), f (x ^ n) = f x ^ n) : Group M₁ := { hf.divInvMonoid f one mul inv div npow zpow with mul_left_inv := fun x => hf <| by erw [mul, inv, mul_left_inv, one] } /-- A type endowed with `0`, `1` and `+` is an additive group with one, if it admits an injective map that preserves `0`, `1` and `+` to an additive group with one. See note [reducible non-instances]. -/ protected abbrev addGroupWithOne {M₁} [Zero M₁] [One M₁] [Add M₁] [SMul ℕ M₁] [Neg M₁] [Sub M₁] [SMul ℤ M₁] [NatCast M₁] [IntCast M₁] [AddGroupWithOne M₂] (f : M₁ → M₂) (hf : Injective f) (zero : f 0 = 0) (one : f 1 = 1) (add : ∀ x y, f (x + y) = f x + f y) (neg : ∀ x, f (-x) = -f x) (sub : ∀ x y, f (x - y) = f x - f y) (nsmul : ∀ (n : ℕ) (x), f (n • x) = n • f x) (zsmul : ∀ (n : ℤ) (x), f (n • x) = n • f x) (natCast : ∀ n : ℕ, f n = n) (intCast : ∀ n : ℤ, f n = n) : AddGroupWithOne M₁ := { hf.addGroup f zero add neg sub (swap nsmul) (swap zsmul), hf.addMonoidWithOne f zero one add nsmul natCast with intCast := Int.cast, intCast_ofNat := fun n => hf (by rw [natCast, ← Int.cast, intCast, Int.cast_natCast]), intCast_negSucc := fun n => hf (by erw [intCast, neg, natCast, Int.cast_negSucc] ) } /-- A type endowed with `1`, `*` and `⁻¹` is a commutative group, if it admits an injective map that preserves `1`, `*` and `⁻¹` to a commutative group. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `0` and `+` is an additive commutative group, if it admits an injective map that preserves `0` and `+` to an additive commutative group."] protected def commGroup [CommGroup M₂] (f : M₁ → M₂) (hf : Injective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) (inv : ∀ x, f x⁻¹ = (f x)⁻¹) (div : ∀ x y, f (x / y) = f x / f y) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) (zpow : ∀ (x) (n : ℤ), f (x ^ n) = f x ^ n) : CommGroup M₁ := { hf.commMonoid f one mul npow, hf.group f one mul inv div npow zpow with } /-- A type endowed with `0`, `1` and `+` is an additive commutative group with one, if it admits an injective map that preserves `0`, `1` and `+` to an additive commutative group with one. See note [reducible non-instances]. -/ protected abbrev addCommGroupWithOne {M₁} [Zero M₁] [One M₁] [Add M₁] [SMul ℕ M₁] [Neg M₁] [Sub M₁] [SMul ℤ M₁] [NatCast M₁] [IntCast M₁] [AddCommGroupWithOne M₂] (f : M₁ → M₂) (hf : Injective f) (zero : f 0 = 0) (one : f 1 = 1) (add : ∀ x y, f (x + y) = f x + f y) (neg : ∀ x, f (-x) = -f x) (sub : ∀ x y, f (x - y) = f x - f y) (nsmul : ∀ (n : ℕ) (x), f (n • x) = n • f x) (zsmul : ∀ (n : ℤ) (x), f (n • x) = n • f x) (natCast : ∀ n : ℕ, f n = n) (intCast : ∀ n : ℤ, f n = n) : AddCommGroupWithOne M₁ := { hf.addGroupWithOne f zero one add neg sub nsmul zsmul natCast intCast, hf.addCommMonoid _ zero add (swap nsmul) with } end Injective /-! ### Surjective -/ namespace Surjective variable {M₁ : Type*} {M₂ : Type*} [Mul M₂] /-- A type endowed with `*` is a semigroup, if it admits a surjective map that preserves `*` from a semigroup. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `+` is an additive semigroup, if it admits a surjective map that preserves `+` from an additive semigroup."] protected def semigroup [Semigroup M₁] (f : M₁ → M₂) (hf : Surjective f) (mul : ∀ x y, f (x * y) = f x * f y) : Semigroup M₂ := { ‹Mul M₂› with mul_assoc := hf.forall₃.2 fun x y z => by simp only [← mul, mul_assoc] } /-- A type endowed with `*` is a commutative semigroup, if it admits a surjective map that preserves `*` from a commutative semigroup. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `+` is an additive commutative semigroup, if it admits a surjective map that preserves `+` from an additive commutative semigroup."] protected def commMagma [CommMagma M₁] (f : M₁ → M₂) (hf : Surjective f) (mul : ∀ x y, f (x * y) = f x * f y) : CommMagma M₂ where mul_comm := hf.forall₂.2 fun x y => by erw [← mul, ← mul, mul_comm] /-- A type endowed with `*` is a commutative semigroup, if it admits a surjective map that preserves `*` from a commutative semigroup. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `+` is an additive commutative semigroup, if it admits a surjective map that preserves `+` from an additive commutative semigroup."] protected def commSemigroup [CommSemigroup M₁] (f : M₁ → M₂) (hf : Surjective f) (mul : ∀ x y, f (x * y) = f x * f y) : CommSemigroup M₂ where toSemigroup := hf.semigroup f mul __ := hf.commMagma f mul variable [One M₂] /-- A type endowed with `1` and `*` is a `MulOneClass`, if it admits a surjective map that preserves `1` and `*` from a `MulOneClass`. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `0` and `+` is an `AddZeroClass`, if it admits a surjective map that preserves `0` and `+` to an `AddZeroClass`."] protected def mulOneClass [MulOneClass M₁] (f : M₁ → M₂) (hf : Surjective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) : MulOneClass M₂ := { ‹One M₂›, ‹Mul M₂› with one_mul := hf.forall.2 fun x => by erw [← one, ← mul, one_mul], mul_one := hf.forall.2 fun x => by erw [← one, ← mul, mul_one] } variable [Pow M₂ ℕ] /-- A type endowed with `1` and `*` is a monoid, if it admits a surjective map that preserves `1` and `*` to a monoid. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `0` and `+` is an additive monoid, if it admits a surjective map that preserves `0` and `+` to an additive monoid. This version takes a custom `nsmul` as a `[SMul ℕ M₂]` argument."] protected def monoid [Monoid M₁] (f : M₁ → M₂) (hf : Surjective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) : Monoid M₂ := { hf.semigroup f mul, hf.mulOneClass f one mul with npow := fun n x => x ^ n, npow_zero := hf.forall.2 fun x => by dsimp only; erw [← npow, pow_zero, ← one], npow_succ := fun n => hf.forall.2 fun x => by dsimp only erw [← npow, pow_succ, ← npow, ← mul] } /-- A type endowed with `0`, `1` and `+` is an additive monoid with one, if it admits a surjective map that preserves `0`, `1` and `*` from an additive monoid with one. See note [reducible non-instances]. -/ protected abbrev addMonoidWithOne {M₂} [Zero M₂] [One M₂] [Add M₂] [SMul ℕ M₂] [NatCast M₂] [AddMonoidWithOne M₁] (f : M₁ → M₂) (hf : Surjective f) (zero : f 0 = 0) (one : f 1 = 1) (add : ∀ x y, f (x + y) = f x + f y) (nsmul : ∀ (n : ℕ) (x), f (n • x) = n • f x) (natCast : ∀ n : ℕ, f n = n) : AddMonoidWithOne M₂ := { hf.addMonoid f zero add (swap nsmul) with natCast := Nat.cast, natCast_zero := by rw [← Nat.cast, ← natCast, Nat.cast_zero, zero] natCast_succ := fun n => by rw [← Nat.cast, ← natCast, Nat.cast_succ, add, one, natCast] one := 1 } /-- A type endowed with `1` and `*` is a commutative monoid, if it admits a surjective map that preserves `1` and `*` from a commutative monoid. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `0` and `+` is an additive commutative monoid, if it admits a surjective map that preserves `0` and `+` to an additive commutative monoid."] protected def commMonoid [CommMonoid M₁] (f : M₁ → M₂) (hf : Surjective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) : CommMonoid M₂ := { hf.commSemigroup f mul, hf.monoid f one mul npow with } /-- A type endowed with `0`, `1` and `+` is an additive monoid with one, if it admits a surjective map that preserves `0`, `1` and `*` from an additive monoid with one. See note [reducible non-instances]. -/ protected abbrev addCommMonoidWithOne {M₂} [Zero M₂] [One M₂] [Add M₂] [SMul ℕ M₂] [NatCast M₂] [AddCommMonoidWithOne M₁] (f : M₁ → M₂) (hf : Surjective f) (zero : f 0 = 0) (one : f 1 = 1) (add : ∀ x y, f (x + y) = f x + f y) (nsmul : ∀ (n : ℕ) (x), f (n • x) = n • f x) (natCast : ∀ n : ℕ, f n = n) : AddCommMonoidWithOne M₂ where __ := hf.addMonoidWithOne f zero one add nsmul natCast __ := hf.addCommMonoid _ zero add (swap nsmul) /-- A type has an involutive inversion if it admits a surjective map that preserves `⁻¹` to a type which has an involutive inversion. See note [reducible non-instances] -/ @[to_additive (attr := reducible) "A type has an involutive negation if it admits a surjective map that preserves `-` to a type which has an involutive negation."] protected def involutiveInv {M₂ : Type*} [Inv M₂] [InvolutiveInv M₁] (f : M₁ → M₂) (hf : Surjective f) (inv : ∀ x, f x⁻¹ = (f x)⁻¹) : InvolutiveInv M₂ where inv := Inv.inv inv_inv := hf.forall.2 fun x => by erw [← inv, ← inv, inv_inv] variable [Inv M₂] [Div M₂] [Pow M₂ ℤ] /-- A type endowed with `1`, `*`, `⁻¹`, and `/` is a `DivInvMonoid` if it admits a surjective map that preserves `1`, `*`, `⁻¹`, and `/` to a `DivInvMonoid`. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) subNegMonoid "A type endowed with `0`, `+`, unary `-`, and binary `-` is a `SubNegMonoid` if it admits a surjective map that preserves `0`, `+`, unary `-`, and binary `-` to a `SubNegMonoid`."] protected def divInvMonoid [DivInvMonoid M₁] (f : M₁ → M₂) (hf : Surjective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) (inv : ∀ x, f x⁻¹ = (f x)⁻¹) (div : ∀ x y, f (x / y) = f x / f y) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) (zpow : ∀ (x) (n : ℤ), f (x ^ n) = f x ^ n) : DivInvMonoid M₂ := { hf.monoid f one mul npow, ‹Div M₂›, ‹Inv M₂› with zpow := fun n x => x ^ n, zpow_zero' := hf.forall.2 fun x => by dsimp only; erw [← zpow, zpow_zero, ← one], zpow_succ' := fun n => hf.forall.2 fun x => by dsimp only erw [← zpow, ← zpow, zpow_natCast, zpow_natCast, pow_succ, ← mul], zpow_neg' := fun n => hf.forall.2 fun x => by dsimp only erw [← zpow, ← zpow, zpow_negSucc, zpow_natCast, inv], div_eq_mul_inv := hf.forall₂.2 fun x y => by erw [← inv, ← mul, ← div, div_eq_mul_inv] } /-- A type endowed with `1`, `*` and `⁻¹` is a group, if it admits a surjective map that preserves `1`, `*` and `⁻¹` to a group. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `0` and `+` is an additive group, if it admits a surjective map that preserves `0` and `+` to an additive group."] protected def group [Group M₁] (f : M₁ → M₂) (hf : Surjective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) (inv : ∀ x, f x⁻¹ = (f x)⁻¹) (div : ∀ x y, f (x / y) = f x / f y) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) (zpow : ∀ (x) (n : ℤ), f (x ^ n) = f x ^ n) : Group M₂ := { hf.divInvMonoid f one mul inv div npow zpow with mul_left_inv := hf.forall.2 fun x => by erw [← inv, ← mul, mul_left_inv, one] } /-- A type endowed with `0`, `1`, `+` is an additive group with one, if it admits a surjective map that preserves `0`, `1`, and `+` to an additive group with one. See note [reducible non-instances]. -/ protected abbrev addGroupWithOne {M₂} [Zero M₂] [One M₂] [Add M₂] [Neg M₂] [Sub M₂] [SMul ℕ M₂] [SMul ℤ M₂] [NatCast M₂] [IntCast M₂] [AddGroupWithOne M₁] (f : M₁ → M₂) (hf : Surjective f) (zero : f 0 = 0) (one : f 1 = 1) (add : ∀ x y, f (x + y) = f x + f y) (neg : ∀ x, f (-x) = -f x) (sub : ∀ x y, f (x - y) = f x - f y) (nsmul : ∀ (n : ℕ) (x), f (n • x) = n • f x) (zsmul : ∀ (n : ℤ) (x), f (n • x) = n • f x) (natCast : ∀ n : ℕ, f n = n) (intCast : ∀ n : ℤ, f n = n) : AddGroupWithOne M₂ := { hf.addMonoidWithOne f zero one add nsmul natCast, hf.addGroup f zero add neg sub (swap nsmul) (swap zsmul) with intCast := Int.cast, intCast_ofNat := fun n => by rw [← Int.cast, ← intCast, Int.cast_natCast, natCast], intCast_negSucc := fun n => by rw [← Int.cast, ← intCast, Int.cast_negSucc, neg, natCast] } /-- A type endowed with `1`, `*`, `⁻¹`, and `/` is a commutative group, if it admits a surjective map that preserves `1`, `*`, `⁻¹`, and `/` from a commutative group. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "A type endowed with `0` and `+` is an additive commutative group, if it admits a surjective map that preserves `0` and `+` to an additive commutative group."] protected def commGroup [CommGroup M₁] (f : M₁ → M₂) (hf : Surjective f) (one : f 1 = 1) (mul : ∀ x y, f (x * y) = f x * f y) (inv : ∀ x, f x⁻¹ = (f x)⁻¹) (div : ∀ x y, f (x / y) = f x / f y) (npow : ∀ (x) (n : ℕ), f (x ^ n) = f x ^ n) (zpow : ∀ (x) (n : ℤ), f (x ^ n) = f x ^ n) : CommGroup M₂ := { hf.commMonoid f one mul npow, hf.group f one mul inv div npow zpow with } /-- A type endowed with `0`, `1`, `+` is an additive commutative group with one, if it admits a surjective map that preserves `0`, `1`, and `+` to an additive commutative group with one. See note [reducible non-instances]. -/ protected abbrev addCommGroupWithOne {M₂} [Zero M₂] [One M₂] [Add M₂] [Neg M₂] [Sub M₂] [SMul ℕ M₂] [SMul ℤ M₂] [NatCast M₂] [IntCast M₂] [AddCommGroupWithOne M₁] (f : M₁ → M₂) (hf : Surjective f) (zero : f 0 = 0) (one : f 1 = 1) (add : ∀ x y, f (x + y) = f x + f y) (neg : ∀ x, f (-x) = -f x) (sub : ∀ x y, f (x - y) = f x - f y) (nsmul : ∀ (n : ℕ) (x), f (n • x) = n • f x) (zsmul : ∀ (n : ℤ) (x), f (n • x) = n • f x) (natCast : ∀ n : ℕ, f n = n) (intCast : ∀ n : ℤ, f n = n) : AddCommGroupWithOne M₂ := { hf.addGroupWithOne f zero one add neg sub nsmul zsmul natCast intCast, hf.addCommMonoid _ zero add (swap nsmul) with } end Surjective end Function
Algebra\Group\Int.lean
/- Copyright (c) 2016 Jeremy Avigad. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Jeremy Avigad -/ import Mathlib.Algebra.Group.Nat import Mathlib.Data.Int.Sqrt /-! # The integers form a group This file contains the additive group and multiplicative monoid instances on the integers. See note [foundational algebra order theory]. -/ assert_not_exists Ring assert_not_exists DenselyOrdered assert_not_exists Set.range open Nat namespace Int /-! ### Instances -/ instance instCommMonoid : CommMonoid ℤ where mul_comm := Int.mul_comm mul_one := Int.mul_one one_mul := Int.one_mul npow n x := x ^ n npow_zero _ := rfl npow_succ _ _ := rfl mul_assoc := Int.mul_assoc instance instAddCommGroup : AddCommGroup ℤ where add_comm := Int.add_comm add_assoc := Int.add_assoc add_zero := Int.add_zero zero_add := Int.zero_add add_left_neg := Int.add_left_neg nsmul := (·*·) nsmul_zero := Int.zero_mul nsmul_succ n x := show (n + 1 : ℤ) * x = n * x + x by rw [Int.add_mul, Int.one_mul] zsmul := (·*·) zsmul_zero' := Int.zero_mul zsmul_succ' m n := by simp only [ofNat_eq_coe, ofNat_succ, Int.add_mul, Int.add_comm, Int.one_mul] zsmul_neg' m n := by simp only [negSucc_coe, ofNat_succ, Int.neg_mul] sub_eq_add_neg _ _ := Int.sub_eq_add_neg /-! ### Extra instances to short-circuit type class resolution These also prevent non-computable instances like `Int.normedCommRing` being used to construct these instances non-computably. -/ instance instAddCommMonoid : AddCommMonoid ℤ := by infer_instance instance instAddMonoid : AddMonoid ℤ := by infer_instance instance instMonoid : Monoid ℤ := by infer_instance instance instCommSemigroup : CommSemigroup ℤ := by infer_instance instance instSemigroup : Semigroup ℤ := by infer_instance instance instAddGroup : AddGroup ℤ := by infer_instance instance instAddCommSemigroup : AddCommSemigroup ℤ := by infer_instance instance instAddSemigroup : AddSemigroup ℤ := by infer_instance /-! ### Miscellaneous lemmas -/ section Multiplicative open Multiplicative lemma toAdd_pow (a : Multiplicative ℤ) (b : ℕ) : toAdd (a ^ b) = toAdd a * b := mul_comm _ _ lemma toAdd_zpow (a : Multiplicative ℤ) (b : ℤ) : toAdd (a ^ b) = toAdd a * b := mul_comm _ _ @[simp] lemma ofAdd_mul (a b : ℤ) : ofAdd (a * b) = ofAdd a ^ b := (toAdd_zpow ..).symm end Multiplicative /-! #### Units -/ variable {u v : ℤ} lemma units_natAbs (u : ℤˣ) : natAbs u = 1 := Units.ext_iff.1 <| Nat.units_eq_one ⟨natAbs u, natAbs ↑u⁻¹, by rw [← natAbs_mul, Units.mul_inv]; rfl, by rw [← natAbs_mul, Units.inv_mul]; rfl⟩ @[simp] lemma natAbs_of_isUnit (hu : IsUnit u) : natAbs u = 1 := units_natAbs hu.unit lemma isUnit_eq_one_or (hu : IsUnit u) : u = 1 ∨ u = -1 := by simpa only [natAbs_of_isUnit hu] using natAbs_eq u lemma isUnit_ne_iff_eq_neg (hu : IsUnit u) (hv : IsUnit v) : u ≠ v ↔ u = -v := by obtain rfl | rfl := isUnit_eq_one_or hu <;> obtain rfl | rfl := isUnit_eq_one_or hv <;> decide lemma isUnit_eq_or_eq_neg (hu : IsUnit u) (hv : IsUnit v) : u = v ∨ u = -v := or_iff_not_imp_left.2 (isUnit_ne_iff_eq_neg hu hv).1 lemma isUnit_iff : IsUnit u ↔ u = 1 ∨ u = -1 := by refine ⟨fun h ↦ isUnit_eq_one_or h, fun h ↦ ?_⟩ rcases h with (rfl | rfl) · exact isUnit_one · exact ⟨⟨-1, -1, by decide, by decide⟩, rfl⟩ lemma eq_one_or_neg_one_of_mul_eq_one (h : u * v = 1) : u = 1 ∨ u = -1 := isUnit_iff.1 (isUnit_of_mul_eq_one u v h) lemma eq_one_or_neg_one_of_mul_eq_one' (h : u * v = 1) : u = 1 ∧ v = 1 ∨ u = -1 ∧ v = -1 := by have h' : v * u = 1 := mul_comm u v ▸ h obtain rfl | rfl := eq_one_or_neg_one_of_mul_eq_one h <;> obtain rfl | rfl := eq_one_or_neg_one_of_mul_eq_one h' <;> tauto lemma eq_of_mul_eq_one (h : u * v = 1) : u = v := (eq_one_or_neg_one_of_mul_eq_one' h).elim (and_imp.2 (·.trans ·.symm)) (and_imp.2 (·.trans ·.symm)) lemma mul_eq_one_iff_eq_one_or_neg_one : u * v = 1 ↔ u = 1 ∧ v = 1 ∨ u = -1 ∧ v = -1 := by refine ⟨eq_one_or_neg_one_of_mul_eq_one', fun h ↦ Or.elim h (fun H ↦ ?_) fun H ↦ ?_⟩ <;> obtain ⟨rfl, rfl⟩ := H <;> rfl lemma eq_one_or_neg_one_of_mul_eq_neg_one' (h : u * v = -1) : u = 1 ∧ v = -1 ∨ u = -1 ∧ v = 1 := by obtain rfl | rfl := isUnit_eq_one_or (IsUnit.mul_iff.mp (Int.isUnit_iff.mpr (Or.inr h))).1 · exact Or.inl ⟨rfl, one_mul v ▸ h⟩ · simpa [Int.neg_mul] using h lemma mul_eq_neg_one_iff_eq_one_or_neg_one : u * v = -1 ↔ u = 1 ∧ v = -1 ∨ u = -1 ∧ v = 1 := by refine ⟨eq_one_or_neg_one_of_mul_eq_neg_one', fun h ↦ Or.elim h (fun H ↦ ?_) fun H ↦ ?_⟩ <;> obtain ⟨rfl, rfl⟩ := H <;> rfl lemma isUnit_iff_natAbs_eq : IsUnit u ↔ u.natAbs = 1 := by simp [natAbs_eq_iff, isUnit_iff] alias ⟨IsUnit.natAbs_eq, _⟩ := isUnit_iff_natAbs_eq -- Porting note: `rw` didn't work on `natAbs_ofNat`, so had to change to `simp`, -- presumably because `(n : ℤ)` is `Nat.cast` and not just `ofNat` @[norm_cast] lemma ofNat_isUnit {n : ℕ} : IsUnit (n : ℤ) ↔ IsUnit n := by simp [isUnit_iff_natAbs_eq] lemma isUnit_mul_self (hu : IsUnit u) : u * u = 1 := (isUnit_eq_one_or hu).elim (fun h ↦ h.symm ▸ rfl) fun h ↦ h.symm ▸ rfl -- Porting note: this was proven in mathlib3 with `tidy` which hasn't been ported yet lemma isUnit_add_isUnit_eq_isUnit_add_isUnit {a b c d : ℤ} (ha : IsUnit a) (hb : IsUnit b) (hc : IsUnit c) (hd : IsUnit d) : a + b = c + d ↔ a = c ∧ b = d ∨ a = d ∧ b = c := by rw [isUnit_iff] at ha hb hc hd cases ha <;> cases hb <;> cases hc <;> cases hd <;> subst a <;> subst b <;> subst c <;> subst d <;> simp (config := {decide := true}) lemma eq_one_or_neg_one_of_mul_eq_neg_one (h : u * v = -1) : u = 1 ∨ u = -1 := Or.elim (eq_one_or_neg_one_of_mul_eq_neg_one' h) (fun H => Or.inl H.1) fun H => Or.inr H.1 /-! #### Parity -/ variable {m n : ℤ} @[simp] lemma emod_two_ne_one : ¬n % 2 = 1 ↔ n % 2 = 0 := by cases' emod_two_eq_zero_or_one n with h h <;> simp [h] @[simp] lemma one_emod_two : (1 : Int) % 2 = 1 := rfl -- `EuclideanDomain.mod_eq_zero` uses (2 ∣ n) as normal form @[local simp] lemma emod_two_ne_zero : ¬n % 2 = 0 ↔ n % 2 = 1 := by cases' emod_two_eq_zero_or_one n with h h <;> simp [h] lemma even_iff : Even n ↔ n % 2 = 0 where mp := fun ⟨m, hm⟩ ↦ by simp [← Int.two_mul, hm] mpr h := ⟨n / 2, (emod_add_ediv n 2).symm.trans (by simp [← Int.two_mul, h])⟩ lemma not_even_iff : ¬Even n ↔ n % 2 = 1 := by rw [even_iff, emod_two_ne_zero] @[simp] lemma two_dvd_ne_zero : ¬2 ∣ n ↔ n % 2 = 1 := (even_iff_exists_two_nsmul _).symm.not.trans not_even_iff instance : DecidablePred (Even : ℤ → Prop) := fun _ ↦ decidable_of_iff _ even_iff.symm /-- `IsSquare` can be decided on `ℤ` by checking against the square root. -/ instance : DecidablePred (IsSquare : ℤ → Prop) := fun m ↦ decidable_of_iff' (sqrt m * sqrt m = m) <| by simp_rw [← exists_mul_self m, IsSquare, eq_comm] @[simp] lemma not_even_one : ¬Even (1 : ℤ) := by simp [even_iff] @[parity_simps] lemma even_add : Even (m + n) ↔ (Even m ↔ Even n) := by cases' emod_two_eq_zero_or_one m with h₁ h₁ <;> cases' emod_two_eq_zero_or_one n with h₂ h₂ <;> simp [even_iff, h₁, h₂, Int.add_emod, one_add_one_eq_two, emod_self] lemma two_not_dvd_two_mul_add_one (n : ℤ) : ¬2 ∣ 2 * n + 1 := by simp [add_emod] @[parity_simps] lemma even_sub : Even (m - n) ↔ (Even m ↔ Even n) := by simp [sub_eq_add_neg, parity_simps] @[parity_simps] lemma even_add_one : Even (n + 1) ↔ ¬Even n := by simp [even_add] @[parity_simps] lemma even_sub_one : Even (n - 1) ↔ ¬Even n := by simp [even_sub] @[parity_simps] lemma even_mul : Even (m * n) ↔ Even m ∨ Even n := by cases' emod_two_eq_zero_or_one m with h₁ h₁ <;> cases' emod_two_eq_zero_or_one n with h₂ h₂ <;> simp [even_iff, h₁, h₂, Int.mul_emod] @[parity_simps] lemma even_pow {n : ℕ} : Even (m ^ n) ↔ Even m ∧ n ≠ 0 := by induction' n with n ih <;> simp [*, even_mul, pow_succ]; tauto lemma even_pow' {n : ℕ} (h : n ≠ 0) : Even (m ^ n) ↔ Even m := even_pow.trans <| and_iff_left h @[simp, norm_cast] lemma even_coe_nat (n : ℕ) : Even (n : ℤ) ↔ Even n := by rw_mod_cast [even_iff, Nat.even_iff] lemma two_mul_ediv_two_of_even : Even n → 2 * (n / 2) = n := fun h ↦ Int.mul_ediv_cancel' ((even_iff_exists_two_nsmul _).mp h) lemma ediv_two_mul_two_of_even : Even n → n / 2 * 2 = n := fun h ↦ Int.ediv_mul_cancel ((even_iff_exists_two_nsmul _).mp h) -- Here are examples of how `parity_simps` can be used with `Int`. example (m n : ℤ) (h : Even m) : ¬Even (n + 3) ↔ Even (m ^ 2 + m + n) := by simp (config := {decide := true}) [*, (by decide : ¬2 = 0), parity_simps] example : ¬Even (25394535 : ℤ) := by decide end Int -- TODO: Do we really need this lemma? This is just `smul_eq_mul` lemma zsmul_int_int (a b : ℤ) : a • b = a * b := rfl lemma zsmul_int_one (n : ℤ) : n • (1 : ℤ) = n := mul_one _
Algebra\Group\MinimalAxioms.lean
/- Copyright (c) 2023 Chris Hughes. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Chris Hughes -/ import Mathlib.Algebra.Group.Defs /-! # Minimal Axioms for a Group This file defines constructors to define a group structure on a Type, while proving only three equalities. ## Main Definitions * `Group.ofLeftAxioms`: Define a group structure on a Type by proving `∀ a, 1 * a = a` and `∀ a, a⁻¹ * a = 1` and associativity. * `Group.ofRightAxioms`: Define a group structure on a Type by proving `∀ a, a * 1 = a` and `∀ a, a * a⁻¹ = 1` and associativity. -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered universe u /-- Define a `Group` structure on a Type by proving `∀ a, 1 * a = a` and `∀ a, a⁻¹ * a = 1`. Note that this uses the default definitions for `npow`, `zpow` and `div`. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "Define an `AddGroup` structure on a Type by proving `∀ a, 0 + a = a` and `∀ a, -a + a = 0`. Note that this uses the default definitions for `nsmul`, `zsmul` and `sub`. See note [reducible non-instances]."] def Group.ofLeftAxioms {G : Type u} [Mul G] [Inv G] [One G] (assoc : ∀ a b c : G, (a * b) * c = a * (b * c)) (one_mul : ∀ a : G, 1 * a = a) (mul_left_inv : ∀ a : G, a⁻¹ * a = 1) : Group G := { mul_assoc := assoc, one_mul := one_mul, mul_left_inv := mul_left_inv, mul_one := fun a => by have mul_right_inv : ∀ a : G, a * a⁻¹ = 1 := fun a => calc a * a⁻¹ = 1 * (a * a⁻¹) := (one_mul _).symm _ = ((a * a⁻¹)⁻¹ * (a * a⁻¹)) * (a * a⁻¹) := by rw [mul_left_inv] _ = (a * a⁻¹)⁻¹ * (a * ((a⁻¹ * a) * a⁻¹)) := by simp only [assoc] _ = 1 := by rw [mul_left_inv, one_mul, mul_left_inv] rw [← mul_left_inv a, ← assoc, mul_right_inv a, one_mul] } /-- Define a `Group` structure on a Type by proving `∀ a, a * 1 = a` and `∀ a, a * a⁻¹ = 1`. Note that this uses the default definitions for `npow`, `zpow` and `div`. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "Define an `AddGroup` structure on a Type by proving `∀ a, a + 0 = a` and `∀ a, a + -a = 0`. Note that this uses the default definitions for `nsmul`, `zsmul` and `sub`. See note [reducible non-instances]."] def Group.ofRightAxioms {G : Type u} [Mul G] [Inv G] [One G] (assoc : ∀ a b c : G, (a * b) * c = a * (b * c)) (mul_one : ∀ a : G, a * 1 = a) (mul_right_inv : ∀ a : G, a * a⁻¹ = 1) : Group G := have mul_left_inv : ∀ a : G, a⁻¹ * a = 1 := fun a => calc a⁻¹ * a = (a⁻¹ * a) * 1 := (mul_one _).symm _ = (a⁻¹ * a) * ((a⁻¹ * a) * (a⁻¹ * a)⁻¹) := by rw [mul_right_inv] _ = ((a⁻¹ * (a * a⁻¹)) * a) * (a⁻¹ * a)⁻¹ := by simp only [assoc] _ = 1 := by rw [mul_right_inv, mul_one, mul_right_inv] { mul_assoc := assoc, mul_one := mul_one, mul_left_inv := mul_left_inv, one_mul := fun a => by rw [← mul_right_inv a, assoc, mul_left_inv, mul_one] }
Algebra\Group\Nat.lean
/- Copyright (c) 2014 Floris van Doorn (c) 2016 Microsoft Corporation. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Floris van Doorn, Leonardo de Moura, Jeremy Avigad, Mario Carneiro -/ import Mathlib.Algebra.Group.Even import Mathlib.Algebra.Group.Units /-! # The natural numbers form a monoid This file contains the additive and multiplicative monoid instances on the natural numbers. See note [foundational algebra order theory]. -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered open Multiplicative namespace Nat /-! ### Instances -/ instance instAddCancelCommMonoid : AddCancelCommMonoid ℕ where add := Nat.add add_assoc := Nat.add_assoc zero := Nat.zero zero_add := Nat.zero_add add_zero := Nat.add_zero add_comm := Nat.add_comm nsmul m n := m * n nsmul_zero := Nat.zero_mul nsmul_succ := succ_mul add_left_cancel _ _ _ := Nat.add_left_cancel instance instCommMonoid : CommMonoid ℕ where mul := Nat.mul mul_assoc := Nat.mul_assoc one := Nat.succ Nat.zero one_mul := Nat.one_mul mul_one := Nat.mul_one mul_comm := Nat.mul_comm npow m n := n ^ m npow_zero := Nat.pow_zero npow_succ _ _ := rfl /-! ### Extra instances to short-circuit type class resolution These also prevent non-computable instances being used to construct these instances non-computably. -/ instance instAddCommMonoid : AddCommMonoid ℕ := by infer_instance instance instAddMonoid : AddMonoid ℕ := by infer_instance instance instMonoid : Monoid ℕ := by infer_instance instance instCommSemigroup : CommSemigroup ℕ := by infer_instance instance instSemigroup : Semigroup ℕ := by infer_instance instance instAddCommSemigroup : AddCommSemigroup ℕ := by infer_instance instance instAddSemigroup : AddSemigroup ℕ := by infer_instance /-! ### Miscellaneous lemmas -/ -- We want to use this lemma earlier than the lemmas simp can prove it with @[simp, nolint simpNF] protected lemma nsmul_eq_mul (m n : ℕ) : m • n = m * n := rfl section Multiplicative lemma toAdd_pow (a : Multiplicative ℕ) (b : ℕ) : toAdd (a ^ b) = toAdd a * b := mul_comm _ _ @[simp] lemma ofAdd_mul (a b : ℕ) : ofAdd (a * b) = ofAdd a ^ b := (toAdd_pow _ _).symm end Multiplicative /-! #### Parity -/ variable {m n : ℕ} lemma even_iff : Even n ↔ n % 2 = 0 where mp := fun ⟨m, hm⟩ ↦ by simp [← Nat.two_mul, hm] mpr h := ⟨n / 2, (mod_add_div n 2).symm.trans (by simp [← Nat.two_mul, h])⟩ instance : DecidablePred (Even : ℕ → Prop) := fun _ ↦ decidable_of_iff _ even_iff.symm /-- `IsSquare` can be decided on `ℕ` by checking against the square root. -/ instance : DecidablePred (IsSquare : ℕ → Prop) := fun m ↦ decidable_of_iff' (Nat.sqrt m * Nat.sqrt m = m) <| by simp_rw [← Nat.exists_mul_self m, IsSquare, eq_comm] lemma not_even_iff : ¬ Even n ↔ n % 2 = 1 := by rw [even_iff, mod_two_ne_zero] @[simp] lemma two_dvd_ne_zero : ¬2 ∣ n ↔ n % 2 = 1 := (even_iff_exists_two_nsmul _).symm.not.trans not_even_iff @[simp] lemma not_even_one : ¬Even 1 := by simp [even_iff] @[parity_simps] lemma even_add : Even (m + n) ↔ (Even m ↔ Even n) := by cases' mod_two_eq_zero_or_one m with h₁ h₁ <;> cases' mod_two_eq_zero_or_one n with h₂ h₂ <;> simp [even_iff, h₁, h₂, Nat.add_mod] @[parity_simps] lemma even_add_one : Even (n + 1) ↔ ¬Even n := by simp [even_add] lemma succ_mod_two_eq_zero_iff {m : ℕ} : (m + 1) % 2 = 0 ↔ m % 2 = 1 := by simp [← Nat.even_iff, ← Nat.not_even_iff, parity_simps] lemma succ_mod_two_eq_one_iff {m : ℕ} : (m + 1) % 2 = 1 ↔ m % 2 = 0 := by simp [← Nat.even_iff, ← Nat.not_even_iff, parity_simps] lemma two_not_dvd_two_mul_add_one (n : ℕ) : ¬2 ∣ 2 * n + 1 := by simp [add_mod] lemma two_not_dvd_two_mul_sub_one : ∀ {n}, 0 < n → ¬2 ∣ 2 * n - 1 | n + 1, _ => two_not_dvd_two_mul_add_one n @[parity_simps] lemma even_sub (h : n ≤ m) : Even (m - n) ↔ (Even m ↔ Even n) := by conv_rhs => rw [← Nat.sub_add_cancel h, even_add] by_cases h : Even n <;> simp [h] @[parity_simps] lemma even_mul : Even (m * n) ↔ Even m ∨ Even n := by cases' mod_two_eq_zero_or_one m with h₁ h₁ <;> cases' mod_two_eq_zero_or_one n with h₂ h₂ <;> simp [even_iff, h₁, h₂, Nat.mul_mod] /-- If `m` and `n` are natural numbers, then the natural number `m^n` is even if and only if `m` is even and `n` is positive. -/ @[parity_simps] lemma even_pow : Even (m ^ n) ↔ Even m ∧ n ≠ 0 := by induction' n with n ih <;> simp (config := { contextual := true }) [*, pow_succ', even_mul] lemma even_pow' (h : n ≠ 0) : Even (m ^ n) ↔ Even m := even_pow.trans <| and_iff_left h lemma even_mul_succ_self (n : ℕ) : Even (n * (n + 1)) := by rw [even_mul, even_add_one]; exact em _ lemma even_mul_pred_self : ∀ n : ℕ, Even (n * (n - 1)) | 0 => even_zero | (n + 1) => mul_comm (n + 1 - 1) (n + 1) ▸ even_mul_succ_self n @[deprecated (since := "2024-01-20")] alias even_mul_self_pred := even_mul_pred_self lemma two_mul_div_two_of_even : Even n → 2 * (n / 2) = n := fun h ↦ Nat.mul_div_cancel_left' ((even_iff_exists_two_nsmul _).1 h) lemma div_two_mul_two_of_even : Even n → n / 2 * 2 = n := fun h ↦ Nat.div_mul_cancel ((even_iff_exists_two_nsmul _).1 h) -- Here are examples of how `parity_simps` can be used with `Nat`. example (m n : ℕ) (h : Even m) : ¬Even (n + 3) ↔ Even (m ^ 2 + m + n) := by simp [*, parity_simps] -- Porting note: the `simp` lemmas about `bit*` no longer apply. example : ¬Even 25394535 := by decide /-! #### Units -/ lemma units_eq_one (u : ℕˣ) : u = 1 := Units.ext <| Nat.eq_one_of_dvd_one ⟨u.inv, u.val_inv.symm⟩ lemma addUnits_eq_zero (u : AddUnits ℕ) : u = 0 := AddUnits.ext <| (Nat.eq_zero_of_add_eq_zero u.val_neg).1 @[simp] protected lemma isUnit_iff {n : ℕ} : IsUnit n ↔ n = 1 where mp := by rintro ⟨u, rfl⟩; obtain rfl := Nat.units_eq_one u; rfl mpr h := h.symm ▸ ⟨1, rfl⟩ instance unique_units : Unique ℕˣ where default := 1 uniq := Nat.units_eq_one instance unique_addUnits : Unique (AddUnits ℕ) where default := 0 uniq := Nat.addUnits_eq_zero end Nat
Algebra\Group\NatPowAssoc.lean
/- Copyright (c) 2023 Scott Carnahan. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Carnahan -/ import Mathlib.Algebra.Group.Action.Prod import Mathlib.Algebra.Ring.Int import Mathlib.Data.Nat.Cast.Basic /-! # Typeclasses for power-associative structures In this file we define power-associativity for algebraic structures with a multiplication operation. The class is a Prop-valued mixin named `NatPowAssoc`. ## Results - `npow_add` a defining property: `x ^ (k + n) = x ^ k * x ^ n` - `npow_one` a defining property: `x ^ 1 = x` - `npow_assoc` strictly positive powers of an element have associative multiplication. - `npow_comm` `x ^ m * x ^ n = x ^ n * x ^ m` for strictly positive `m` and `n`. - `npow_mul` `x ^ (m * n) = (x ^ m) ^ n` for strictly positive `m` and `n`. - `npow_eq_pow` monoid exponentiation coincides with semigroup exponentiation. ## Instances We also produce the following instances: - `NatPowAssoc` for Monoids, Pi types and products. ## TODO * to_additive? -/ assert_not_exists DenselyOrdered variable {M : Type*} /-- A mixin for power-associative multiplication. -/ class NatPowAssoc (M : Type*) [MulOneClass M] [Pow M ℕ] : Prop where /-- Multiplication is power-associative. -/ protected npow_add : ∀ (k n : ℕ) (x : M), x ^ (k + n) = x ^ k * x ^ n /-- Exponent zero is one. -/ protected npow_zero : ∀ (x : M), x ^ 0 = 1 /-- Exponent one is identity. -/ protected npow_one : ∀ (x : M), x ^ 1 = x section MulOneClass variable [MulOneClass M] [Pow M ℕ] [NatPowAssoc M] theorem npow_add (k n : ℕ) (x : M) : x ^ (k + n) = x ^ k * x ^ n := NatPowAssoc.npow_add k n x @[simp] theorem npow_zero (x : M) : x ^ 0 = 1 := NatPowAssoc.npow_zero x @[simp] theorem npow_one (x : M) : x ^ 1 = x := NatPowAssoc.npow_one x theorem npow_mul_assoc (k m n : ℕ) (x : M) : (x ^ k * x ^ m) * x ^ n = x ^ k * (x ^ m * x ^ n) := by simp only [← npow_add, add_assoc] theorem npow_mul_comm (m n : ℕ) (x : M) : x ^ m * x ^ n = x ^ n * x ^ m := by simp only [← npow_add, add_comm] theorem npow_mul (x : M) (m n : ℕ) : x ^ (m * n) = (x ^ m) ^ n := by induction n with | zero => rw [npow_zero, Nat.mul_zero, npow_zero] | succ n ih => rw [mul_add, npow_add, ih, mul_one, npow_add, npow_one] theorem npow_mul' (x : M) (m n : ℕ) : x ^ (m * n) = (x ^ n) ^ m := by rw [mul_comm] exact npow_mul x n m end MulOneClass section Neg theorem neg_npow_assoc {R : Type*} [NonAssocRing R] [Pow R ℕ] [NatPowAssoc R] (a b : R) (k : ℕ) : (-1)^k * a * b = (-1)^k * (a * b) := by induction k with | zero => simp only [npow_zero, one_mul] | succ k ih => rw [npow_add, npow_one, ← neg_mul_comm, mul_one] simp only [neg_mul, ih] end Neg instance Pi.instNatPowAssoc {ι : Type*} {α : ι → Type*} [∀ i, MulOneClass <| α i] [∀ i, Pow (α i) ℕ] [∀ i, NatPowAssoc <| α i] : NatPowAssoc (∀ i, α i) where npow_add _ _ _ := by ext; simp [npow_add] npow_zero _ := by ext; simp npow_one _ := by ext; simp instance Prod.instNatPowAssoc {N : Type*} [MulOneClass M] [Pow M ℕ] [NatPowAssoc M] [MulOneClass N] [Pow N ℕ] [NatPowAssoc N] : NatPowAssoc (M × N) where npow_add _ _ _ := by ext <;> simp [npow_add] npow_zero _ := by ext <;> simp npow_one _ := by ext <;> simp section Monoid variable [Monoid M] instance Monoid.PowAssoc : NatPowAssoc M where npow_add _ _ _ := pow_add _ _ _ npow_zero _ := pow_zero _ npow_one _ := pow_one _ @[simp, norm_cast] theorem Nat.cast_npow (R : Type*) [NonAssocSemiring R] [Pow R ℕ] [NatPowAssoc R] (n m : ℕ) : (↑(n ^ m) : R) = (↑n : R) ^ m := by induction' m with m ih · simp only [pow_zero, Nat.cast_one, npow_zero] · rw [npow_add, npow_add, Nat.cast_mul, ih, npow_one, npow_one] @[simp, norm_cast] theorem Int.cast_npow (R : Type*) [NonAssocRing R] [Pow R ℕ] [NatPowAssoc R] (n : ℤ) : ∀(m : ℕ), @Int.cast R NonAssocRing.toIntCast (n ^ m) = (n : R) ^ m | 0 => by rw [pow_zero, npow_zero, Int.cast_one] | m + 1 => by rw [npow_add, npow_one, Int.cast_mul, Int.cast_npow R n m, npow_add, npow_one] end Monoid
Algebra\Group\Opposite.lean
/- Copyright (c) 2018 Kenny Lau. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Kenny Lau -/ import Mathlib.Algebra.Group.Commute.Defs import Mathlib.Algebra.Group.Equiv.Basic import Mathlib.Algebra.Group.InjSurj import Mathlib.Algebra.Group.Units import Mathlib.Algebra.Opposites import Mathlib.Data.Int.Cast.Defs import Mathlib.Tactic.Spread /-! # Group structures on the multiplicative and additive opposites -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered variable {α : Type*} namespace MulOpposite /-! ### Additive structures on `αᵐᵒᵖ` -/ @[to_additive] instance instNatCast [NatCast α] : NatCast αᵐᵒᵖ where natCast n := op n @[to_additive] instance instIntCast [IntCast α] : IntCast αᵐᵒᵖ where intCast n := op n instance instAddSemigroup [AddSemigroup α] : AddSemigroup αᵐᵒᵖ := unop_injective.addSemigroup _ fun _ _ => rfl instance instAddLeftCancelSemigroup [AddLeftCancelSemigroup α] : AddLeftCancelSemigroup αᵐᵒᵖ := unop_injective.addLeftCancelSemigroup _ fun _ _ => rfl instance instAddRightCancelSemigroup [AddRightCancelSemigroup α] : AddRightCancelSemigroup αᵐᵒᵖ := unop_injective.addRightCancelSemigroup _ fun _ _ => rfl instance instAddCommSemigroup [AddCommSemigroup α] : AddCommSemigroup αᵐᵒᵖ := unop_injective.addCommSemigroup _ fun _ _ => rfl instance instAddZeroClass [AddZeroClass α] : AddZeroClass αᵐᵒᵖ := unop_injective.addZeroClass _ (by exact rfl) fun _ _ => rfl instance instAddMonoid [AddMonoid α] : AddMonoid αᵐᵒᵖ := unop_injective.addMonoid _ (by exact rfl) (fun _ _ => rfl) fun _ _ => rfl instance instAddCommMonoid [AddCommMonoid α] : AddCommMonoid αᵐᵒᵖ := unop_injective.addCommMonoid _ rfl (fun _ _ => rfl) fun _ _ => rfl instance instAddMonoidWithOne [AddMonoidWithOne α] : AddMonoidWithOne αᵐᵒᵖ where toNatCast := instNatCast toAddMonoid := instAddMonoid toOne := instOne natCast_zero := show op ((0 : ℕ) : α) = 0 by rw [Nat.cast_zero, op_zero] natCast_succ := show ∀ n, op ((n + 1 : ℕ) : α) = op ↑(n : ℕ) + 1 by simp instance instAddCommMonoidWithOne [AddCommMonoidWithOne α] : AddCommMonoidWithOne αᵐᵒᵖ where toAddMonoidWithOne := instAddMonoidWithOne __ := instAddCommMonoid instance instSubNegMonoid [SubNegMonoid α] : SubNegMonoid αᵐᵒᵖ := unop_injective.subNegMonoid _ (by exact rfl) (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) fun _ _ => rfl instance instAddGroup [AddGroup α] : AddGroup αᵐᵒᵖ := unop_injective.addGroup _ (by exact rfl) (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) fun _ _ => rfl instance instAddCommGroup [AddCommGroup α] : AddCommGroup αᵐᵒᵖ := unop_injective.addCommGroup _ rfl (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) fun _ _ => rfl instance instAddGroupWithOne [AddGroupWithOne α] : AddGroupWithOne αᵐᵒᵖ where toAddMonoidWithOne := instAddMonoidWithOne toIntCast := instIntCast __ := instAddGroup intCast_ofNat n := show op ((n : ℤ) : α) = op (n : α) by rw [Int.cast_natCast] intCast_negSucc n := show op _ = op (-unop (op ((n + 1 : ℕ) : α))) by simp instance instAddCommGroupWithOne [AddCommGroupWithOne α] : AddCommGroupWithOne αᵐᵒᵖ where toAddCommGroup := instAddCommGroup __ := instAddGroupWithOne /-! ### Multiplicative structures on `αᵐᵒᵖ` We also generate additive structures on `αᵃᵒᵖ` using `to_additive` -/ @[to_additive] instance instIsRightCancelMul [Mul α] [IsLeftCancelMul α] : IsRightCancelMul αᵐᵒᵖ where mul_right_cancel _ _ _ h := unop_injective <| mul_left_cancel <| op_injective h @[to_additive] instance instIsLeftCancelMul [Mul α] [IsRightCancelMul α] : IsLeftCancelMul αᵐᵒᵖ where mul_left_cancel _ _ _ h := unop_injective <| mul_right_cancel <| op_injective h @[to_additive] instance instSemigroup [Semigroup α] : Semigroup αᵐᵒᵖ where mul_assoc x y z := unop_injective <| Eq.symm <| mul_assoc (unop z) (unop y) (unop x) @[to_additive] instance instLeftCancelSemigroup [RightCancelSemigroup α] : LeftCancelSemigroup αᵐᵒᵖ where mul_left_cancel _ _ _ := mul_left_cancel @[to_additive] instance instRightCancelSemigroup [LeftCancelSemigroup α] : RightCancelSemigroup αᵐᵒᵖ where mul_right_cancel _ _ _ := mul_right_cancel @[to_additive] instance instCommSemigroup [CommSemigroup α] : CommSemigroup αᵐᵒᵖ where mul_comm x y := unop_injective <| mul_comm (unop y) (unop x) @[to_additive] instance instMulOneClass [MulOneClass α] : MulOneClass αᵐᵒᵖ where toMul := instMul toOne := instOne one_mul _ := unop_injective <| mul_one _ mul_one _ := unop_injective <| one_mul _ @[to_additive] instance instMonoid [Monoid α] : Monoid αᵐᵒᵖ where toSemigroup := instSemigroup __ := instMulOneClass npow n a := op <| a.unop ^ n npow_zero _ := unop_injective <| pow_zero _ npow_succ _ _ := unop_injective <| pow_succ' _ _ @[to_additive] instance instLeftCancelMonoid [RightCancelMonoid α] : LeftCancelMonoid αᵐᵒᵖ where toLeftCancelSemigroup := instLeftCancelSemigroup __ := instMonoid @[to_additive] instance instRightCancelMonoid [LeftCancelMonoid α] : RightCancelMonoid αᵐᵒᵖ where toRightCancelSemigroup := instRightCancelSemigroup __ := instMonoid @[to_additive] instance instCancelMonoid [CancelMonoid α] : CancelMonoid αᵐᵒᵖ where toLeftCancelMonoid := instLeftCancelMonoid __ := instRightCancelMonoid @[to_additive] instance instCommMonoid [CommMonoid α] : CommMonoid αᵐᵒᵖ where toMonoid := instMonoid __ := instCommSemigroup @[to_additive] instance instCancelCommMonoid [CancelCommMonoid α] : CancelCommMonoid αᵐᵒᵖ where toLeftCancelMonoid := instLeftCancelMonoid __ := instCommMonoid @[to_additive AddOpposite.instSubNegMonoid] instance instDivInvMonoid [DivInvMonoid α] : DivInvMonoid αᵐᵒᵖ where toMonoid := instMonoid toInv := instInv zpow n a := op <| a.unop ^ n zpow_zero' _ := unop_injective <| zpow_zero _ zpow_succ' _ _ := unop_injective <| by simp only [Int.ofNat_eq_coe] rw [unop_op, zpow_natCast, pow_succ', unop_mul, unop_op, zpow_natCast] zpow_neg' _ _ := unop_injective <| DivInvMonoid.zpow_neg' _ _ @[to_additive AddOpposite.instSubtractionMonoid] instance instDivisionMonoid [DivisionMonoid α] : DivisionMonoid αᵐᵒᵖ where toDivInvMonoid := instDivInvMonoid __ := instInvolutiveInv mul_inv_rev _ _ := unop_injective <| mul_inv_rev _ _ inv_eq_of_mul _ _ h := unop_injective <| inv_eq_of_mul_eq_one_left <| congr_arg unop h @[to_additive AddOpposite.instSubtractionCommMonoid] instance instDivisionCommMonoid [DivisionCommMonoid α] : DivisionCommMonoid αᵐᵒᵖ where toDivisionMonoid := instDivisionMonoid __ := instCommSemigroup @[to_additive] instance instGroup [Group α] : Group αᵐᵒᵖ where toDivInvMonoid := instDivInvMonoid mul_left_inv _ := unop_injective <| mul_inv_self _ @[to_additive] instance instCommGroup [CommGroup α] : CommGroup αᵐᵒᵖ where toGroup := instGroup __ := instCommSemigroup section Monoid variable [Monoid α] @[simp] lemma op_pow (x : α) (n : ℕ) : op (x ^ n) = op x ^ n := rfl @[simp] lemma unop_pow (x : αᵐᵒᵖ) (n : ℕ) : unop (x ^ n) = unop x ^ n := rfl end Monoid section DivInvMonoid variable [DivInvMonoid α] @[simp] lemma op_zpow (x : α) (z : ℤ) : op (x ^ z) = op x ^ z := rfl @[simp] lemma unop_zpow (x : αᵐᵒᵖ) (z : ℤ) : unop (x ^ z) = unop x ^ z := rfl end DivInvMonoid @[to_additive (attr := simp, norm_cast)] theorem op_natCast [NatCast α] (n : ℕ) : op (n : α) = n := rfl -- See note [no_index around OfNat.ofNat] @[to_additive (attr := simp)] theorem op_ofNat [NatCast α] (n : ℕ) [n.AtLeastTwo] : op (no_index (OfNat.ofNat n : α)) = OfNat.ofNat n := rfl @[to_additive (attr := simp, norm_cast)] theorem op_intCast [IntCast α] (n : ℤ) : op (n : α) = n := rfl @[to_additive (attr := simp, norm_cast)] theorem unop_natCast [NatCast α] (n : ℕ) : unop (n : αᵐᵒᵖ) = n := rfl -- See note [no_index around OfNat.ofNat] @[to_additive (attr := simp)] theorem unop_ofNat [NatCast α] (n : ℕ) [n.AtLeastTwo] : unop (no_index (OfNat.ofNat n : αᵐᵒᵖ)) = OfNat.ofNat n := rfl @[to_additive (attr := simp, norm_cast)] theorem unop_intCast [IntCast α] (n : ℤ) : unop (n : αᵐᵒᵖ) = n := rfl @[to_additive (attr := simp)] theorem unop_div [DivInvMonoid α] (x y : αᵐᵒᵖ) : unop (x / y) = (unop y)⁻¹ * unop x := rfl @[to_additive (attr := simp)] theorem op_div [DivInvMonoid α] (x y : α) : op (x / y) = (op y)⁻¹ * op x := by simp [div_eq_mul_inv] @[to_additive (attr := simp)] theorem semiconjBy_op [Mul α] {a x y : α} : SemiconjBy (op a) (op y) (op x) ↔ SemiconjBy a x y := by simp only [SemiconjBy, ← op_mul, op_inj, eq_comm] @[to_additive (attr := simp, nolint simpComm)] theorem semiconjBy_unop [Mul α] {a x y : αᵐᵒᵖ} : SemiconjBy (unop a) (unop y) (unop x) ↔ SemiconjBy a x y := by conv_rhs => rw [← op_unop a, ← op_unop x, ← op_unop y, semiconjBy_op] attribute [nolint simpComm] AddOpposite.addSemiconjBy_unop @[to_additive] theorem _root_.SemiconjBy.op [Mul α] {a x y : α} (h : SemiconjBy a x y) : SemiconjBy (op a) (op y) (op x) := semiconjBy_op.2 h @[to_additive] theorem _root_.SemiconjBy.unop [Mul α] {a x y : αᵐᵒᵖ} (h : SemiconjBy a x y) : SemiconjBy (unop a) (unop y) (unop x) := semiconjBy_unop.2 h @[to_additive] theorem _root_.Commute.op [Mul α] {x y : α} (h : Commute x y) : Commute (op x) (op y) := SemiconjBy.op h @[to_additive] nonrec theorem _root_.Commute.unop [Mul α] {x y : αᵐᵒᵖ} (h : Commute x y) : Commute (unop x) (unop y) := h.unop @[to_additive (attr := simp)] theorem commute_op [Mul α] {x y : α} : Commute (op x) (op y) ↔ Commute x y := semiconjBy_op @[to_additive (attr := simp, nolint simpComm)] theorem commute_unop [Mul α] {x y : αᵐᵒᵖ} : Commute (unop x) (unop y) ↔ Commute x y := semiconjBy_unop attribute [nolint simpComm] AddOpposite.addCommute_unop /-- The function `MulOpposite.op` is an additive equivalence. -/ @[simps! (config := { fullyApplied := false, simpRhs := true }) apply symm_apply] def opAddEquiv [Add α] : α ≃+ αᵐᵒᵖ := { opEquiv with map_add' := fun _ _ => rfl } @[simp] theorem opAddEquiv_toEquiv [Add α] : ((opAddEquiv : α ≃+ αᵐᵒᵖ) : α ≃ αᵐᵒᵖ) = opEquiv := rfl end MulOpposite /-! ### Multiplicative structures on `αᵃᵒᵖ` -/ namespace AddOpposite instance instSemigroup [Semigroup α] : Semigroup αᵃᵒᵖ := unop_injective.semigroup _ fun _ _ ↦ rfl instance instLeftCancelSemigroup [LeftCancelSemigroup α] : LeftCancelSemigroup αᵃᵒᵖ := unop_injective.leftCancelSemigroup _ fun _ _ => rfl instance instRightCancelSemigroup [RightCancelSemigroup α] : RightCancelSemigroup αᵃᵒᵖ := unop_injective.rightCancelSemigroup _ fun _ _ => rfl instance instCommSemigroup [CommSemigroup α] : CommSemigroup αᵃᵒᵖ := unop_injective.commSemigroup _ fun _ _ => rfl instance instMulOneClass [MulOneClass α] : MulOneClass αᵃᵒᵖ := unop_injective.mulOneClass _ (by exact rfl) fun _ _ => rfl instance pow {β} [Pow α β] : Pow αᵃᵒᵖ β where pow a b := op (unop a ^ b) @[simp] theorem op_pow {β} [Pow α β] (a : α) (b : β) : op (a ^ b) = op a ^ b := rfl @[simp] theorem unop_pow {β} [Pow α β] (a : αᵃᵒᵖ) (b : β) : unop (a ^ b) = unop a ^ b := rfl instance instMonoid [Monoid α] : Monoid αᵃᵒᵖ := unop_injective.monoid _ (by exact rfl) (fun _ _ => rfl) fun _ _ => rfl instance instCommMonoid [CommMonoid α] : CommMonoid αᵃᵒᵖ := unop_injective.commMonoid _ (by exact rfl) (fun _ _ => rfl) fun _ _ => rfl instance instDivInvMonoid [DivInvMonoid α] : DivInvMonoid αᵃᵒᵖ := unop_injective.divInvMonoid _ (by exact rfl) (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) fun _ _ => rfl instance instGroup [Group α] : Group αᵃᵒᵖ := unop_injective.group _ (by exact rfl) (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) fun _ _ => rfl instance instCommGroup [CommGroup α] : CommGroup αᵃᵒᵖ := unop_injective.commGroup _ (by exact rfl) (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) fun _ _ => rfl -- NOTE: `addMonoidWithOne α → addMonoidWithOne αᵃᵒᵖ` does not hold instance instAddCommMonoidWithOne [AddCommMonoidWithOne α] : AddCommMonoidWithOne αᵃᵒᵖ where toNatCast := instNatCast toOne := instOne __ := instAddCommMonoid natCast_zero := show op ((0 : ℕ) : α) = 0 by rw [Nat.cast_zero, op_zero] natCast_succ := show ∀ n, op ((n + 1 : ℕ) : α) = op ↑(n : ℕ) + 1 by simp [add_comm] instance instAddCommGroupWithOne [AddCommGroupWithOne α] : AddCommGroupWithOne αᵃᵒᵖ where toIntCast := instIntCast toAddCommGroup := instAddCommGroup __ := instAddCommMonoidWithOne intCast_ofNat _ := congr_arg op <| Int.cast_natCast _ intCast_negSucc _ := congr_arg op <| Int.cast_negSucc _ /-- The function `AddOpposite.op` is a multiplicative equivalence. -/ @[simps! (config := { fullyApplied := false, simpRhs := true })] def opMulEquiv [Mul α] : α ≃* αᵃᵒᵖ := { opEquiv with map_mul' := fun _ _ => rfl } @[simp] theorem opMulEquiv_toEquiv [Mul α] : ((opMulEquiv : α ≃* αᵃᵒᵖ) : α ≃ αᵃᵒᵖ) = opEquiv := rfl end AddOpposite open MulOpposite /-- Inversion on a group is a `MulEquiv` to the opposite group. When `G` is commutative, there is `MulEquiv.inv`. -/ @[to_additive (attr := simps! (config := { fullyApplied := false, simpRhs := true })) "Negation on an additive group is an `AddEquiv` to the opposite group. When `G` is commutative, there is `AddEquiv.inv`."] def MulEquiv.inv' (G : Type*) [DivisionMonoid G] : G ≃* Gᵐᵒᵖ := { (Equiv.inv G).trans opEquiv with map_mul' := fun x y => unop_injective <| mul_inv_rev x y } /-- A semigroup homomorphism `f : M →ₙ* N` such that `f x` commutes with `f y` for all `x, y` defines a semigroup homomorphism to `Nᵐᵒᵖ`. -/ @[to_additive (attr := simps (config := .asFn)) "An additive semigroup homomorphism `f : AddHom M N` such that `f x` additively commutes with `f y` for all `x, y` defines an additive semigroup homomorphism to `Sᵃᵒᵖ`."] def MulHom.toOpposite {M N : Type*} [Mul M] [Mul N] (f : M →ₙ* N) (hf : ∀ x y, Commute (f x) (f y)) : M →ₙ* Nᵐᵒᵖ where toFun := op ∘ f map_mul' x y := by simp [(hf x y).eq] /-- A semigroup homomorphism `f : M →ₙ* N` such that `f x` commutes with `f y` for all `x, y` defines a semigroup homomorphism from `Mᵐᵒᵖ`. -/ @[to_additive (attr := simps (config := .asFn)) "An additive semigroup homomorphism `f : AddHom M N` such that `f x` additively commutes with `f y` for all `x`, `y` defines an additive semigroup homomorphism from `Mᵃᵒᵖ`."] def MulHom.fromOpposite {M N : Type*} [Mul M] [Mul N] (f : M →ₙ* N) (hf : ∀ x y, Commute (f x) (f y)) : Mᵐᵒᵖ →ₙ* N where toFun := f ∘ MulOpposite.unop map_mul' _ _ := (f.map_mul _ _).trans (hf _ _).eq /-- A monoid homomorphism `f : M →* N` such that `f x` commutes with `f y` for all `x, y` defines a monoid homomorphism to `Nᵐᵒᵖ`. -/ @[to_additive (attr := simps (config := .asFn)) "An additive monoid homomorphism `f : M →+ N` such that `f x` additively commutes with `f y` for all `x, y` defines an additive monoid homomorphism to `Sᵃᵒᵖ`."] def MonoidHom.toOpposite {M N : Type*} [MulOneClass M] [MulOneClass N] (f : M →* N) (hf : ∀ x y, Commute (f x) (f y)) : M →* Nᵐᵒᵖ where toFun := op ∘ f map_one' := congrArg op f.map_one map_mul' x y := by simp [(hf x y).eq] /-- A monoid homomorphism `f : M →* N` such that `f x` commutes with `f y` for all `x, y` defines a monoid homomorphism from `Mᵐᵒᵖ`. -/ @[to_additive (attr := simps (config := .asFn)) "An additive monoid homomorphism `f : M →+ N` such that `f x` additively commutes with `f y` for all `x`, `y` defines an additive monoid homomorphism from `Mᵃᵒᵖ`."] def MonoidHom.fromOpposite {M N : Type*} [MulOneClass M] [MulOneClass N] (f : M →* N) (hf : ∀ x y, Commute (f x) (f y)) : Mᵐᵒᵖ →* N where toFun := f ∘ MulOpposite.unop map_one' := f.map_one map_mul' _ _ := (f.map_mul _ _).trans (hf _ _).eq /-- The units of the opposites are equivalent to the opposites of the units. -/ @[to_additive "The additive units of the additive opposites are equivalent to the additive opposites of the additive units."] def Units.opEquiv {M} [Monoid M] : Mᵐᵒᵖˣ ≃* Mˣᵐᵒᵖ where toFun u := op ⟨unop u, unop ↑u⁻¹, op_injective u.4, op_injective u.3⟩ invFun := MulOpposite.rec' fun u => ⟨op ↑u, op ↑u⁻¹, unop_injective <| u.4, unop_injective u.3⟩ map_mul' x y := unop_injective <| Units.ext <| rfl left_inv x := Units.ext <| by simp right_inv x := unop_injective <| Units.ext <| by rfl @[to_additive (attr := simp)] theorem Units.coe_unop_opEquiv {M} [Monoid M] (u : Mᵐᵒᵖˣ) : ((Units.opEquiv u).unop : M) = unop (u : Mᵐᵒᵖ) := rfl @[to_additive (attr := simp)] theorem Units.coe_opEquiv_symm {M} [Monoid M] (u : Mˣᵐᵒᵖ) : (Units.opEquiv.symm u : Mᵐᵒᵖ) = op (u.unop : M) := rfl @[to_additive] nonrec theorem IsUnit.op {M} [Monoid M] {m : M} (h : IsUnit m) : IsUnit (op m) := let ⟨u, hu⟩ := h hu ▸ ⟨Units.opEquiv.symm (op u), rfl⟩ @[to_additive] nonrec theorem IsUnit.unop {M} [Monoid M] {m : Mᵐᵒᵖ} (h : IsUnit m) : IsUnit (unop m) := let ⟨u, hu⟩ := h hu ▸ ⟨unop (Units.opEquiv u), rfl⟩ @[to_additive (attr := simp)] theorem isUnit_op {M} [Monoid M] {m : M} : IsUnit (op m) ↔ IsUnit m := ⟨IsUnit.unop, IsUnit.op⟩ @[to_additive (attr := simp)] theorem isUnit_unop {M} [Monoid M] {m : Mᵐᵒᵖ} : IsUnit (unop m) ↔ IsUnit m := ⟨IsUnit.op, IsUnit.unop⟩ /-- A semigroup homomorphism `M →ₙ* N` can equivalently be viewed as a semigroup homomorphism `Mᵐᵒᵖ →ₙ* Nᵐᵒᵖ`. This is the action of the (fully faithful) `ᵐᵒᵖ`-functor on morphisms. -/ @[to_additive (attr := simps) "An additive semigroup homomorphism `AddHom M N` can equivalently be viewed as an additive semigroup homomorphism `AddHom Mᵃᵒᵖ Nᵃᵒᵖ`. This is the action of the (fully faithful)`ᵃᵒᵖ`-functor on morphisms."] def MulHom.op {M N} [Mul M] [Mul N] : (M →ₙ* N) ≃ (Mᵐᵒᵖ →ₙ* Nᵐᵒᵖ) where toFun f := { toFun := MulOpposite.op ∘ f ∘ unop, map_mul' := fun x y => unop_injective (f.map_mul y.unop x.unop) } invFun f := { toFun := unop ∘ f ∘ MulOpposite.op, map_mul' := fun x y => congrArg unop (f.map_mul (MulOpposite.op y) (MulOpposite.op x)) } left_inv _ := rfl right_inv _ := rfl /-- The 'unopposite' of a semigroup homomorphism `Mᵐᵒᵖ →ₙ* Nᵐᵒᵖ`. Inverse to `MulHom.op`. -/ @[to_additive (attr := simp) "The 'unopposite' of an additive semigroup homomorphism `Mᵃᵒᵖ →ₙ+ Nᵃᵒᵖ`. Inverse to `AddHom.op`."] def MulHom.unop {M N} [Mul M] [Mul N] : (Mᵐᵒᵖ →ₙ* Nᵐᵒᵖ) ≃ (M →ₙ* N) := MulHom.op.symm /-- An additive semigroup homomorphism `AddHom M N` can equivalently be viewed as an additive homomorphism `AddHom Mᵐᵒᵖ Nᵐᵒᵖ`. This is the action of the (fully faithful) `ᵐᵒᵖ`-functor on morphisms. -/ @[simps] def AddHom.mulOp {M N} [Add M] [Add N] : AddHom M N ≃ AddHom Mᵐᵒᵖ Nᵐᵒᵖ where toFun f := { toFun := MulOpposite.op ∘ f ∘ MulOpposite.unop, map_add' := fun x y => unop_injective (f.map_add x.unop y.unop) } invFun f := { toFun := MulOpposite.unop ∘ f ∘ MulOpposite.op, map_add' := fun x y => congrArg MulOpposite.unop (f.map_add (MulOpposite.op x) (MulOpposite.op y)) } left_inv _ := rfl right_inv _ := rfl /-- The 'unopposite' of an additive semigroup hom `αᵐᵒᵖ →+ βᵐᵒᵖ`. Inverse to `AddHom.mul_op`. -/ @[simp] def AddHom.mulUnop {α β} [Add α] [Add β] : AddHom αᵐᵒᵖ βᵐᵒᵖ ≃ AddHom α β := AddHom.mulOp.symm /-- A monoid homomorphism `M →* N` can equivalently be viewed as a monoid homomorphism `Mᵐᵒᵖ →* Nᵐᵒᵖ`. This is the action of the (fully faithful) `ᵐᵒᵖ`-functor on morphisms. -/ @[to_additive (attr := simps) "An additive monoid homomorphism `M →+ N` can equivalently be viewed as an additive monoid homomorphism `Mᵃᵒᵖ →+ Nᵃᵒᵖ`. This is the action of the (fully faithful) `ᵃᵒᵖ`-functor on morphisms."] def MonoidHom.op {M N} [MulOneClass M] [MulOneClass N] : (M →* N) ≃ (Mᵐᵒᵖ →* Nᵐᵒᵖ) where toFun f := { toFun := MulOpposite.op ∘ f ∘ unop, map_one' := congrArg MulOpposite.op f.map_one, map_mul' := fun x y => unop_injective (f.map_mul y.unop x.unop) } invFun f := { toFun := unop ∘ f ∘ MulOpposite.op, map_one' := congrArg unop f.map_one, map_mul' := fun x y => congrArg unop (f.map_mul (MulOpposite.op y) (MulOpposite.op x)) } left_inv _ := rfl right_inv _ := rfl /-- The 'unopposite' of a monoid homomorphism `Mᵐᵒᵖ →* Nᵐᵒᵖ`. Inverse to `MonoidHom.op`. -/ @[to_additive (attr := simp) "The 'unopposite' of an additive monoid homomorphism `Mᵃᵒᵖ →+ Nᵃᵒᵖ`. Inverse to `AddMonoidHom.op`."] def MonoidHom.unop {M N} [MulOneClass M] [MulOneClass N] : (Mᵐᵒᵖ →* Nᵐᵒᵖ) ≃ (M →* N) := MonoidHom.op.symm /-- A monoid is isomorphic to the opposite of its opposite. -/ @[to_additive (attr := simps!) "A additive monoid is isomorphic to the opposite of its opposite."] def MulEquiv.opOp (M : Type*) [Mul M] : M ≃* Mᵐᵒᵖᵐᵒᵖ where __ := MulOpposite.opEquiv.trans MulOpposite.opEquiv map_mul' _ _ := rfl /-- An additive homomorphism `M →+ N` can equivalently be viewed as an additive homomorphism `Mᵐᵒᵖ →+ Nᵐᵒᵖ`. This is the action of the (fully faithful) `ᵐᵒᵖ`-functor on morphisms. -/ @[simps] def AddMonoidHom.mulOp {M N} [AddZeroClass M] [AddZeroClass N] : (M →+ N) ≃ (Mᵐᵒᵖ →+ Nᵐᵒᵖ) where toFun f := { toFun := MulOpposite.op ∘ f ∘ MulOpposite.unop, map_zero' := unop_injective f.map_zero, map_add' := fun x y => unop_injective (f.map_add x.unop y.unop) } invFun f := { toFun := MulOpposite.unop ∘ f ∘ MulOpposite.op, map_zero' := congrArg MulOpposite.unop f.map_zero, map_add' := fun x y => congrArg MulOpposite.unop (f.map_add (MulOpposite.op x) (MulOpposite.op y)) } left_inv _ := rfl right_inv _ := rfl /-- The 'unopposite' of an additive monoid hom `αᵐᵒᵖ →+ βᵐᵒᵖ`. Inverse to `AddMonoidHom.mul_op`. -/ @[simp] def AddMonoidHom.mulUnop {α β} [AddZeroClass α] [AddZeroClass β] : (αᵐᵒᵖ →+ βᵐᵒᵖ) ≃ (α →+ β) := AddMonoidHom.mulOp.symm /-- An iso `α ≃+ β` can equivalently be viewed as an iso `αᵐᵒᵖ ≃+ βᵐᵒᵖ`. -/ @[simps] def AddEquiv.mulOp {α β} [Add α] [Add β] : α ≃+ β ≃ (αᵐᵒᵖ ≃+ βᵐᵒᵖ) where toFun f := opAddEquiv.symm.trans (f.trans opAddEquiv) invFun f := opAddEquiv.trans (f.trans opAddEquiv.symm) left_inv _ := rfl right_inv _ := rfl /-- The 'unopposite' of an iso `αᵐᵒᵖ ≃+ βᵐᵒᵖ`. Inverse to `AddEquiv.mul_op`. -/ @[simp] def AddEquiv.mulUnop {α β} [Add α] [Add β] : αᵐᵒᵖ ≃+ βᵐᵒᵖ ≃ (α ≃+ β) := AddEquiv.mulOp.symm /-- An iso `α ≃* β` can equivalently be viewed as an iso `αᵐᵒᵖ ≃* βᵐᵒᵖ`. -/ @[to_additive (attr := simps) "An iso `α ≃+ β` can equivalently be viewed as an iso `αᵃᵒᵖ ≃+ βᵃᵒᵖ`."] def MulEquiv.op {α β} [Mul α] [Mul β] : α ≃* β ≃ (αᵐᵒᵖ ≃* βᵐᵒᵖ) where toFun f := { toFun := MulOpposite.op ∘ f ∘ unop, invFun := MulOpposite.op ∘ f.symm ∘ unop, left_inv := fun x => unop_injective (f.symm_apply_apply x.unop), right_inv := fun x => unop_injective (f.apply_symm_apply x.unop), map_mul' := fun x y => unop_injective (f.map_mul y.unop x.unop) } invFun f := { toFun := unop ∘ f ∘ MulOpposite.op, invFun := unop ∘ f.symm ∘ MulOpposite.op, left_inv := fun x => by simp, right_inv := fun x => by simp, map_mul' := fun x y => congr_arg unop (f.map_mul (MulOpposite.op y) (MulOpposite.op x)) } left_inv _ := rfl right_inv _ := rfl /-- The 'unopposite' of an iso `αᵐᵒᵖ ≃* βᵐᵒᵖ`. Inverse to `MulEquiv.op`. -/ @[to_additive (attr := simp) "The 'unopposite' of an iso `αᵃᵒᵖ ≃+ βᵃᵒᵖ`. Inverse to `AddEquiv.op`."] def MulEquiv.unop {α β} [Mul α] [Mul β] : αᵐᵒᵖ ≃* βᵐᵒᵖ ≃ (α ≃* β) := MulEquiv.op.symm section Ext /-- This ext lemma changes equalities on `αᵐᵒᵖ →+ β` to equalities on `α →+ β`. This is useful because there are often ext lemmas for specific `α`s that will apply to an equality of `α →+ β` such as `Finsupp.addHom_ext'`. -/ @[ext] theorem AddMonoidHom.mul_op_ext {α β} [AddZeroClass α] [AddZeroClass β] (f g : αᵐᵒᵖ →+ β) (h : f.comp (opAddEquiv : α ≃+ αᵐᵒᵖ).toAddMonoidHom = g.comp (opAddEquiv : α ≃+ αᵐᵒᵖ).toAddMonoidHom) : f = g := AddMonoidHom.ext <| MulOpposite.rec' fun x => (DFunLike.congr_fun h : _) x end Ext
Algebra\Group\PNatPowAssoc.lean
/- Copyright (c) 2023 Scott Carnahan. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Carnahan -/ import Mathlib.Algebra.Group.Action.Prod import Mathlib.Data.PNat.Basic /-! # Typeclasses for power-associative structures In this file we define power-associativity for algebraic structures with a multiplication operation. The class is a Prop-valued mixin named `PNatPowAssoc`, where `PNat` means only strictly positive powers are considered. ## Results - `ppow_add` a defining property: `x ^ (k + n) = x ^ k * x ^ n` - `ppow_one` a defining property: `x ^ 1 = x` - `ppow_assoc` strictly positive powers of an element have associative multiplication. - `ppow_comm` `x ^ m * x ^ n = x ^ n * x ^ m` for strictly positive `m` and `n`. - `ppow_mul` `x ^ (m * n) = (x ^ m) ^ n` for strictly positive `m` and `n`. - `ppow_eq_pow` monoid exponentiation coincides with semigroup exponentiation. ## Instances - PNatPowAssoc for products and Pi types ## TODO * `NatPowAssoc` for `MulOneClass` - more or less the same flow * It seems unlikely that anyone will want `NatSMulAssoc` and `PNatSMulAssoc` as additive versions of power-associativity, but we have found that it is not hard to write. -/ -- TODO: -- assert_not_exists MonoidWithZero variable {M : Type*} /-- A `Prop`-valued mixin for power-associative multiplication in the non-unital setting. -/ class PNatPowAssoc (M : Type*) [Mul M] [Pow M ℕ+] : Prop where /-- Multiplication is power-associative. -/ protected ppow_add : ∀ (k n : ℕ+) (x : M), x ^ (k + n) = x ^ k * x ^ n /-- Exponent one is identity. -/ protected ppow_one : ∀ (x : M), x ^ (1 : ℕ+) = x section Mul variable [Mul M] [Pow M ℕ+] [PNatPowAssoc M] theorem ppow_add (k n : ℕ+) (x : M) : x ^ (k + n) = x ^ k * x ^ n := PNatPowAssoc.ppow_add k n x @[simp] theorem ppow_one (x : M) : x ^ (1 : ℕ+) = x := PNatPowAssoc.ppow_one x theorem ppow_mul_assoc (k m n : ℕ+) (x : M) : (x ^ k * x ^ m) * x ^ n = x ^ k * (x ^ m * x ^ n) := by simp only [← ppow_add, add_assoc] theorem ppow_mul_comm (m n : ℕ+) (x : M) : x ^ m * x ^ n = x ^ n * x ^ m := by simp only [← ppow_add, add_comm] theorem ppow_mul (x : M) (m n : ℕ+) : x ^ (m * n) = (x ^ m) ^ n := by refine PNat.recOn n ?_ fun k hk ↦ ?_ · rw [ppow_one, mul_one] · rw [ppow_add, ppow_one, mul_add, ppow_add, mul_one, hk] theorem ppow_mul' (x : M) (m n : ℕ+) : x ^ (m * n) = (x ^ n) ^ m := by rw [mul_comm] exact ppow_mul x n m end Mul instance Pi.instPNatPowAssoc {ι : Type*} {α : ι → Type*} [∀ i, Mul <| α i] [∀ i, Pow (α i) ℕ+] [∀ i, PNatPowAssoc <| α i] : PNatPowAssoc (∀ i, α i) where ppow_add _ _ _ := by ext; simp [ppow_add] ppow_one _ := by ext; simp instance Prod.instPNatPowAssoc {N : Type*} [Mul M] [Pow M ℕ+] [PNatPowAssoc M] [Mul N] [Pow N ℕ+] [PNatPowAssoc N] : PNatPowAssoc (M × N) where ppow_add _ _ _ := by ext <;> simp [ppow_add] ppow_one _ := by ext <;> simp theorem ppow_eq_pow [Monoid M] [Pow M ℕ+] [PNatPowAssoc M] (x : M) (n : ℕ+) : x ^ n = x ^ (n : ℕ) := by refine PNat.recOn n ?_ fun k hk ↦ ?_ · rw [ppow_one, PNat.one_coe, pow_one] · rw [ppow_add, ppow_one, PNat.add_coe, pow_add, PNat.one_coe, pow_one, ← hk]
Algebra\Group\Prod.lean
/- Copyright (c) 2020 Yury Kudryashov. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Simon Hudon, Patrick Massot, Yury Kudryashov -/ import Mathlib.Algebra.Group.Opposite import Mathlib.Algebra.Group.Units.Hom /-! # Monoid, group etc structures on `M × N` In this file we define one-binop (`Monoid`, `Group` etc) structures on `M × N`. We also prove trivial `simp` lemmas, and define the following operations on `MonoidHom`s: * `fst M N : M × N →* M`, `snd M N : M × N →* N`: projections `Prod.fst` and `Prod.snd` as `MonoidHom`s; * `inl M N : M →* M × N`, `inr M N : N →* M × N`: inclusions of first/second monoid into the product; * `f.prod g` : `M →* N × P`: sends `x` to `(f x, g x)`; * When `P` is commutative, `f.coprod g : M × N →* P` sends `(x, y)` to `f x * g y` (without the commutativity assumption on `P`, see `MonoidHom.noncommPiCoprod`); * `f.prodMap g : M × N → M' × N'`: `prod.map f g` as a `MonoidHom`, sends `(x, y)` to `(f x, g y)`. ## Main declarations * `mulMulHom`/`mulMonoidHom`: Multiplication bundled as a multiplicative/monoid homomorphism. * `divMonoidHom`: Division bundled as a monoid homomorphism. -/ assert_not_exists MonoidWithZero -- TODO: -- assert_not_exists AddMonoidWithOne assert_not_exists DenselyOrdered variable {A : Type*} {B : Type*} {G : Type*} {H : Type*} {M : Type*} {N : Type*} {P : Type*} namespace Prod @[to_additive] instance instMul [Mul M] [Mul N] : Mul (M × N) := ⟨fun p q => ⟨p.1 * q.1, p.2 * q.2⟩⟩ @[to_additive (attr := simp)] theorem fst_mul [Mul M] [Mul N] (p q : M × N) : (p * q).1 = p.1 * q.1 := rfl @[to_additive (attr := simp)] theorem snd_mul [Mul M] [Mul N] (p q : M × N) : (p * q).2 = p.2 * q.2 := rfl @[to_additive (attr := simp)] theorem mk_mul_mk [Mul M] [Mul N] (a₁ a₂ : M) (b₁ b₂ : N) : (a₁, b₁) * (a₂, b₂) = (a₁ * a₂, b₁ * b₂) := rfl @[to_additive (attr := simp)] theorem swap_mul [Mul M] [Mul N] (p q : M × N) : (p * q).swap = p.swap * q.swap := rfl @[to_additive] theorem mul_def [Mul M] [Mul N] (p q : M × N) : p * q = (p.1 * q.1, p.2 * q.2) := rfl @[to_additive] theorem one_mk_mul_one_mk [Monoid M] [Mul N] (b₁ b₂ : N) : ((1 : M), b₁) * (1, b₂) = (1, b₁ * b₂) := by rw [mk_mul_mk, mul_one] @[to_additive] theorem mk_one_mul_mk_one [Mul M] [Monoid N] (a₁ a₂ : M) : (a₁, (1 : N)) * (a₂, 1) = (a₁ * a₂, 1) := by rw [mk_mul_mk, mul_one] @[to_additive] instance instOne [One M] [One N] : One (M × N) := ⟨(1, 1)⟩ @[to_additive (attr := simp)] theorem fst_one [One M] [One N] : (1 : M × N).1 = 1 := rfl @[to_additive (attr := simp)] theorem snd_one [One M] [One N] : (1 : M × N).2 = 1 := rfl @[to_additive] theorem one_eq_mk [One M] [One N] : (1 : M × N) = (1, 1) := rfl @[to_additive (attr := simp)] theorem mk_eq_one [One M] [One N] {x : M} {y : N} : (x, y) = 1 ↔ x = 1 ∧ y = 1 := mk.inj_iff @[to_additive (attr := simp)] theorem swap_one [One M] [One N] : (1 : M × N).swap = 1 := rfl @[to_additive] theorem fst_mul_snd [MulOneClass M] [MulOneClass N] (p : M × N) : (p.fst, 1) * (1, p.snd) = p := Prod.ext (mul_one p.1) (one_mul p.2) @[to_additive] instance instInv [Inv M] [Inv N] : Inv (M × N) := ⟨fun p => (p.1⁻¹, p.2⁻¹)⟩ @[to_additive (attr := simp)] theorem fst_inv [Inv G] [Inv H] (p : G × H) : p⁻¹.1 = p.1⁻¹ := rfl @[to_additive (attr := simp)] theorem snd_inv [Inv G] [Inv H] (p : G × H) : p⁻¹.2 = p.2⁻¹ := rfl @[to_additive (attr := simp)] theorem inv_mk [Inv G] [Inv H] (a : G) (b : H) : (a, b)⁻¹ = (a⁻¹, b⁻¹) := rfl @[to_additive (attr := simp)] theorem swap_inv [Inv G] [Inv H] (p : G × H) : p⁻¹.swap = p.swap⁻¹ := rfl @[to_additive] instance [InvolutiveInv M] [InvolutiveInv N] : InvolutiveInv (M × N) := { inv_inv := fun _ => Prod.ext (inv_inv _) (inv_inv _) } @[to_additive] instance instDiv [Div M] [Div N] : Div (M × N) := ⟨fun p q => ⟨p.1 / q.1, p.2 / q.2⟩⟩ @[to_additive (attr := simp)] theorem fst_div [Div G] [Div H] (a b : G × H) : (a / b).1 = a.1 / b.1 := rfl @[to_additive (attr := simp)] theorem snd_div [Div G] [Div H] (a b : G × H) : (a / b).2 = a.2 / b.2 := rfl @[to_additive (attr := simp)] theorem mk_div_mk [Div G] [Div H] (x₁ x₂ : G) (y₁ y₂ : H) : (x₁, y₁) / (x₂, y₂) = (x₁ / x₂, y₁ / y₂) := rfl @[to_additive (attr := simp)] theorem swap_div [Div G] [Div H] (a b : G × H) : (a / b).swap = a.swap / b.swap := rfl @[to_additive] instance instSemigroup [Semigroup M] [Semigroup N] : Semigroup (M × N) := { mul_assoc := fun _ _ _ => mk.inj_iff.mpr ⟨mul_assoc _ _ _, mul_assoc _ _ _⟩ } @[to_additive] instance instCommSemigroup [CommSemigroup G] [CommSemigroup H] : CommSemigroup (G × H) := { mul_comm := fun _ _ => mk.inj_iff.mpr ⟨mul_comm _ _, mul_comm _ _⟩ } @[to_additive] instance instMulOneClass [MulOneClass M] [MulOneClass N] : MulOneClass (M × N) := { one_mul := fun a => Prod.recOn a fun _ _ => mk.inj_iff.mpr ⟨one_mul _, one_mul _⟩, mul_one := fun a => Prod.recOn a fun _ _ => mk.inj_iff.mpr ⟨mul_one _, mul_one _⟩ } @[to_additive] instance instMonoid [Monoid M] [Monoid N] : Monoid (M × N) := { npow := fun z a => ⟨Monoid.npow z a.1, Monoid.npow z a.2⟩, npow_zero := fun z => Prod.ext (Monoid.npow_zero _) (Monoid.npow_zero _), npow_succ := fun z a => Prod.ext (Monoid.npow_succ _ _) (Monoid.npow_succ _ _), one_mul := by simp, mul_one := by simp } @[to_additive Prod.subNegMonoid] instance [DivInvMonoid G] [DivInvMonoid H] : DivInvMonoid (G × H) := { div_eq_mul_inv := fun _ _ => mk.inj_iff.mpr ⟨div_eq_mul_inv _ _, div_eq_mul_inv _ _⟩, zpow := fun z a => ⟨DivInvMonoid.zpow z a.1, DivInvMonoid.zpow z a.2⟩, zpow_zero' := fun _ => Prod.ext (DivInvMonoid.zpow_zero' _) (DivInvMonoid.zpow_zero' _), zpow_succ' := fun _ _ => Prod.ext (DivInvMonoid.zpow_succ' _ _) (DivInvMonoid.zpow_succ' _ _), zpow_neg' := fun _ _ => Prod.ext (DivInvMonoid.zpow_neg' _ _) (DivInvMonoid.zpow_neg' _ _) } @[to_additive] instance [DivisionMonoid G] [DivisionMonoid H] : DivisionMonoid (G × H) := { mul_inv_rev := fun a b => Prod.ext (mul_inv_rev _ _) (mul_inv_rev _ _), inv_eq_of_mul := fun a b h => Prod.ext (inv_eq_of_mul_eq_one_right <| congr_arg fst h) (inv_eq_of_mul_eq_one_right <| congr_arg snd h), inv_inv := by simp } @[to_additive SubtractionCommMonoid] instance [DivisionCommMonoid G] [DivisionCommMonoid H] : DivisionCommMonoid (G × H) := { mul_comm := fun ⟨g₁ , h₁⟩ ⟨_, _⟩ => by rw [mk_mul_mk, mul_comm g₁, mul_comm h₁]; rfl } @[to_additive] instance instGroup [Group G] [Group H] : Group (G × H) := { mul_left_inv := fun _ => mk.inj_iff.mpr ⟨mul_left_inv _, mul_left_inv _⟩ } @[to_additive] instance [Mul G] [Mul H] [IsLeftCancelMul G] [IsLeftCancelMul H] : IsLeftCancelMul (G × H) where mul_left_cancel _ _ _ h := Prod.ext (mul_left_cancel (Prod.ext_iff.1 h).1) (mul_left_cancel (Prod.ext_iff.1 h).2) @[to_additive] instance [Mul G] [Mul H] [IsRightCancelMul G] [IsRightCancelMul H] : IsRightCancelMul (G × H) where mul_right_cancel _ _ _ h := Prod.ext (mul_right_cancel (Prod.ext_iff.1 h).1) (mul_right_cancel (Prod.ext_iff.1 h).2) @[to_additive] instance [Mul G] [Mul H] [IsCancelMul G] [IsCancelMul H] : IsCancelMul (G × H) where @[to_additive] instance [LeftCancelSemigroup G] [LeftCancelSemigroup H] : LeftCancelSemigroup (G × H) := { mul_left_cancel := fun _ _ _ => mul_left_cancel } @[to_additive] instance [RightCancelSemigroup G] [RightCancelSemigroup H] : RightCancelSemigroup (G × H) := { mul_right_cancel := fun _ _ _ => mul_right_cancel } @[to_additive] instance [LeftCancelMonoid M] [LeftCancelMonoid N] : LeftCancelMonoid (M × N) := { mul_one := by simp, one_mul := by simp } @[to_additive] instance [RightCancelMonoid M] [RightCancelMonoid N] : RightCancelMonoid (M × N) := { mul_one := by simp, one_mul := by simp } @[to_additive] instance [CancelMonoid M] [CancelMonoid N] : CancelMonoid (M × N) := { mul_right_cancel := by simp only [mul_left_inj, imp_self, forall_const] } @[to_additive] instance instCommMonoid [CommMonoid M] [CommMonoid N] : CommMonoid (M × N) := { mul_comm := fun ⟨m₁, n₁⟩ ⟨_, _⟩ => by rw [mk_mul_mk, mk_mul_mk, mul_comm m₁, mul_comm n₁] } @[to_additive] instance [CancelCommMonoid M] [CancelCommMonoid N] : CancelCommMonoid (M × N) := { mul_comm := fun ⟨m₁, n₁⟩ ⟨_, _⟩ => by rw [mk_mul_mk, mk_mul_mk, mul_comm m₁, mul_comm n₁] } @[to_additive] instance instCommGroup [CommGroup G] [CommGroup H] : CommGroup (G × H) := { mul_comm := fun ⟨g₁, h₁⟩ ⟨_, _⟩ => by rw [mk_mul_mk, mk_mul_mk, mul_comm g₁, mul_comm h₁] } end Prod section variable [Mul M] [Mul N] @[to_additive AddSemiconjBy.prod] theorem SemiconjBy.prod {x y z : M × N} (hm : SemiconjBy x.1 y.1 z.1) (hn : SemiconjBy x.2 y.2 z.2) : SemiconjBy x y z := Prod.ext hm hn @[to_additive] theorem Prod.semiconjBy_iff {x y z : M × N} : SemiconjBy x y z ↔ SemiconjBy x.1 y.1 z.1 ∧ SemiconjBy x.2 y.2 z.2 := Prod.ext_iff @[to_additive AddCommute.prod] theorem Commute.prod {x y : M × N} (hm : Commute x.1 y.1) (hn : Commute x.2 y.2) : Commute x y := .prod hm hn @[to_additive] theorem Prod.commute_iff {x y : M × N} : Commute x y ↔ Commute x.1 y.1 ∧ Commute x.2 y.2 := semiconjBy_iff end namespace MulHom section Prod variable (M N) [Mul M] [Mul N] [Mul P] /-- Given magmas `M`, `N`, the natural projection homomorphism from `M × N` to `M`. -/ @[to_additive "Given additive magmas `A`, `B`, the natural projection homomorphism from `A × B` to `A`"] def fst : M × N →ₙ* M := ⟨Prod.fst, fun _ _ => rfl⟩ /-- Given magmas `M`, `N`, the natural projection homomorphism from `M × N` to `N`. -/ @[to_additive "Given additive magmas `A`, `B`, the natural projection homomorphism from `A × B` to `B`"] def snd : M × N →ₙ* N := ⟨Prod.snd, fun _ _ => rfl⟩ variable {M N} @[to_additive (attr := simp)] theorem coe_fst : ⇑(fst M N) = Prod.fst := rfl @[to_additive (attr := simp)] theorem coe_snd : ⇑(snd M N) = Prod.snd := rfl /-- Combine two `MonoidHom`s `f : M →ₙ* N`, `g : M →ₙ* P` into `f.prod g : M →ₙ* (N × P)` given by `(f.prod g) x = (f x, g x)`. -/ @[to_additive prod "Combine two `AddMonoidHom`s `f : AddHom M N`, `g : AddHom M P` into `f.prod g : AddHom M (N × P)` given by `(f.prod g) x = (f x, g x)`"] protected def prod (f : M →ₙ* N) (g : M →ₙ* P) : M →ₙ* N × P where toFun := Pi.prod f g map_mul' x y := Prod.ext (f.map_mul x y) (g.map_mul x y) @[to_additive coe_prod] theorem coe_prod (f : M →ₙ* N) (g : M →ₙ* P) : ⇑(f.prod g) = Pi.prod f g := rfl @[to_additive (attr := simp) prod_apply] theorem prod_apply (f : M →ₙ* N) (g : M →ₙ* P) (x) : f.prod g x = (f x, g x) := rfl @[to_additive (attr := simp) fst_comp_prod] theorem fst_comp_prod (f : M →ₙ* N) (g : M →ₙ* P) : (fst N P).comp (f.prod g) = f := ext fun _ => rfl @[to_additive (attr := simp) snd_comp_prod] theorem snd_comp_prod (f : M →ₙ* N) (g : M →ₙ* P) : (snd N P).comp (f.prod g) = g := ext fun _ => rfl @[to_additive (attr := simp) prod_unique] theorem prod_unique (f : M →ₙ* N × P) : ((fst N P).comp f).prod ((snd N P).comp f) = f := ext fun x => by simp only [prod_apply, coe_fst, coe_snd, comp_apply] end Prod section prodMap variable {M' : Type*} {N' : Type*} [Mul M] [Mul N] [Mul M'] [Mul N'] [Mul P] (f : M →ₙ* M') (g : N →ₙ* N') /-- `Prod.map` as a `MonoidHom`. -/ @[to_additive prodMap "`Prod.map` as an `AddMonoidHom`"] def prodMap : M × N →ₙ* M' × N' := (f.comp (fst M N)).prod (g.comp (snd M N)) @[to_additive prodMap_def] theorem prodMap_def : prodMap f g = (f.comp (fst M N)).prod (g.comp (snd M N)) := rfl @[to_additive (attr := simp) coe_prodMap] theorem coe_prodMap : ⇑(prodMap f g) = Prod.map f g := rfl @[to_additive prod_comp_prodMap] theorem prod_comp_prodMap (f : P →ₙ* M) (g : P →ₙ* N) (f' : M →ₙ* M') (g' : N →ₙ* N') : (f'.prodMap g').comp (f.prod g) = (f'.comp f).prod (g'.comp g) := rfl end prodMap section Coprod variable [Mul M] [Mul N] [CommSemigroup P] (f : M →ₙ* P) (g : N →ₙ* P) /-- Coproduct of two `MulHom`s with the same codomain: `f.coprod g (p : M × N) = f p.1 * g p.2`. (Commutative codomain; for the general case, see `MulHom.noncommCoprod`) -/ @[to_additive "Coproduct of two `AddHom`s with the same codomain: `f.coprod g (p : M × N) = f p.1 + g p.2`. (Commutative codomain; for the general case, see `AddHom.noncommCoprod`)"] def coprod : M × N →ₙ* P := f.comp (fst M N) * g.comp (snd M N) @[to_additive (attr := simp)] theorem coprod_apply (p : M × N) : f.coprod g p = f p.1 * g p.2 := rfl @[to_additive] theorem comp_coprod {Q : Type*} [CommSemigroup Q] (h : P →ₙ* Q) (f : M →ₙ* P) (g : N →ₙ* P) : h.comp (f.coprod g) = (h.comp f).coprod (h.comp g) := ext fun x => by simp end Coprod end MulHom namespace MonoidHom variable (M N) [MulOneClass M] [MulOneClass N] /-- Given monoids `M`, `N`, the natural projection homomorphism from `M × N` to `M`. -/ @[to_additive "Given additive monoids `A`, `B`, the natural projection homomorphism from `A × B` to `A`"] def fst : M × N →* M := { toFun := Prod.fst, map_one' := rfl, map_mul' := fun _ _ => rfl } /-- Given monoids `M`, `N`, the natural projection homomorphism from `M × N` to `N`. -/ @[to_additive "Given additive monoids `A`, `B`, the natural projection homomorphism from `A × B` to `B`"] def snd : M × N →* N := { toFun := Prod.snd, map_one' := rfl, map_mul' := fun _ _ => rfl } /-- Given monoids `M`, `N`, the natural inclusion homomorphism from `M` to `M × N`. -/ @[to_additive "Given additive monoids `A`, `B`, the natural inclusion homomorphism from `A` to `A × B`."] def inl : M →* M × N := { toFun := fun x => (x, 1), map_one' := rfl, map_mul' := fun _ _ => Prod.ext rfl (one_mul 1).symm } /-- Given monoids `M`, `N`, the natural inclusion homomorphism from `N` to `M × N`. -/ @[to_additive "Given additive monoids `A`, `B`, the natural inclusion homomorphism from `B` to `A × B`."] def inr : N →* M × N := { toFun := fun y => (1, y), map_one' := rfl, map_mul' := fun _ _ => Prod.ext (one_mul 1).symm rfl } variable {M N} @[to_additive (attr := simp)] theorem coe_fst : ⇑(fst M N) = Prod.fst := rfl @[to_additive (attr := simp)] theorem coe_snd : ⇑(snd M N) = Prod.snd := rfl @[to_additive (attr := simp)] theorem inl_apply (x) : inl M N x = (x, 1) := rfl @[to_additive (attr := simp)] theorem inr_apply (y) : inr M N y = (1, y) := rfl @[to_additive (attr := simp)] theorem fst_comp_inl : (fst M N).comp (inl M N) = id M := rfl @[to_additive (attr := simp)] theorem snd_comp_inl : (snd M N).comp (inl M N) = 1 := rfl @[to_additive (attr := simp)] theorem fst_comp_inr : (fst M N).comp (inr M N) = 1 := rfl @[to_additive (attr := simp)] theorem snd_comp_inr : (snd M N).comp (inr M N) = id N := rfl @[to_additive] theorem commute_inl_inr (m : M) (n : N) : Commute (inl M N m) (inr M N n) := Commute.prod (.one_right m) (.one_left n) section Prod variable [MulOneClass P] /-- Combine two `MonoidHom`s `f : M →* N`, `g : M →* P` into `f.prod g : M →* N × P` given by `(f.prod g) x = (f x, g x)`. -/ @[to_additive prod "Combine two `AddMonoidHom`s `f : M →+ N`, `g : M →+ P` into `f.prod g : M →+ N × P` given by `(f.prod g) x = (f x, g x)`"] protected def prod (f : M →* N) (g : M →* P) : M →* N × P where toFun := Pi.prod f g map_one' := Prod.ext f.map_one g.map_one map_mul' x y := Prod.ext (f.map_mul x y) (g.map_mul x y) @[to_additive coe_prod] theorem coe_prod (f : M →* N) (g : M →* P) : ⇑(f.prod g) = Pi.prod f g := rfl @[to_additive (attr := simp) prod_apply] theorem prod_apply (f : M →* N) (g : M →* P) (x) : f.prod g x = (f x, g x) := rfl @[to_additive (attr := simp) fst_comp_prod] theorem fst_comp_prod (f : M →* N) (g : M →* P) : (fst N P).comp (f.prod g) = f := ext fun _ => rfl @[to_additive (attr := simp) snd_comp_prod] theorem snd_comp_prod (f : M →* N) (g : M →* P) : (snd N P).comp (f.prod g) = g := ext fun _ => rfl @[to_additive (attr := simp) prod_unique] theorem prod_unique (f : M →* N × P) : ((fst N P).comp f).prod ((snd N P).comp f) = f := ext fun x => by simp only [prod_apply, coe_fst, coe_snd, comp_apply] end Prod section prodMap variable {M' : Type*} {N' : Type*} [MulOneClass M'] [MulOneClass N'] [MulOneClass P] (f : M →* M') (g : N →* N') /-- `prod.map` as a `MonoidHom`. -/ @[to_additive prodMap "`prod.map` as an `AddMonoidHom`."] def prodMap : M × N →* M' × N' := (f.comp (fst M N)).prod (g.comp (snd M N)) @[to_additive prodMap_def] theorem prodMap_def : prodMap f g = (f.comp (fst M N)).prod (g.comp (snd M N)) := rfl @[to_additive (attr := simp) coe_prodMap] theorem coe_prodMap : ⇑(prodMap f g) = Prod.map f g := rfl @[to_additive prod_comp_prodMap] theorem prod_comp_prodMap (f : P →* M) (g : P →* N) (f' : M →* M') (g' : N →* N') : (f'.prodMap g').comp (f.prod g) = (f'.comp f).prod (g'.comp g) := rfl end prodMap section Coprod variable [CommMonoid P] (f : M →* P) (g : N →* P) /-- Coproduct of two `MonoidHom`s with the same codomain: `f.coprod g (p : M × N) = f p.1 * g p.2`. (Commutative case; for the general case, see `MonoidHom.noncommCoprod`.)-/ @[to_additive "Coproduct of two `AddMonoidHom`s with the same codomain: `f.coprod g (p : M × N) = f p.1 + g p.2`. (Commutative case; for the general case, see `AddHom.noncommCoprod`.)"] def coprod : M × N →* P := f.comp (fst M N) * g.comp (snd M N) @[to_additive (attr := simp)] theorem coprod_apply (p : M × N) : f.coprod g p = f p.1 * g p.2 := rfl @[to_additive (attr := simp)] theorem coprod_comp_inl : (f.coprod g).comp (inl M N) = f := ext fun x => by simp [coprod_apply] @[to_additive (attr := simp)] theorem coprod_comp_inr : (f.coprod g).comp (inr M N) = g := ext fun x => by simp [coprod_apply] @[to_additive (attr := simp)] theorem coprod_unique (f : M × N →* P) : (f.comp (inl M N)).coprod (f.comp (inr M N)) = f := ext fun x => by simp [coprod_apply, inl_apply, inr_apply, ← map_mul] @[to_additive (attr := simp)] theorem coprod_inl_inr {M N : Type*} [CommMonoid M] [CommMonoid N] : (inl M N).coprod (inr M N) = id (M × N) := coprod_unique (id <| M × N) @[to_additive] theorem comp_coprod {Q : Type*} [CommMonoid Q] (h : P →* Q) (f : M →* P) (g : N →* P) : h.comp (f.coprod g) = (h.comp f).coprod (h.comp g) := ext fun x => by simp end Coprod end MonoidHom namespace MulEquiv section variable [MulOneClass M] [MulOneClass N] /-- The equivalence between `M × N` and `N × M` given by swapping the components is multiplicative. -/ @[to_additive prodComm "The equivalence between `M × N` and `N × M` given by swapping the components is additive."] def prodComm : M × N ≃* N × M := { Equiv.prodComm M N with map_mul' := fun ⟨_, _⟩ ⟨_, _⟩ => rfl } @[to_additive (attr := simp) coe_prodComm] theorem coe_prodComm : ⇑(prodComm : M × N ≃* N × M) = Prod.swap := rfl @[to_additive (attr := simp) coe_prodComm_symm] theorem coe_prodComm_symm : ⇑(prodComm : M × N ≃* N × M).symm = Prod.swap := rfl variable {M' N' : Type*} [MulOneClass M'] [MulOneClass N'] section variable (M N M' N') /-- Four-way commutativity of `Prod`. The name matches `mul_mul_mul_comm`. -/ @[to_additive (attr := simps apply) prodProdProdComm "Four-way commutativity of `Prod`.\nThe name matches `mul_mul_mul_comm`"] def prodProdProdComm : (M × N) × M' × N' ≃* (M × M') × N × N' := { Equiv.prodProdProdComm M N M' N' with toFun := fun mnmn => ((mnmn.1.1, mnmn.2.1), (mnmn.1.2, mnmn.2.2)) invFun := fun mmnn => ((mmnn.1.1, mmnn.2.1), (mmnn.1.2, mmnn.2.2)) map_mul' := fun _mnmn _mnmn' => rfl } @[to_additive (attr := simp) prodProdProdComm_toEquiv] theorem prodProdProdComm_toEquiv : (prodProdProdComm M N M' N' : _ ≃ _) = Equiv.prodProdProdComm M N M' N' := rfl @[simp] theorem prodProdProdComm_symm : (prodProdProdComm M N M' N').symm = prodProdProdComm M M' N N' := rfl end /-- Product of multiplicative isomorphisms; the maps come from `Equiv.prodCongr`. -/ @[to_additive prodCongr "Product of additive isomorphisms; the maps come from `Equiv.prodCongr`."] def prodCongr (f : M ≃* M') (g : N ≃* N') : M × N ≃* M' × N' := { f.toEquiv.prodCongr g.toEquiv with map_mul' := fun _ _ => Prod.ext (f.map_mul _ _) (g.map_mul _ _) } /-- Multiplying by the trivial monoid doesn't change the structure. -/ @[to_additive uniqueProd "Multiplying by the trivial monoid doesn't change the structure."] def uniqueProd [Unique N] : N × M ≃* M := { Equiv.uniqueProd M N with map_mul' := fun _ _ => rfl } /-- Multiplying by the trivial monoid doesn't change the structure. -/ @[to_additive prodUnique "Multiplying by the trivial monoid doesn't change the structure."] def prodUnique [Unique N] : M × N ≃* M := { Equiv.prodUnique M N with map_mul' := fun _ _ => rfl } end section variable [Monoid M] [Monoid N] /-- The monoid equivalence between units of a product of two monoids, and the product of the units of each monoid. -/ @[to_additive prodAddUnits "The additive monoid equivalence between additive units of a product of two additive monoids, and the product of the additive units of each additive monoid."] def prodUnits : (M × N)ˣ ≃* Mˣ × Nˣ where toFun := (Units.map (MonoidHom.fst M N)).prod (Units.map (MonoidHom.snd M N)) invFun u := ⟨(u.1, u.2), (↑u.1⁻¹, ↑u.2⁻¹), by simp, by simp⟩ left_inv u := by simp only [MonoidHom.prod_apply, Units.coe_map, MonoidHom.coe_fst, MonoidHom.coe_snd, Prod.mk.eta, Units.coe_map_inv, Units.mk_val] right_inv := fun ⟨u₁, u₂⟩ => by simp only [Units.map, MonoidHom.coe_fst, Units.inv_eq_val_inv, MonoidHom.coe_snd, MonoidHom.prod_apply, Prod.mk.injEq] exact ⟨rfl, rfl⟩ map_mul' := MonoidHom.map_mul _ end end MulEquiv namespace Units open MulOpposite /-- Canonical homomorphism of monoids from `αˣ` into `α × αᵐᵒᵖ`. Used mainly to define the natural topology of `αˣ`. -/ @[to_additive (attr := simps) "Canonical homomorphism of additive monoids from `AddUnits α` into `α × αᵃᵒᵖ`. Used mainly to define the natural topology of `AddUnits α`."] def embedProduct (α : Type*) [Monoid α] : αˣ →* α × αᵐᵒᵖ where toFun x := ⟨x, op ↑x⁻¹⟩ map_one' := by simp only [inv_one, eq_self_iff_true, Units.val_one, op_one, Prod.mk_eq_one, and_self_iff] map_mul' x y := by simp only [mul_inv_rev, op_mul, Units.val_mul, Prod.mk_mul_mk] @[to_additive] theorem embedProduct_injective (α : Type*) [Monoid α] : Function.Injective (embedProduct α) := fun _ _ h => Units.ext <| (congr_arg Prod.fst h : _) end Units /-! ### Multiplication and division as homomorphisms -/ section BundledMulDiv variable {α : Type*} /-- Multiplication as a multiplicative homomorphism. -/ @[to_additive (attr := simps) "Addition as an additive homomorphism."] def mulMulHom [CommSemigroup α] : α × α →ₙ* α where toFun a := a.1 * a.2 map_mul' _ _ := mul_mul_mul_comm _ _ _ _ /-- Multiplication as a monoid homomorphism. -/ @[to_additive (attr := simps) "Addition as an additive monoid homomorphism."] def mulMonoidHom [CommMonoid α] : α × α →* α := { mulMulHom with map_one' := mul_one _ } /-- Division as a monoid homomorphism. -/ @[to_additive (attr := simps) "Subtraction as an additive monoid homomorphism."] def divMonoidHom [DivisionCommMonoid α] : α × α →* α where toFun a := a.1 / a.2 map_one' := div_one _ map_mul' _ _ := mul_div_mul_comm _ _ _ _ end BundledMulDiv
Algebra\Group\Support.lean
/- Copyright (c) 2020 Yury Kudryashov. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Yury Kudryashov -/ import Mathlib.Algebra.Group.Prod import Mathlib.Order.Cover /-! # Support of a function In this file we define `Function.support f = {x | f x ≠ 0}` and prove its basic properties. We also define `Function.mulSupport f = {x | f x ≠ 1}`. -/ assert_not_exists MonoidWithZero open Set namespace Function variable {α β A B M M' N P G : Type*} section One variable [One M] [One N] [One P] /-- `mulSupport` of a function is the set of points `x` such that `f x ≠ 1`. -/ @[to_additive "`support` of a function is the set of points `x` such that `f x ≠ 0`."] def mulSupport (f : α → M) : Set α := {x | f x ≠ 1} @[to_additive] theorem mulSupport_eq_preimage (f : α → M) : mulSupport f = f ⁻¹' {1}ᶜ := rfl @[to_additive] theorem nmem_mulSupport {f : α → M} {x : α} : x ∉ mulSupport f ↔ f x = 1 := not_not @[to_additive] theorem compl_mulSupport {f : α → M} : (mulSupport f)ᶜ = { x | f x = 1 } := ext fun _ => nmem_mulSupport @[to_additive (attr := simp)] theorem mem_mulSupport {f : α → M} {x : α} : x ∈ mulSupport f ↔ f x ≠ 1 := Iff.rfl @[to_additive (attr := simp)] theorem mulSupport_subset_iff {f : α → M} {s : Set α} : mulSupport f ⊆ s ↔ ∀ x, f x ≠ 1 → x ∈ s := Iff.rfl @[to_additive] theorem mulSupport_subset_iff' {f : α → M} {s : Set α} : mulSupport f ⊆ s ↔ ∀ x ∉ s, f x = 1 := forall_congr' fun _ => not_imp_comm @[to_additive] theorem mulSupport_eq_iff {f : α → M} {s : Set α} : mulSupport f = s ↔ (∀ x, x ∈ s → f x ≠ 1) ∧ ∀ x, x ∉ s → f x = 1 := by simp (config := { contextual := true }) only [Set.ext_iff, mem_mulSupport, ne_eq, iff_def, not_imp_comm, and_comm, forall_and] @[to_additive] theorem ext_iff_mulSupport {f g : α → M} : f = g ↔ f.mulSupport = g.mulSupport ∧ ∀ x ∈ f.mulSupport, f x = g x := ⟨fun h ↦ h ▸ ⟨rfl, fun _ _ ↦ rfl⟩, fun ⟨h₁, h₂⟩ ↦ funext fun x ↦ by if hx : x ∈ f.mulSupport then exact h₂ x hx else rw [nmem_mulSupport.1 hx, nmem_mulSupport.1 (mt (Set.ext_iff.1 h₁ x).2 hx)]⟩ @[to_additive] theorem mulSupport_update_of_ne_one [DecidableEq α] (f : α → M) (x : α) {y : M} (hy : y ≠ 1) : mulSupport (update f x y) = insert x (mulSupport f) := by ext a; rcases eq_or_ne a x with rfl | hne <;> simp [*] @[to_additive] theorem mulSupport_update_one [DecidableEq α] (f : α → M) (x : α) : mulSupport (update f x 1) = mulSupport f \ {x} := by ext a; rcases eq_or_ne a x with rfl | hne <;> simp [*] @[to_additive] theorem mulSupport_update_eq_ite [DecidableEq α] [DecidableEq M] (f : α → M) (x : α) (y : M) : mulSupport (update f x y) = if y = 1 then mulSupport f \ {x} else insert x (mulSupport f) := by rcases eq_or_ne y 1 with rfl | hy <;> simp [mulSupport_update_one, mulSupport_update_of_ne_one, *] @[to_additive] theorem mulSupport_extend_one_subset {f : α → M'} {g : α → N} : mulSupport (f.extend g 1) ⊆ f '' mulSupport g := mulSupport_subset_iff'.mpr fun x hfg ↦ by by_cases hf : ∃ a, f a = x · rw [extend, dif_pos hf, ← nmem_mulSupport] rw [← Classical.choose_spec hf] at hfg exact fun hg ↦ hfg ⟨_, hg, rfl⟩ · rw [extend_apply' _ _ _ hf]; rfl @[to_additive] theorem mulSupport_extend_one {f : α → M'} {g : α → N} (hf : f.Injective) : mulSupport (f.extend g 1) = f '' mulSupport g := mulSupport_extend_one_subset.antisymm <| by rintro _ ⟨x, hx, rfl⟩; rwa [mem_mulSupport, hf.extend_apply] @[to_additive] theorem mulSupport_disjoint_iff {f : α → M} {s : Set α} : Disjoint (mulSupport f) s ↔ EqOn f 1 s := by simp_rw [← subset_compl_iff_disjoint_right, mulSupport_subset_iff', not_mem_compl_iff, EqOn, Pi.one_apply] @[to_additive] theorem disjoint_mulSupport_iff {f : α → M} {s : Set α} : Disjoint s (mulSupport f) ↔ EqOn f 1 s := by rw [disjoint_comm, mulSupport_disjoint_iff] @[to_additive (attr := simp)] theorem mulSupport_eq_empty_iff {f : α → M} : mulSupport f = ∅ ↔ f = 1 := by #adaptation_note /-- This used to be `simp_rw` rather than `rw`, but this broke `to_additive` as of `nightly-2024-03-07` -/ rw [← subset_empty_iff, mulSupport_subset_iff', funext_iff] simp @[to_additive (attr := simp)] theorem mulSupport_nonempty_iff {f : α → M} : (mulSupport f).Nonempty ↔ f ≠ 1 := by rw [nonempty_iff_ne_empty, Ne, mulSupport_eq_empty_iff] @[to_additive] theorem range_subset_insert_image_mulSupport (f : α → M) : range f ⊆ insert 1 (f '' mulSupport f) := by simpa only [range_subset_iff, mem_insert_iff, or_iff_not_imp_left] using fun x (hx : x ∈ mulSupport f) => mem_image_of_mem f hx @[to_additive] lemma range_eq_image_or_of_mulSupport_subset {f : α → M} {k : Set α} (h : mulSupport f ⊆ k) : range f = f '' k ∨ range f = insert 1 (f '' k) := by apply (wcovBy_insert _ _).eq_or_eq (image_subset_range _ _) exact (range_subset_insert_image_mulSupport f).trans (insert_subset_insert (image_subset f h)) @[to_additive (attr := simp)] theorem mulSupport_one' : mulSupport (1 : α → M) = ∅ := mulSupport_eq_empty_iff.2 rfl @[to_additive (attr := simp)] theorem mulSupport_one : (mulSupport fun _ : α => (1 : M)) = ∅ := mulSupport_one' @[to_additive] theorem mulSupport_const {c : M} (hc : c ≠ 1) : (mulSupport fun _ : α => c) = Set.univ := by ext x simp [hc] @[to_additive] theorem mulSupport_binop_subset (op : M → N → P) (op1 : op 1 1 = 1) (f : α → M) (g : α → N) : (mulSupport fun x => op (f x) (g x)) ⊆ mulSupport f ∪ mulSupport g := fun x hx => not_or_of_imp fun hf hg => hx <| by simp only [hf, hg, op1] @[to_additive] theorem mulSupport_comp_subset {g : M → N} (hg : g 1 = 1) (f : α → M) : mulSupport (g ∘ f) ⊆ mulSupport f := fun x => mt fun h => by simp only [(· ∘ ·), *] @[to_additive] theorem mulSupport_subset_comp {g : M → N} (hg : ∀ {x}, g x = 1 → x = 1) (f : α → M) : mulSupport f ⊆ mulSupport (g ∘ f) := fun _ => mt hg @[to_additive] theorem mulSupport_comp_eq (g : M → N) (hg : ∀ {x}, g x = 1 ↔ x = 1) (f : α → M) : mulSupport (g ∘ f) = mulSupport f := Set.ext fun _ => not_congr hg @[to_additive] theorem mulSupport_comp_eq_of_range_subset {g : M → N} {f : α → M} (hg : ∀ {x}, x ∈ range f → (g x = 1 ↔ x = 1)) : mulSupport (g ∘ f) = mulSupport f := Set.ext fun x ↦ not_congr <| by rw [Function.comp, hg (mem_range_self x)] @[to_additive] theorem mulSupport_comp_eq_preimage (g : β → M) (f : α → β) : mulSupport (g ∘ f) = f ⁻¹' mulSupport g := rfl @[to_additive support_prod_mk] theorem mulSupport_prod_mk (f : α → M) (g : α → N) : (mulSupport fun x => (f x, g x)) = mulSupport f ∪ mulSupport g := Set.ext fun x => by simp only [mulSupport, not_and_or, mem_union, mem_setOf_eq, Prod.mk_eq_one, Ne] @[to_additive support_prod_mk'] theorem mulSupport_prod_mk' (f : α → M × N) : mulSupport f = (mulSupport fun x => (f x).1) ∪ mulSupport fun x => (f x).2 := by simp only [← mulSupport_prod_mk] @[to_additive] theorem mulSupport_along_fiber_subset (f : α × β → M) (a : α) : (mulSupport fun b => f (a, b)) ⊆ (mulSupport f).image Prod.snd := fun x hx => ⟨(a, x), by simpa using hx⟩ @[to_additive] theorem mulSupport_curry (f : α × β → M) : (mulSupport f.curry) = (mulSupport f).image Prod.fst := by simp [mulSupport, funext_iff, image] @[to_additive] theorem mulSupport_curry' (f : α × β → M) : (mulSupport fun a b ↦ f (a, b)) = (mulSupport f).image Prod.fst := mulSupport_curry f end One @[to_additive] theorem mulSupport_mul [MulOneClass M] (f g : α → M) : (mulSupport fun x => f x * g x) ⊆ mulSupport f ∪ mulSupport g := mulSupport_binop_subset (· * ·) (one_mul _) f g @[to_additive] theorem mulSupport_pow [Monoid M] (f : α → M) (n : ℕ) : (mulSupport fun x => f x ^ n) ⊆ mulSupport f := by induction' n with n hfn · simp [pow_zero, mulSupport_one] · simpa only [pow_succ'] using (mulSupport_mul f _).trans (union_subset Subset.rfl hfn) section DivisionMonoid variable [DivisionMonoid G] (f g : α → G) @[to_additive (attr := simp)] theorem mulSupport_inv : (mulSupport fun x => (f x)⁻¹) = mulSupport f := ext fun _ => inv_ne_one @[to_additive (attr := simp)] theorem mulSupport_inv' : mulSupport f⁻¹ = mulSupport f := mulSupport_inv f @[to_additive] theorem mulSupport_mul_inv : (mulSupport fun x => f x * (g x)⁻¹) ⊆ mulSupport f ∪ mulSupport g := mulSupport_binop_subset (fun a b => a * b⁻¹) (by simp) f g @[to_additive] theorem mulSupport_div : (mulSupport fun x => f x / g x) ⊆ mulSupport f ∪ mulSupport g := mulSupport_binop_subset (· / ·) one_div_one f g end DivisionMonoid end Function namespace Set open Function variable {α β M : Type*} [One M] {f : α → M} @[to_additive] theorem image_inter_mulSupport_eq {s : Set β} {g : β → α} : g '' s ∩ mulSupport f = g '' (s ∩ mulSupport (f ∘ g)) := by rw [mulSupport_comp_eq_preimage f g, image_inter_preimage] end Set namespace Pi variable {A : Type*} {B : Type*} [DecidableEq A] [One B] {a : A} {b : B} open Function @[to_additive] theorem mulSupport_mulSingle_subset : mulSupport (mulSingle a b) ⊆ {a} := fun _ hx => by_contra fun hx' => hx <| mulSingle_eq_of_ne hx' _ @[to_additive] theorem mulSupport_mulSingle_one : mulSupport (mulSingle a (1 : B)) = ∅ := by simp @[to_additive (attr := simp)] theorem mulSupport_mulSingle_of_ne (h : b ≠ 1) : mulSupport (mulSingle a b) = {a} := mulSupport_mulSingle_subset.antisymm fun x (hx : x = a) => by rwa [mem_mulSupport, hx, mulSingle_eq_same] @[to_additive] theorem mulSupport_mulSingle [DecidableEq B] : mulSupport (mulSingle a b) = if b = 1 then ∅ else {a} := by split_ifs with h <;> simp [h] @[to_additive] theorem mulSupport_mulSingle_disjoint {b' : B} (hb : b ≠ 1) (hb' : b' ≠ 1) {i j : A} : Disjoint (mulSupport (mulSingle i b)) (mulSupport (mulSingle j b')) ↔ i ≠ j := by rw [mulSupport_mulSingle_of_ne hb, mulSupport_mulSingle_of_ne hb', disjoint_singleton] end Pi
Algebra\Group\TypeTags.lean
/- Copyright (c) 2018 Mario Carneiro. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Mario Carneiro -/ import Mathlib.Algebra.Group.Hom.Defs import Mathlib.Data.Finite.Defs import Mathlib.Logic.Nontrivial.Basic /-! # Type tags that turn additive structures into multiplicative, and vice versa We define two type tags: * `Additive α`: turns any multiplicative structure on `α` into the corresponding additive structure on `Additive α`; * `Multiplicative α`: turns any additive structure on `α` into the corresponding multiplicative structure on `Multiplicative α`. We also define instances `Additive.*` and `Multiplicative.*` that actually transfer the structures. ## See also This file is similar to `Order.Synonym`. ## Porting notes - Since bundled morphism applications that rely on `CoeFun` currently don't work, they are ported as `toFoo a` rather than `a.toFoo` for now. (https://github.com/leanprover/lean4/issues/1910) -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered universe u v variable {α : Type u} {β : Type v} /-- If `α` carries some multiplicative structure, then `Additive α` carries the corresponding additive structure. -/ def Additive (α : Type*) := α /-- If `α` carries some additive structure, then `Multiplicative α` carries the corresponding multiplicative structure. -/ def Multiplicative (α : Type*) := α namespace Additive /-- Reinterpret `x : α` as an element of `Additive α`. -/ def ofMul : α ≃ Additive α := ⟨fun x => x, fun x => x, fun _ => rfl, fun _ => rfl⟩ /-- Reinterpret `x : Additive α` as an element of `α`. -/ def toMul : Additive α ≃ α := ofMul.symm @[simp] theorem ofMul_symm_eq : (@ofMul α).symm = toMul := rfl @[simp] theorem toMul_symm_eq : (@toMul α).symm = ofMul := rfl @[simp] protected lemma «forall» {p : Additive α → Prop} : (∀ a, p a) ↔ ∀ a, p (ofMul a) := Iff.rfl @[simp] protected lemma «exists» {p : Additive α → Prop} : (∃ a, p a) ↔ ∃ a, p (ofMul a) := Iff.rfl /-- Recursion principle for `Additive`, supported by `cases` and `induction`. -/ @[elab_as_elim, cases_eliminator, induction_eliminator] def rec {motive : Additive α → Sort*} (ofMul : ∀ a, motive (ofMul a)) : ∀ a, motive a := fun a => ofMul (toMul a) end Additive namespace Multiplicative /-- Reinterpret `x : α` as an element of `Multiplicative α`. -/ def ofAdd : α ≃ Multiplicative α := ⟨fun x => x, fun x => x, fun _ => rfl, fun _ => rfl⟩ /-- Reinterpret `x : Multiplicative α` as an element of `α`. -/ def toAdd : Multiplicative α ≃ α := ofAdd.symm @[simp] theorem ofAdd_symm_eq : (@ofAdd α).symm = toAdd := rfl @[simp] theorem toAdd_symm_eq : (@toAdd α).symm = ofAdd := rfl @[simp] protected lemma «forall» {p : Multiplicative α → Prop} : (∀ a, p a) ↔ ∀ a, p (ofAdd a) := Iff.rfl @[simp] protected lemma «exists» {p : Multiplicative α → Prop} : (∃ a, p a) ↔ ∃ a, p (ofAdd a) := Iff.rfl /-- Recursion principle for `Multiplicative`, supported by `cases` and `induction`. -/ @[elab_as_elim, cases_eliminator, induction_eliminator] def rec {motive : Multiplicative α → Sort*} (ofAdd : ∀ a, motive (ofAdd a)) : ∀ a, motive a := fun a => ofAdd (toAdd a) end Multiplicative open Additive (ofMul toMul) open Multiplicative (ofAdd toAdd) @[simp] theorem toAdd_ofAdd (x : α) : toAdd (ofAdd x) = x := rfl @[simp] theorem ofAdd_toAdd (x : Multiplicative α) : ofAdd (toAdd x) = x := rfl @[simp] theorem toMul_ofMul (x : α) : toMul (ofMul x) = x := rfl @[simp] theorem ofMul_toMul (x : Additive α) : ofMul (toMul x) = x := rfl instance [Subsingleton α] : Subsingleton (Additive α) := toMul.injective.subsingleton instance [Subsingleton α] : Subsingleton (Multiplicative α) := toAdd.injective.subsingleton instance [Inhabited α] : Inhabited (Additive α) := ⟨ofMul default⟩ instance [Inhabited α] : Inhabited (Multiplicative α) := ⟨ofAdd default⟩ instance [Unique α] : Unique (Additive α) := toMul.unique instance [Unique α] : Unique (Multiplicative α) := toAdd.unique instance [Finite α] : Finite (Additive α) := Finite.of_equiv α (by rfl) instance [Finite α] : Finite (Multiplicative α) := Finite.of_equiv α (by rfl) instance [h : Infinite α] : Infinite (Additive α) := h instance [h : Infinite α] : Infinite (Multiplicative α) := h instance [h : DecidableEq α] : DecidableEq (Multiplicative α) := h instance [h : DecidableEq α] : DecidableEq (Additive α) := h instance Additive.instNontrivial [Nontrivial α] : Nontrivial (Additive α) := ofMul.injective.nontrivial instance Multiplicative.instNontrivial [Nontrivial α] : Nontrivial (Multiplicative α) := ofAdd.injective.nontrivial instance Additive.add [Mul α] : Add (Additive α) where add x y := ofMul (toMul x * toMul y) instance Multiplicative.mul [Add α] : Mul (Multiplicative α) where mul x y := ofAdd (toAdd x + toAdd y) @[simp] theorem ofAdd_add [Add α] (x y : α) : ofAdd (x + y) = ofAdd x * ofAdd y := rfl @[simp] theorem toAdd_mul [Add α] (x y : Multiplicative α) : toAdd (x * y) = toAdd x + toAdd y := rfl @[simp] theorem ofMul_mul [Mul α] (x y : α) : ofMul (x * y) = ofMul x + ofMul y := rfl @[simp] theorem toMul_add [Mul α] (x y : Additive α) : toMul (x + y) = toMul x * toMul y := rfl instance Additive.addSemigroup [Semigroup α] : AddSemigroup (Additive α) := { Additive.add with add_assoc := @mul_assoc α _ } instance Multiplicative.semigroup [AddSemigroup α] : Semigroup (Multiplicative α) := { Multiplicative.mul with mul_assoc := @add_assoc α _ } instance Additive.addCommSemigroup [CommSemigroup α] : AddCommSemigroup (Additive α) := { Additive.addSemigroup with add_comm := @mul_comm α _ } instance Multiplicative.commSemigroup [AddCommSemigroup α] : CommSemigroup (Multiplicative α) := { Multiplicative.semigroup with mul_comm := @add_comm α _ } instance Additive.isLeftCancelAdd [Mul α] [IsLeftCancelMul α] : IsLeftCancelAdd (Additive α) := ⟨@mul_left_cancel α _ _⟩ instance Multiplicative.isLeftCancelMul [Add α] [IsLeftCancelAdd α] : IsLeftCancelMul (Multiplicative α) := ⟨@add_left_cancel α _ _⟩ instance Additive.isRightCancelAdd [Mul α] [IsRightCancelMul α] : IsRightCancelAdd (Additive α) := ⟨@mul_right_cancel α _ _⟩ instance Multiplicative.isRightCancelMul [Add α] [IsRightCancelAdd α] : IsRightCancelMul (Multiplicative α) := ⟨@add_right_cancel α _ _⟩ instance Additive.isCancelAdd [Mul α] [IsCancelMul α] : IsCancelAdd (Additive α) := ⟨⟩ instance Multiplicative.isCancelMul [Add α] [IsCancelAdd α] : IsCancelMul (Multiplicative α) := ⟨⟩ instance Additive.addLeftCancelSemigroup [LeftCancelSemigroup α] : AddLeftCancelSemigroup (Additive α) := { Additive.addSemigroup, Additive.isLeftCancelAdd with } instance Multiplicative.leftCancelSemigroup [AddLeftCancelSemigroup α] : LeftCancelSemigroup (Multiplicative α) := { Multiplicative.semigroup, Multiplicative.isLeftCancelMul with } instance Additive.addRightCancelSemigroup [RightCancelSemigroup α] : AddRightCancelSemigroup (Additive α) := { Additive.addSemigroup, Additive.isRightCancelAdd with } instance Multiplicative.rightCancelSemigroup [AddRightCancelSemigroup α] : RightCancelSemigroup (Multiplicative α) := { Multiplicative.semigroup, Multiplicative.isRightCancelMul with } instance [One α] : Zero (Additive α) := ⟨Additive.ofMul 1⟩ @[simp] theorem ofMul_one [One α] : @Additive.ofMul α 1 = 0 := rfl @[simp] theorem ofMul_eq_zero {A : Type*} [One A] {x : A} : Additive.ofMul x = 0 ↔ x = 1 := Iff.rfl @[simp] theorem toMul_zero [One α] : toMul (0 : Additive α) = 1 := rfl @[simp] lemma toMul_eq_one {α : Type*} [One α] {x : Additive α} : Additive.toMul x = 1 ↔ x = 0 := Iff.rfl instance [Zero α] : One (Multiplicative α) := ⟨Multiplicative.ofAdd 0⟩ @[simp] theorem ofAdd_zero [Zero α] : @Multiplicative.ofAdd α 0 = 1 := rfl @[simp] theorem ofAdd_eq_one {A : Type*} [Zero A] {x : A} : Multiplicative.ofAdd x = 1 ↔ x = 0 := Iff.rfl @[simp] theorem toAdd_one [Zero α] : toAdd (1 : Multiplicative α) = 0 := rfl @[simp] lemma toAdd_eq_zero {α : Type*} [Zero α] {x : Multiplicative α} : Multiplicative.toAdd x = 0 ↔ x = 1 := Iff.rfl instance Additive.addZeroClass [MulOneClass α] : AddZeroClass (Additive α) where zero := 0 add := (· + ·) zero_add := @one_mul α _ add_zero := @mul_one α _ instance Multiplicative.mulOneClass [AddZeroClass α] : MulOneClass (Multiplicative α) where one := 1 mul := (· * ·) one_mul := @zero_add α _ mul_one := @add_zero α _ instance Additive.addMonoid [h : Monoid α] : AddMonoid (Additive α) := { Additive.addZeroClass, Additive.addSemigroup with nsmul := @Monoid.npow α h nsmul_zero := @Monoid.npow_zero α h nsmul_succ := @Monoid.npow_succ α h } instance Multiplicative.monoid [h : AddMonoid α] : Monoid (Multiplicative α) := { Multiplicative.mulOneClass, Multiplicative.semigroup with npow := @AddMonoid.nsmul α h npow_zero := @AddMonoid.nsmul_zero α h npow_succ := @AddMonoid.nsmul_succ α h } @[simp] theorem ofMul_pow [Monoid α] (n : ℕ) (a : α) : ofMul (a ^ n) = n • ofMul a := rfl @[simp] theorem toMul_nsmul [Monoid α] (n : ℕ) (a : Additive α) : toMul (n • a) = toMul a ^ n := rfl @[simp] theorem ofAdd_nsmul [AddMonoid α] (n : ℕ) (a : α) : ofAdd (n • a) = ofAdd a ^ n := rfl @[simp] theorem toAdd_pow [AddMonoid α] (a : Multiplicative α) (n : ℕ) : toAdd (a ^ n) = n • toAdd a := rfl instance Additive.addLeftCancelMonoid [LeftCancelMonoid α] : AddLeftCancelMonoid (Additive α) := { Additive.addMonoid, Additive.addLeftCancelSemigroup with } instance Multiplicative.leftCancelMonoid [AddLeftCancelMonoid α] : LeftCancelMonoid (Multiplicative α) := { Multiplicative.monoid, Multiplicative.leftCancelSemigroup with } instance Additive.addRightCancelMonoid [RightCancelMonoid α] : AddRightCancelMonoid (Additive α) := { Additive.addMonoid, Additive.addRightCancelSemigroup with } instance Multiplicative.rightCancelMonoid [AddRightCancelMonoid α] : RightCancelMonoid (Multiplicative α) := { Multiplicative.monoid, Multiplicative.rightCancelSemigroup with } instance Additive.addCommMonoid [CommMonoid α] : AddCommMonoid (Additive α) := { Additive.addMonoid, Additive.addCommSemigroup with } instance Multiplicative.commMonoid [AddCommMonoid α] : CommMonoid (Multiplicative α) := { Multiplicative.monoid, Multiplicative.commSemigroup with } instance Additive.neg [Inv α] : Neg (Additive α) := ⟨fun x => ofAdd (toMul x)⁻¹⟩ @[simp] theorem ofMul_inv [Inv α] (x : α) : ofMul x⁻¹ = -ofMul x := rfl @[simp] theorem toMul_neg [Inv α] (x : Additive α) : toMul (-x) = (toMul x)⁻¹ := rfl instance Multiplicative.inv [Neg α] : Inv (Multiplicative α) := ⟨fun x => ofMul (-toAdd x)⟩ @[simp] theorem ofAdd_neg [Neg α] (x : α) : ofAdd (-x) = (ofAdd x)⁻¹ := rfl @[simp] theorem toAdd_inv [Neg α] (x : Multiplicative α) : toAdd x⁻¹ = -(toAdd x) := rfl instance Additive.sub [Div α] : Sub (Additive α) where sub x y := ofMul (toMul x / toMul y) instance Multiplicative.div [Sub α] : Div (Multiplicative α) where div x y := ofAdd (toAdd x - toAdd y) @[simp] theorem ofAdd_sub [Sub α] (x y : α) : ofAdd (x - y) = ofAdd x / ofAdd y := rfl @[simp] theorem toAdd_div [Sub α] (x y : Multiplicative α) : toAdd (x / y) = toAdd x - toAdd y := rfl @[simp] theorem ofMul_div [Div α] (x y : α) : ofMul (x / y) = ofMul x - ofMul y := rfl @[simp] theorem toMul_sub [Div α] (x y : Additive α) : toMul (x - y) = toMul x / toMul y := rfl instance Additive.involutiveNeg [InvolutiveInv α] : InvolutiveNeg (Additive α) := { Additive.neg with neg_neg := @inv_inv α _ } instance Multiplicative.involutiveInv [InvolutiveNeg α] : InvolutiveInv (Multiplicative α) := { Multiplicative.inv with inv_inv := @neg_neg α _ } instance Additive.subNegMonoid [DivInvMonoid α] : SubNegMonoid (Additive α) := { Additive.neg, Additive.sub, Additive.addMonoid with sub_eq_add_neg := @div_eq_mul_inv α _ zsmul := @DivInvMonoid.zpow α _ zsmul_zero' := @DivInvMonoid.zpow_zero' α _ zsmul_succ' := @DivInvMonoid.zpow_succ' α _ zsmul_neg' := @DivInvMonoid.zpow_neg' α _ } instance Multiplicative.divInvMonoid [SubNegMonoid α] : DivInvMonoid (Multiplicative α) := { Multiplicative.inv, Multiplicative.div, Multiplicative.monoid with div_eq_mul_inv := @sub_eq_add_neg α _ zpow := @SubNegMonoid.zsmul α _ zpow_zero' := @SubNegMonoid.zsmul_zero' α _ zpow_succ' := @SubNegMonoid.zsmul_succ' α _ zpow_neg' := @SubNegMonoid.zsmul_neg' α _ } @[simp] theorem ofMul_zpow [DivInvMonoid α] (z : ℤ) (a : α) : ofMul (a ^ z) = z • ofMul a := rfl @[simp] theorem toMul_zsmul [DivInvMonoid α] (z : ℤ) (a : Additive α) : toMul (z • a) = toMul a ^ z := rfl @[simp] theorem ofAdd_zsmul [SubNegMonoid α] (z : ℤ) (a : α) : ofAdd (z • a) = ofAdd a ^ z := rfl @[simp] theorem toAdd_zpow [SubNegMonoid α] (a : Multiplicative α) (z : ℤ) : toAdd (a ^ z) = z • toAdd a := rfl instance Additive.subtractionMonoid [DivisionMonoid α] : SubtractionMonoid (Additive α) := { Additive.subNegMonoid, Additive.involutiveNeg with neg_add_rev := @mul_inv_rev α _ neg_eq_of_add := @inv_eq_of_mul_eq_one_right α _ } instance Multiplicative.divisionMonoid [SubtractionMonoid α] : DivisionMonoid (Multiplicative α) := { Multiplicative.divInvMonoid, Multiplicative.involutiveInv with mul_inv_rev := @neg_add_rev α _ inv_eq_of_mul := @neg_eq_of_add_eq_zero_right α _ } instance Additive.subtractionCommMonoid [DivisionCommMonoid α] : SubtractionCommMonoid (Additive α) := { Additive.subtractionMonoid, Additive.addCommSemigroup with } instance Multiplicative.divisionCommMonoid [SubtractionCommMonoid α] : DivisionCommMonoid (Multiplicative α) := { Multiplicative.divisionMonoid, Multiplicative.commSemigroup with } instance Additive.addGroup [Group α] : AddGroup (Additive α) := { Additive.subNegMonoid with add_left_neg := @mul_left_inv α _ } instance Multiplicative.group [AddGroup α] : Group (Multiplicative α) := { Multiplicative.divInvMonoid with mul_left_inv := @add_left_neg α _ } instance Additive.addCommGroup [CommGroup α] : AddCommGroup (Additive α) := { Additive.addGroup, Additive.addCommMonoid with } instance Multiplicative.commGroup [AddCommGroup α] : CommGroup (Multiplicative α) := { Multiplicative.group, Multiplicative.commMonoid with } /-- Reinterpret `α →+ β` as `Multiplicative α →* Multiplicative β`. -/ @[simps] def AddMonoidHom.toMultiplicative [AddZeroClass α] [AddZeroClass β] : (α →+ β) ≃ (Multiplicative α →* Multiplicative β) where toFun f := { toFun := fun a => ofAdd (f (toAdd a)) map_mul' := f.map_add map_one' := f.map_zero } invFun f := { toFun := fun a => toAdd (f (ofAdd a)) map_add' := f.map_mul map_zero' := f.map_one } left_inv _ := rfl right_inv _ := rfl @[simp, norm_cast] lemma AddMonoidHom.coe_toMultiplicative [AddZeroClass α] [AddZeroClass β] (f : α →+ β) : ⇑(toMultiplicative f) = ofAdd ∘ f ∘ toAdd := rfl /-- Reinterpret `α →* β` as `Additive α →+ Additive β`. -/ @[simps] def MonoidHom.toAdditive [MulOneClass α] [MulOneClass β] : (α →* β) ≃ (Additive α →+ Additive β) where toFun f := { toFun := fun a => ofMul (f (toMul a)) map_add' := f.map_mul map_zero' := f.map_one } invFun f := { toFun := fun a => toMul (f (ofMul a)) map_mul' := f.map_add map_one' := f.map_zero } left_inv _ := rfl right_inv _ := rfl @[simp, norm_cast] lemma MonoidHom.coe_toMultiplicative [MulOneClass α] [MulOneClass β] (f : α →* β) : ⇑(toAdditive f) = ofMul ∘ f ∘ toMul := rfl /-- Reinterpret `Additive α →+ β` as `α →* Multiplicative β`. -/ @[simps] def AddMonoidHom.toMultiplicative' [MulOneClass α] [AddZeroClass β] : (Additive α →+ β) ≃ (α →* Multiplicative β) where toFun f := { toFun := fun a => ofAdd (f (ofMul a)) map_mul' := f.map_add map_one' := f.map_zero } invFun f := { toFun := fun a => toAdd (f (toMul a)) map_add' := f.map_mul map_zero' := f.map_one } left_inv _ := rfl right_inv _ := rfl @[simp, norm_cast] lemma AddMonoidHom.coe_toMultiplicative' [MulOneClass α] [AddZeroClass β] (f : Additive α →+ β) : ⇑(toMultiplicative' f) = ofAdd ∘ f ∘ ofMul := rfl /-- Reinterpret `α →* Multiplicative β` as `Additive α →+ β`. -/ @[simps!] def MonoidHom.toAdditive' [MulOneClass α] [AddZeroClass β] : (α →* Multiplicative β) ≃ (Additive α →+ β) := AddMonoidHom.toMultiplicative'.symm @[simp, norm_cast] lemma MonoidHom.coe_toAdditive' [MulOneClass α] [AddZeroClass β] (f : α →* Multiplicative β) : ⇑(toAdditive' f) = toAdd ∘ f ∘ toMul := rfl /-- Reinterpret `α →+ Additive β` as `Multiplicative α →* β`. -/ @[simps] def AddMonoidHom.toMultiplicative'' [AddZeroClass α] [MulOneClass β] : (α →+ Additive β) ≃ (Multiplicative α →* β) where toFun f := { toFun := fun a => toMul (f (toAdd a)) map_mul' := f.map_add map_one' := f.map_zero } invFun f := { toFun := fun a => ofMul (f (ofAdd a)) map_add' := f.map_mul map_zero' := f.map_one } left_inv _ := rfl right_inv _ := rfl @[simp, norm_cast] lemma AddMonoidHom.coe_toMultiplicative'' [AddZeroClass α] [MulOneClass β] (f : α →+ Additive β) : ⇑(toMultiplicative'' f) = toMul ∘ f ∘ toAdd := rfl /-- Reinterpret `Multiplicative α →* β` as `α →+ Additive β`. -/ @[simps!] def MonoidHom.toAdditive'' [AddZeroClass α] [MulOneClass β] : (Multiplicative α →* β) ≃ (α →+ Additive β) := AddMonoidHom.toMultiplicative''.symm @[simp, norm_cast] lemma MonoidHom.coe_toAdditive'' [AddZeroClass α] [MulOneClass β] (f : Multiplicative α →* β) : ⇑(toAdditive'' f) = ofMul ∘ f ∘ ofAdd := rfl /-- If `α` has some multiplicative structure and coerces to a function, then `Additive α` should also coerce to the same function. This allows `Additive` to be used on bundled function types with a multiplicative structure, which is often used for composition, without affecting the behavior of the function itself. -/ instance Additive.coeToFun {α : Type*} {β : α → Sort*} [CoeFun α β] : CoeFun (Additive α) fun a => β (toMul a) := ⟨fun a => CoeFun.coe (toMul a)⟩ /-- If `α` has some additive structure and coerces to a function, then `Multiplicative α` should also coerce to the same function. This allows `Multiplicative` to be used on bundled function types with an additive structure, which is often used for composition, without affecting the behavior of the function itself. -/ instance Multiplicative.coeToFun {α : Type*} {β : α → Sort*} [CoeFun α β] : CoeFun (Multiplicative α) fun a => β (toAdd a) := ⟨fun a => CoeFun.coe (toAdd a)⟩
Algebra\Group\ULift.lean
/- Copyright (c) 2020 Scott Morrison. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Scott Morrison -/ import Mathlib.Algebra.Group.Equiv.Basic import Mathlib.Algebra.Group.InjSurj import Mathlib.Logic.Nontrivial.Basic /-! # `ULift` instances for groups and monoids This file defines instances for group, monoid, semigroup and related structures on `ULift` types. (Recall `ULift α` is just a "copy" of a type `α` in a higher universe.) We also provide `MulEquiv.ulift : ULift R ≃* R` (and its additive analogue). -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered universe u v variable {α : Type u} {β : Type*} {x y : ULift.{v} α} namespace ULift @[to_additive] instance one [One α] : One (ULift α) := ⟨⟨1⟩⟩ @[to_additive (attr := simp)] theorem one_down [One α] : (1 : ULift α).down = 1 := rfl @[to_additive] instance mul [Mul α] : Mul (ULift α) := ⟨fun f g => ⟨f.down * g.down⟩⟩ @[to_additive (attr := simp)] theorem mul_down [Mul α] : (x * y).down = x.down * y.down := rfl @[to_additive] instance div [Div α] : Div (ULift α) := ⟨fun f g => ⟨f.down / g.down⟩⟩ @[to_additive (attr := simp)] theorem div_down [Div α] : (x / y).down = x.down / y.down := rfl @[to_additive] instance inv [Inv α] : Inv (ULift α) := ⟨fun f => ⟨f.down⁻¹⟩⟩ @[to_additive (attr := simp)] theorem inv_down [Inv α] : x⁻¹.down = x.down⁻¹ := rfl @[to_additive] instance smul [SMul α β] : SMul α (ULift β) := ⟨fun n x => up (n • x.down)⟩ @[to_additive (attr := simp)] theorem smul_down [SMul α β] (a : α) (b : ULift.{v} β) : (a • b).down = a • b.down := rfl @[to_additive existing (reorder := 1 2) smul] instance pow [Pow α β] : Pow (ULift α) β := ⟨fun x n => up (x.down ^ n)⟩ @[to_additive existing (attr := simp) (reorder := 1 2) smul_down] theorem pow_down [Pow α β] (a : ULift.{v} α) (b : β) : (a ^ b).down = a.down ^ b := rfl /-- The multiplicative equivalence between `ULift α` and `α`. -/ @[to_additive "The additive equivalence between `ULift α` and `α`."] def _root_.MulEquiv.ulift [Mul α] : ULift α ≃* α := { Equiv.ulift with map_mul' := fun _ _ => rfl } -- Porting note: below failed due to error above, manually added --@[to_additive] instance semigroup [Semigroup α] : Semigroup (ULift α) := (MulEquiv.ulift.injective.semigroup _) fun _ _ => rfl instance addSemigroup [AddSemigroup α] : AddSemigroup (ULift α) := (Equiv.ulift.injective.addSemigroup _) fun _ _ => rfl @[to_additive] instance commSemigroup [CommSemigroup α] : CommSemigroup (ULift α) := (Equiv.ulift.injective.commSemigroup _) fun _ _ => rfl @[to_additive] instance mulOneClass [MulOneClass α] : MulOneClass (ULift α) := Equiv.ulift.injective.mulOneClass _ rfl (by intros; rfl) @[to_additive] instance monoid [Monoid α] : Monoid (ULift α) := Equiv.ulift.injective.monoid _ rfl (fun _ _ => rfl) fun _ _ => rfl @[to_additive] instance commMonoid [CommMonoid α] : CommMonoid (ULift α) := Equiv.ulift.injective.commMonoid _ rfl (fun _ _ => rfl) fun _ _ => rfl instance instNatCast [NatCast α] : NatCast (ULift α) := ⟨(up ·)⟩ instance instIntCast [IntCast α] : IntCast (ULift α) := ⟨(up ·)⟩ @[simp, norm_cast] theorem up_natCast [NatCast α] (n : ℕ) : up (n : α) = n := rfl -- See note [no_index around OfNat.ofNat] @[simp] theorem up_ofNat [NatCast α] (n : ℕ) [n.AtLeastTwo] : up (no_index (OfNat.ofNat n : α)) = OfNat.ofNat n := rfl @[simp, norm_cast] theorem up_intCast [IntCast α] (n : ℤ) : up (n : α) = n := rfl @[simp, norm_cast] theorem down_natCast [NatCast α] (n : ℕ) : down (n : ULift α) = n := rfl -- See note [no_index around OfNat.ofNat] @[simp] theorem down_ofNat [NatCast α] (n : ℕ) [n.AtLeastTwo] : down (no_index (OfNat.ofNat n : ULift α)) = OfNat.ofNat n := rfl @[simp, norm_cast] theorem down_intCast [IntCast α] (n : ℤ) : down (n : ULift α) = n := rfl instance addMonoidWithOne [AddMonoidWithOne α] : AddMonoidWithOne (ULift α) := { ULift.one, ULift.addMonoid with natCast := (⟨·⟩) natCast_zero := congr_arg ULift.up Nat.cast_zero, natCast_succ := fun _ => congr_arg ULift.up (Nat.cast_succ _) } instance addCommMonoidWithOne [AddCommMonoidWithOne α] : AddCommMonoidWithOne (ULift α) := { ULift.addMonoidWithOne, ULift.addCommMonoid with } @[to_additive] instance divInvMonoid [DivInvMonoid α] : DivInvMonoid (ULift α) := Equiv.ulift.injective.divInvMonoid _ rfl (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) fun _ _ => rfl @[to_additive] instance group [Group α] : Group (ULift α) := Equiv.ulift.injective.group _ rfl (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) fun _ _ => rfl @[to_additive] instance commGroup [CommGroup α] : CommGroup (ULift α) := Equiv.ulift.injective.commGroup _ rfl (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) fun _ _ => rfl instance addGroupWithOne [AddGroupWithOne α] : AddGroupWithOne (ULift α) := { ULift.addMonoidWithOne, ULift.addGroup with intCast := (⟨·⟩), intCast_ofNat := fun _ => congr_arg ULift.up (Int.cast_natCast _), intCast_negSucc := fun _ => congr_arg ULift.up (Int.cast_negSucc _) } instance addCommGroupWithOne [AddCommGroupWithOne α] : AddCommGroupWithOne (ULift α) := { ULift.addGroupWithOne, ULift.addCommGroup with } @[to_additive] instance leftCancelSemigroup [LeftCancelSemigroup α] : LeftCancelSemigroup (ULift α) := Equiv.ulift.injective.leftCancelSemigroup _ fun _ _ => rfl @[to_additive] instance rightCancelSemigroup [RightCancelSemigroup α] : RightCancelSemigroup (ULift α) := Equiv.ulift.injective.rightCancelSemigroup _ fun _ _ => rfl @[to_additive] instance leftCancelMonoid [LeftCancelMonoid α] : LeftCancelMonoid (ULift α) := Equiv.ulift.injective.leftCancelMonoid _ rfl (fun _ _ => rfl) fun _ _ => rfl @[to_additive] instance rightCancelMonoid [RightCancelMonoid α] : RightCancelMonoid (ULift α) := Equiv.ulift.injective.rightCancelMonoid _ rfl (fun _ _ => rfl) fun _ _ => rfl @[to_additive] instance cancelMonoid [CancelMonoid α] : CancelMonoid (ULift α) := Equiv.ulift.injective.cancelMonoid _ rfl (fun _ _ => rfl) fun _ _ => rfl @[to_additive] instance cancelCommMonoid [CancelCommMonoid α] : CancelCommMonoid (ULift α) := Equiv.ulift.injective.cancelCommMonoid _ rfl (fun _ _ => rfl) fun _ _ => rfl instance nontrivial [Nontrivial α] : Nontrivial (ULift α) := Equiv.ulift.symm.injective.nontrivial -- TODO we don't do `OrderedCancelCommMonoid` or `OrderedCommGroup` -- We'd need to add instances for `ULift` in `Order.Basic`. end ULift
Algebra\Group\UniqueProds.lean
/- Copyright (c) 2022 Damiano Testa. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Damiano Testa -/ import Mathlib.Data.DFinsupp.Basic import Mathlib.Data.Finset.Pointwise import Mathlib.LinearAlgebra.Basis.VectorSpace /-! # Unique products and related notions A group `G` has *unique products* if for any two non-empty finite subsets `A, B ⊆ G`, there is an element `g ∈ A * B` that can be written uniquely as a product of an element of `A` and an element of `B`. We call the formalization this property `UniqueProds`. Since the condition requires no property of the group operation, we define it for a Type simply satisfying `Mul`. We also introduce the analogous "additive" companion, `UniqueSums`, and link the two so that `to_additive` converts `UniqueProds` into `UniqueSums`. A common way of *proving* that a group satisfies the `UniqueProds/Sums` property is by assuming the existence of some kind of ordering on the group that is well-behaved with respect to the group operation and showing that minima/maxima are the "unique products/sums". However, the order is just a convenience and is not part of the `UniqueProds/Sums` setup. Here you can see several examples of Types that have `UniqueSums/Prods` (`inferInstance` uses `Covariant.to_uniqueProds_left` and `Covariant.to_uniqueSums_left`). ```lean import Mathlib.Data.Real.Basic import Mathlib.Data.PNat.Basic import Mathlib.Algebra.Group.UniqueProds example : UniqueSums ℕ := inferInstance example : UniqueSums ℕ+ := inferInstance example : UniqueSums ℤ := inferInstance example : UniqueSums ℚ := inferInstance example : UniqueSums ℝ := inferInstance example : UniqueProds ℕ+ := inferInstance ``` ## Use in `(Add)MonoidAlgebra`s `UniqueProds/Sums` allow to decouple certain arguments about `(Add)MonoidAlgebra`s into an argument about the grading type and then a generic statement of the form "look at the coefficient of the 'unique product/sum'". The file `Algebra/MonoidAlgebra/NoZeroDivisors` contains several examples of this use. -/ /-- Let `G` be a Type with multiplication, let `A B : Finset G` be finite subsets and let `a0 b0 : G` be two elements. `UniqueMul A B a0 b0` asserts `a0 * b0` can be written in at most one way as a product of an element of `A` and an element of `B`. -/ @[to_additive "Let `G` be a Type with addition, let `A B : Finset G` be finite subsets and let `a0 b0 : G` be two elements. `UniqueAdd A B a0 b0` asserts `a0 + b0` can be written in at most one way as a sum of an element from `A` and an element from `B`."] def UniqueMul {G} [Mul G] (A B : Finset G) (a0 b0 : G) : Prop := ∀ ⦃a b⦄, a ∈ A → b ∈ B → a * b = a0 * b0 → a = a0 ∧ b = b0 namespace UniqueMul variable {G H : Type*} [Mul G] [Mul H] {A B : Finset G} {a0 b0 : G} @[to_additive (attr := nontriviality, simp)] theorem of_subsingleton [Subsingleton G] : UniqueMul A B a0 b0 := by simp [UniqueMul, eq_iff_true_of_subsingleton] @[to_additive] theorem of_card_le_one (hA : A.Nonempty) (hB : B.Nonempty) (hA1 : A.card ≤ 1) (hB1 : B.card ≤ 1) : ∃ a ∈ A, ∃ b ∈ B, UniqueMul A B a b := by rw [Finset.card_le_one_iff] at hA1 hB1 obtain ⟨a, ha⟩ := hA; obtain ⟨b, hb⟩ := hB exact ⟨a, ha, b, hb, fun _ _ ha' hb' _ ↦ ⟨hA1 ha' ha, hB1 hb' hb⟩⟩ @[to_additive] theorem mt (h : UniqueMul A B a0 b0) : ∀ ⦃a b⦄, a ∈ A → b ∈ B → a ≠ a0 ∨ b ≠ b0 → a * b ≠ a0 * b0 := fun _ _ ha hb k ↦ by contrapose! k exact h ha hb k @[to_additive] theorem subsingleton (h : UniqueMul A B a0 b0) : Subsingleton { ab : G × G // ab.1 ∈ A ∧ ab.2 ∈ B ∧ ab.1 * ab.2 = a0 * b0 } := ⟨fun ⟨⟨_a, _b⟩, ha, hb, ab⟩ ⟨⟨_a', _b'⟩, ha', hb', ab'⟩ ↦ Subtype.ext <| Prod.ext ((h ha hb ab).1.trans (h ha' hb' ab').1.symm) <| (h ha hb ab).2.trans (h ha' hb' ab').2.symm⟩ @[to_additive] theorem set_subsingleton (h : UniqueMul A B a0 b0) : Set.Subsingleton { ab : G × G | ab.1 ∈ A ∧ ab.2 ∈ B ∧ ab.1 * ab.2 = a0 * b0 } := by rintro ⟨x1, y1⟩ (hx : x1 ∈ A ∧ y1 ∈ B ∧ x1 * y1 = a0 * b0) ⟨x2, y2⟩ (hy : x2 ∈ A ∧ y2 ∈ B ∧ x2 * y2 = a0 * b0) rcases h hx.1 hx.2.1 hx.2.2 with ⟨rfl, rfl⟩ rcases h hy.1 hy.2.1 hy.2.2 with ⟨rfl, rfl⟩ rfl -- Porting note: mathport warning: expanding binder collection -- (ab «expr ∈ » [finset.product/multiset.product/set.prod/list.product](A, B)) -/ @[to_additive] theorem iff_existsUnique (aA : a0 ∈ A) (bB : b0 ∈ B) : UniqueMul A B a0 b0 ↔ ∃! ab, ab ∈ A ×ˢ B ∧ ab.1 * ab.2 = a0 * b0 := ⟨fun _ ↦ ⟨(a0, b0), ⟨Finset.mk_mem_product aA bB, rfl⟩, by simpa⟩, fun h ↦ h.elim (by rintro ⟨x1, x2⟩ _ J x y hx hy l rcases Prod.mk.inj_iff.mp (J (a0, b0) ⟨Finset.mk_mem_product aA bB, rfl⟩) with ⟨rfl, rfl⟩ exact Prod.mk.inj_iff.mp (J (x, y) ⟨Finset.mk_mem_product hx hy, l⟩))⟩ open Finset in @[to_additive] theorem iff_card_le_one [DecidableEq G] (ha0 : a0 ∈ A) (hb0 : b0 ∈ B) : UniqueMul A B a0 b0 ↔ ((A ×ˢ B).filter (fun p ↦ p.1 * p.2 = a0 * b0)).card ≤ 1 := by simp_rw [card_le_one_iff, mem_filter, mem_product] refine ⟨fun h p1 p2 ⟨⟨ha1, hb1⟩, he1⟩ ⟨⟨ha2, hb2⟩, he2⟩ ↦ ?_, fun h a b ha hb he ↦ ?_⟩ · have h1 := h ha1 hb1 he1; have h2 := h ha2 hb2 he2 ext · rw [h1.1, h2.1] · rw [h1.2, h2.2] · exact Prod.ext_iff.1 (@h (a, b) (a0, b0) ⟨⟨ha, hb⟩, he⟩ ⟨⟨ha0, hb0⟩, rfl⟩) -- Porting note: mathport warning: expanding binder collection -- (ab «expr ∈ » [finset.product/multiset.product/set.prod/list.product](A, B)) -/ @[to_additive] theorem exists_iff_exists_existsUnique : (∃ a0 b0 : G, a0 ∈ A ∧ b0 ∈ B ∧ UniqueMul A B a0 b0) ↔ ∃ g : G, ∃! ab, ab ∈ A ×ˢ B ∧ ab.1 * ab.2 = g := ⟨fun ⟨a0, b0, hA, hB, h⟩ ↦ ⟨_, (iff_existsUnique hA hB).mp h⟩, fun ⟨g, h⟩ ↦ by have h' := h rcases h' with ⟨⟨a, b⟩, ⟨hab, rfl, -⟩, -⟩ cases' Finset.mem_product.mp hab with ha hb exact ⟨a, b, ha, hb, (iff_existsUnique ha hb).mpr h⟩⟩ /-- `UniqueMul` is preserved by inverse images under injective, multiplicative maps. -/ @[to_additive "`UniqueAdd` is preserved by inverse images under injective, additive maps."] theorem mulHom_preimage (f : G →ₙ* H) (hf : Function.Injective f) (a0 b0 : G) {A B : Finset H} (u : UniqueMul A B (f a0) (f b0)) : UniqueMul (A.preimage f hf.injOn) (B.preimage f hf.injOn) a0 b0 := by intro a b ha hb ab simp only [← hf.eq_iff, map_mul] at ab ⊢ exact u (Finset.mem_preimage.mp ha) (Finset.mem_preimage.mp hb) ab @[to_additive] theorem of_mulHom_image [DecidableEq H] (f : G →ₙ* H) (hf : ∀ ⦃a b c d : G⦄, a * b = c * d → f a = f c ∧ f b = f d → a = c ∧ b = d) (h : UniqueMul (A.image f) (B.image f) (f a0) (f b0)) : UniqueMul A B a0 b0 := fun a b ha hb ab ↦ hf ab (h (Finset.mem_image_of_mem f ha) (Finset.mem_image_of_mem f hb) <| by simp_rw [← map_mul, ab]) /-- `Unique_Mul` is preserved under multiplicative maps that are injective. See `UniqueMul.mulHom_map_iff` for a version with swapped bundling. -/ @[to_additive "`UniqueAdd` is preserved under additive maps that are injective. See `UniqueAdd.addHom_map_iff` for a version with swapped bundling."] theorem mulHom_image_iff [DecidableEq H] (f : G →ₙ* H) (hf : Function.Injective f) : UniqueMul (A.image f) (B.image f) (f a0) (f b0) ↔ UniqueMul A B a0 b0 := ⟨of_mulHom_image f fun _ _ _ _ _ ↦ .imp (hf ·) (hf ·), fun h _ _ ↦ by simp_rw [Finset.mem_image] rintro ⟨a, aA, rfl⟩ ⟨b, bB, rfl⟩ ab simp_rw [← map_mul, hf.eq_iff] at ab ⊢ exact h aA bB ab⟩ /-- `UniqueMul` is preserved under embeddings that are multiplicative. See `UniqueMul.mulHom_image_iff` for a version with swapped bundling. -/ @[to_additive "`UniqueAdd` is preserved under embeddings that are additive. See `UniqueAdd.addHom_image_iff` for a version with swapped bundling."] theorem mulHom_map_iff (f : G ↪ H) (mul : ∀ x y, f (x * y) = f x * f y) : UniqueMul (A.map f) (B.map f) (f a0) (f b0) ↔ UniqueMul A B a0 b0 := by classical simp_rw [← mulHom_image_iff ⟨f, mul⟩ f.2, Finset.map_eq_image]; rfl section Opposites open Finset MulOpposite @[to_additive] theorem of_mulOpposite (h : UniqueMul (B.map ⟨_, op_injective⟩) (A.map ⟨_, op_injective⟩) (op b0) (op a0)) : UniqueMul A B a0 b0 := fun a b aA bB ab ↦ by simpa [and_comm] using h (mem_map_of_mem _ bB) (mem_map_of_mem _ aA) (congr_arg op ab) @[to_additive] theorem to_mulOpposite (h : UniqueMul A B a0 b0) : UniqueMul (B.map ⟨_, op_injective⟩) (A.map ⟨_, op_injective⟩) (op b0) (op a0) := of_mulOpposite (by simp_rw [map_map]; exact (mulHom_map_iff _ fun _ _ ↦ by rfl).mpr h) @[to_additive] theorem iff_mulOpposite : UniqueMul (B.map ⟨_, op_injective⟩) (A.map ⟨_, op_injective⟩) (op b0) (op a0) ↔ UniqueMul A B a0 b0 := ⟨of_mulOpposite, to_mulOpposite⟩ end Opposites open Finset in @[to_additive] theorem of_image_filter [DecidableEq H] (f : G →ₙ* H) {A B : Finset G} {aG bG : G} {aH bH : H} (hae : f aG = aH) (hbe : f bG = bH) (huH : UniqueMul (A.image f) (B.image f) aH bH) (huG : UniqueMul (A.filter (f · = aH)) (B.filter (f · = bH)) aG bG) : UniqueMul A B aG bG := fun a b ha hb he ↦ by specialize huH (mem_image_of_mem _ ha) (mem_image_of_mem _ hb) rw [← map_mul, he, map_mul, hae, hbe] at huH refine huG ?_ ?_ he <;> rw [mem_filter] exacts [⟨ha, (huH rfl).1⟩, ⟨hb, (huH rfl).2⟩] end UniqueMul /-- Let `G` be a Type with addition. `UniqueSums G` asserts that any two non-empty finite subsets of `G` have the `UniqueAdd` property, with respect to some element of their sum `A + B`. -/ class UniqueSums (G) [Add G] : Prop where /-- For `A B` two nonempty finite sets, there always exist `a0 ∈ A, b0 ∈ B` such that `UniqueAdd A B a0 b0` -/ uniqueAdd_of_nonempty : ∀ {A B : Finset G}, A.Nonempty → B.Nonempty → ∃ a0 ∈ A, ∃ b0 ∈ B, UniqueAdd A B a0 b0 /-- Let `G` be a Type with multiplication. `UniqueProds G` asserts that any two non-empty finite subsets of `G` have the `UniqueMul` property, with respect to some element of their product `A * B`. -/ class UniqueProds (G) [Mul G] : Prop where /-- For `A B` two nonempty finite sets, there always exist `a0 ∈ A, b0 ∈ B` such that `UniqueMul A B a0 b0` -/ uniqueMul_of_nonempty : ∀ {A B : Finset G}, A.Nonempty → B.Nonempty → ∃ a0 ∈ A, ∃ b0 ∈ B, UniqueMul A B a0 b0 attribute [to_additive] UniqueProds /-- Let `G` be a Type with addition. `TwoUniqueSums G` asserts that any two non-empty finite subsets of `G`, at least one of which is not a singleton, possesses at least two pairs of elements satisfying the `UniqueAdd` property. -/ class TwoUniqueSums (G) [Add G] : Prop where /-- For `A B` two finite sets whose product has cardinality at least 2, we can find at least two unique pairs. -/ uniqueAdd_of_one_lt_card : ∀ {A B : Finset G}, 1 < A.card * B.card → ∃ p1 ∈ A ×ˢ B, ∃ p2 ∈ A ×ˢ B, p1 ≠ p2 ∧ UniqueAdd A B p1.1 p1.2 ∧ UniqueAdd A B p2.1 p2.2 /-- Let `G` be a Type with multiplication. `TwoUniqueProds G` asserts that any two non-empty finite subsets of `G`, at least one of which is not a singleton, possesses at least two pairs of elements satisfying the `UniqueMul` property. -/ class TwoUniqueProds (G) [Mul G] : Prop where /-- For `A B` two finite sets whose product has cardinality at least 2, we can find at least two unique pairs. -/ uniqueMul_of_one_lt_card : ∀ {A B : Finset G}, 1 < A.card * B.card → ∃ p1 ∈ A ×ˢ B, ∃ p2 ∈ A ×ˢ B, p1 ≠ p2 ∧ UniqueMul A B p1.1 p1.2 ∧ UniqueMul A B p2.1 p2.2 attribute [to_additive] TwoUniqueProds @[to_additive] lemma uniqueMul_of_twoUniqueMul {G} [Mul G] {A B : Finset G} (h : 1 < A.card * B.card → ∃ p1 ∈ A ×ˢ B, ∃ p2 ∈ A ×ˢ B, p1 ≠ p2 ∧ UniqueMul A B p1.1 p1.2 ∧ UniqueMul A B p2.1 p2.2) (hA : A.Nonempty) (hB : B.Nonempty) : ∃ a ∈ A, ∃ b ∈ B, UniqueMul A B a b := by by_cases hc : A.card ≤ 1 ∧ B.card ≤ 1 · exact UniqueMul.of_card_le_one hA hB hc.1 hc.2 simp_rw [not_and_or, not_le] at hc rw [← Finset.card_pos] at hA hB obtain ⟨p, hp, _, _, _, hu, _⟩ := h (Nat.one_lt_mul_iff.mpr ⟨hA, hB, hc⟩) rw [Finset.mem_product] at hp exact ⟨p.1, hp.1, p.2, hp.2, hu⟩ @[to_additive] instance TwoUniqueProds.toUniqueProds (G) [Mul G] [TwoUniqueProds G] : UniqueProds G where uniqueMul_of_nonempty := uniqueMul_of_twoUniqueMul uniqueMul_of_one_lt_card namespace Multiplicative instance {M} [Add M] [UniqueSums M] : UniqueProds (Multiplicative M) where uniqueMul_of_nonempty := UniqueSums.uniqueAdd_of_nonempty (G := M) instance {M} [Add M] [TwoUniqueSums M] : TwoUniqueProds (Multiplicative M) where uniqueMul_of_one_lt_card := TwoUniqueSums.uniqueAdd_of_one_lt_card (G := M) end Multiplicative namespace Additive instance {M} [Mul M] [UniqueProds M] : UniqueSums (Additive M) where uniqueAdd_of_nonempty := UniqueProds.uniqueMul_of_nonempty (G := M) instance {M} [Mul M] [TwoUniqueProds M] : TwoUniqueSums (Additive M) where uniqueAdd_of_one_lt_card := TwoUniqueProds.uniqueMul_of_one_lt_card (G := M) end Additive universe u v variable (G : Type u) (H : Type v) [Mul G] [Mul H] private abbrev I : Bool → Type max u v := Bool.rec (ULift.{v} G) (ULift.{u} H) @[to_additive] private instance : ∀ b, Mul (I G H b) := Bool.rec ULift.mul ULift.mul @[to_additive] private def Prod.upMulHom : G × H →ₙ* ∀ b, I G H b := ⟨fun x ↦ Bool.rec ⟨x.1⟩ ⟨x.2⟩, fun x y ↦ by ext (_|_) <;> rfl⟩ @[to_additive] private def downMulHom : ULift G →ₙ* G := ⟨ULift.down, fun _ _ ↦ rfl⟩ variable {G H} namespace UniqueProds open Finset @[to_additive] theorem of_mulHom (f : H →ₙ* G) (hf : ∀ ⦃a b c d : H⦄, a * b = c * d → f a = f c ∧ f b = f d → a = c ∧ b = d) [UniqueProds G] : UniqueProds H where uniqueMul_of_nonempty {A B} A0 B0 := by classical obtain ⟨a0, ha0, b0, hb0, h⟩ := uniqueMul_of_nonempty (A0.image f) (B0.image f) obtain ⟨a', ha', rfl⟩ := mem_image.mp ha0 obtain ⟨b', hb', rfl⟩ := mem_image.mp hb0 exact ⟨a', ha', b', hb', UniqueMul.of_mulHom_image f hf h⟩ @[to_additive] theorem of_injective_mulHom (f : H →ₙ* G) (hf : Function.Injective f) (_ : UniqueProds G) : UniqueProds H := of_mulHom f (fun _ _ _ _ _ ↦ .imp (hf ·) (hf ·)) /-- `UniqueProd` is preserved under multiplicative equivalences. -/ @[to_additive "`UniqueSums` is preserved under additive equivalences."] theorem _root_.MulEquiv.uniqueProds_iff (f : G ≃* H) : UniqueProds G ↔ UniqueProds H := ⟨of_injective_mulHom f.symm f.symm.injective, of_injective_mulHom f f.injective⟩ open Finset MulOpposite in @[to_additive] theorem of_mulOpposite (h : UniqueProds Gᵐᵒᵖ) : UniqueProds G where uniqueMul_of_nonempty hA hB := let f : G ↪ Gᵐᵒᵖ := ⟨op, op_injective⟩ let ⟨y, yB, x, xA, hxy⟩ := h.uniqueMul_of_nonempty (hB.map (f := f)) (hA.map (f := f)) ⟨unop x, (mem_map' _).mp xA, unop y, (mem_map' _).mp yB, hxy.of_mulOpposite⟩ @[to_additive] instance [h : UniqueProds G] : UniqueProds Gᵐᵒᵖ := of_mulOpposite <| (MulEquiv.opOp G).uniqueProds_iff.mp h @[to_additive] private theorem toIsLeftCancelMul [UniqueProds G] : IsLeftCancelMul G where mul_left_cancel a b1 b2 he := by classical have := mem_insert_self b1 {b2} obtain ⟨a, ha, b, hb, hu⟩ := uniqueMul_of_nonempty ⟨a, mem_singleton_self a⟩ ⟨b1, this⟩ cases mem_singleton.mp ha simp_rw [mem_insert, mem_singleton] at hb obtain rfl | rfl := hb · exact (hu ha (mem_insert_of_mem <| mem_singleton_self b2) he.symm).2.symm · exact (hu ha this he).2 open MulOpposite in @[to_additive] theorem toIsCancelMul [UniqueProds G] : IsCancelMul G where mul_left_cancel := toIsLeftCancelMul.mul_left_cancel mul_right_cancel _ _ _ h := op_injective <| toIsLeftCancelMul.mul_left_cancel _ _ _ <| unop_injective h /-! Two theorems in [Andrzej Strojnowski, *A note on u.p. groups*][Strojnowski1980] -/ /-- `UniqueProds G` says that for any two nonempty `Finset`s `A` and `B` in `G`, `A × B` contains a unique pair with the `UniqueMul` property. Strojnowski showed that if `G` is a group, then we only need to check this when `A = B`. Here we generalize the result to cancellative semigroups. Non-cancellative counterexample: the AddMonoid {0,1} with 1+1=1. -/ @[to_additive] theorem of_same {G} [Semigroup G] [IsCancelMul G] (h : ∀ {A : Finset G}, A.Nonempty → ∃ a1 ∈ A, ∃ a2 ∈ A, UniqueMul A A a1 a2) : UniqueProds G where uniqueMul_of_nonempty {A B} hA hB := by classical obtain ⟨g1, h1, g2, h2, hu⟩ := h (hB.mul hA) obtain ⟨b1, hb1, a1, ha1, rfl⟩ := mem_mul.mp h1 obtain ⟨b2, hb2, a2, ha2, rfl⟩ := mem_mul.mp h2 refine ⟨a1, ha1, b2, hb2, fun a b ha hb he => ?_⟩ specialize hu (mul_mem_mul hb1 ha) (mul_mem_mul hb ha2) _ · rw [mul_assoc b1, ← mul_assoc a, he, mul_assoc a1, ← mul_assoc b1] exact ⟨mul_left_cancel hu.1, mul_right_cancel hu.2⟩ /-- If a group has `UniqueProds`, then it actually has `TwoUniqueProds`. For an example of a semigroup `G` embeddable into a group that has `UniqueProds` but not `TwoUniqueProds`, see Example 10.13 in [J. Okniński, *Semigroup Algebras*][Okninski1991]. -/ @[to_additive] theorem toTwoUniqueProds_of_group {G} [Group G] [UniqueProds G] : TwoUniqueProds G where uniqueMul_of_one_lt_card {A B} hc := by simp_rw [Nat.one_lt_mul_iff, card_pos] at hc obtain ⟨a, ha, b, hb, hu⟩ := uniqueMul_of_nonempty hc.1 hc.2.1 let C := A.map ⟨_, mul_right_injective a⁻¹⟩ -- C = a⁻¹A let D := B.map ⟨_, mul_left_injective b⁻¹⟩ -- D = Bb⁻¹ have hcard : 1 < C.card ∨ 1 < D.card := by simp_rw [C, D, card_map]; exact hc.2.2 have hC : 1 ∈ C := mem_map.mpr ⟨a, ha, inv_mul_self a⟩ have hD : 1 ∈ D := mem_map.mpr ⟨b, hb, mul_inv_self b⟩ suffices ∃ c ∈ C, ∃ d ∈ D, (c ≠ 1 ∨ d ≠ 1) ∧ UniqueMul C D c d by simp_rw [mem_product] obtain ⟨c, hc, d, hd, hne, hu'⟩ := this obtain ⟨a0, ha0, rfl⟩ := mem_map.mp hc obtain ⟨b0, hb0, rfl⟩ := mem_map.mp hd refine ⟨(_, _), ⟨ha0, hb0⟩, (a, b), ⟨ha, hb⟩, ?_, fun a' b' ha' hb' he => ?_, hu⟩ · simp_rw [Function.Embedding.coeFn_mk, Ne, inv_mul_eq_one, mul_inv_eq_one] at hne rwa [Ne, Prod.mk.inj_iff, not_and_or, eq_comm] specialize hu' (mem_map_of_mem _ ha') (mem_map_of_mem _ hb') simp_rw [Function.Embedding.coeFn_mk, mul_left_cancel_iff, mul_right_cancel_iff] at hu' rw [mul_assoc, ← mul_assoc a', he, mul_assoc, mul_assoc] at hu' exact hu' rfl classical let _ := Finset.mul (α := G) -- E = D⁻¹C, F = DC⁻¹ have := uniqueMul_of_nonempty (A := D.image (·⁻¹) * C) (B := D * C.image (·⁻¹)) ?_ ?_ · obtain ⟨e, he, f, hf, hu⟩ := this clear_value C D simp only [UniqueMul, mem_mul, mem_image] at he hf hu obtain ⟨_, ⟨d1, hd1, rfl⟩, c1, hc1, rfl⟩ := he obtain ⟨d2, hd2, _, ⟨c2, hc2, rfl⟩, rfl⟩ := hf by_cases h12 : c1 ≠ 1 ∨ d2 ≠ 1 · refine ⟨c1, hc1, d2, hd2, h12, fun c3 d3 hc3 hd3 he => ?_⟩ specialize hu ⟨_, ⟨_, hd1, rfl⟩, _, hc3, rfl⟩ ⟨_, hd3, _, ⟨_, hc2, rfl⟩, rfl⟩ rw [mul_left_cancel_iff, mul_right_cancel_iff, mul_assoc, ← mul_assoc c3, he, mul_assoc, mul_assoc] at hu; exact hu rfl push_neg at h12; obtain ⟨rfl, rfl⟩ := h12 by_cases h21 : c2 ≠ 1 ∨ d1 ≠ 1 · refine ⟨c2, hc2, d1, hd1, h21, fun c4 d4 hc4 hd4 he => ?_⟩ specialize hu ⟨_, ⟨_, hd4, rfl⟩, _, hC, rfl⟩ ⟨_, hD, _, ⟨_, hc4, rfl⟩, rfl⟩ simpa only [mul_one, one_mul, ← mul_inv_rev, he, true_imp_iff, inv_inj, and_comm] using hu push_neg at h21; obtain ⟨rfl, rfl⟩ := h21 rcases hcard with hC | hD · obtain ⟨c, hc, hc1⟩ := exists_ne_of_one_lt_card hC 1 refine (hc1 ?_).elim simpa using hu ⟨_, ⟨_, hD, rfl⟩, _, hc, rfl⟩ ⟨_, hD, _, ⟨_, hc, rfl⟩, rfl⟩ · obtain ⟨d, hd, hd1⟩ := exists_ne_of_one_lt_card hD 1 refine (hd1 ?_).elim simpa using hu ⟨_, ⟨_, hd, rfl⟩, _, hC, rfl⟩ ⟨_, hd, _, ⟨_, hC, rfl⟩, rfl⟩ all_goals apply_rules [Nonempty.mul, Nonempty.image, Finset.Nonempty.map, hc.1, hc.2.1] open UniqueMul in @[to_additive] instance instForall {ι} (G : ι → Type*) [∀ i, Mul (G i)] [∀ i, UniqueProds (G i)] : UniqueProds (∀ i, G i) where uniqueMul_of_nonempty {A} := by classical let _ := isWellFounded_ssubset (α := ∀ i, G i) -- why need this? apply IsWellFounded.induction (· ⊂ ·) A; intro A ihA B hA apply IsWellFounded.induction (· ⊂ ·) B; intro B ihB hB by_cases hc : A.card ≤ 1 ∧ B.card ≤ 1 · exact of_card_le_one hA hB hc.1 hc.2 simp_rw [not_and_or, not_le] at hc obtain ⟨i, hc⟩ := exists_or.mpr (hc.imp exists_of_one_lt_card_pi exists_of_one_lt_card_pi) obtain ⟨ai, hA, bi, hB, hi⟩ := uniqueMul_of_nonempty (hA.image (· i)) (hB.image (· i)) rw [mem_image, ← filter_nonempty_iff] at hA hB let A' := A.filter (· i = ai); let B' := B.filter (· i = bi) obtain ⟨a0, ha0, b0, hb0, hu⟩ : ∃ a0 ∈ A', ∃ b0 ∈ B', UniqueMul A' B' a0 b0 := by rcases hc with hc | hc; · exact ihA A' (hc.2 ai) hA hB by_cases hA' : A' = A · rw [hA'] exact ihB B' (hc.2 bi) hB · exact ihA A' ((A.filter_subset _).ssubset_of_ne hA') hA hB rw [mem_filter] at ha0 hb0 exact ⟨a0, ha0.1, b0, hb0.1, of_image_filter (Pi.evalMulHom G i) ha0.2 hb0.2 hi hu⟩ open ULift in @[to_additive] instance [UniqueProds G] [UniqueProds H] : UniqueProds (G × H) := by have : ∀ b, UniqueProds (I G H b) := Bool.rec ?_ ?_ · exact of_injective_mulHom (downMulHom H) down_injective ‹_› · refine of_injective_mulHom (Prod.upMulHom G H) (fun x y he => Prod.ext ?_ ?_) (UniqueProds.instForall <| I G H) <;> apply up_injective exacts [congr_fun he false, congr_fun he true] · exact of_injective_mulHom (downMulHom G) down_injective ‹_› end UniqueProds instance {ι} (G : ι → Type*) [∀ i, AddZeroClass (G i)] [∀ i, UniqueSums (G i)] : UniqueSums (Π₀ i, G i) := UniqueSums.of_injective_addHom DFinsupp.coeFnAddMonoidHom.toAddHom DFunLike.coe_injective inferInstance instance {ι G} [AddZeroClass G] [UniqueSums G] : UniqueSums (ι →₀ G) := UniqueSums.of_injective_addHom Finsupp.coeFnAddHom.toAddHom DFunLike.coe_injective inferInstance namespace TwoUniqueProds open Finset @[to_additive] theorem of_mulHom (f : H →ₙ* G) (hf : ∀ ⦃a b c d : H⦄, a * b = c * d → f a = f c ∧ f b = f d → a = c ∧ b = d) [TwoUniqueProds G] : TwoUniqueProds H where uniqueMul_of_one_lt_card {A B} hc := by classical obtain hc' | hc' := lt_or_le 1 ((A.image f).card * (B.image f).card) · obtain ⟨⟨a1, b1⟩, h1, ⟨a2, b2⟩, h2, hne, hu1, hu2⟩ := uniqueMul_of_one_lt_card hc' simp_rw [mem_product, mem_image] at h1 h2 ⊢ obtain ⟨⟨a1, ha1, rfl⟩, b1, hb1, rfl⟩ := h1 obtain ⟨⟨a2, ha2, rfl⟩, b2, hb2, rfl⟩ := h2 exact ⟨(a1, b1), ⟨ha1, hb1⟩, (a2, b2), ⟨ha2, hb2⟩, mt (congr_arg (Prod.map f f)) hne, UniqueMul.of_mulHom_image f hf hu1, UniqueMul.of_mulHom_image f hf hu2⟩ rw [← card_product] at hc hc' obtain ⟨p1, h1, p2, h2, hne⟩ := one_lt_card_iff_nontrivial.mp hc refine ⟨p1, h1, p2, h2, hne, ?_⟩ cases mem_product.mp h1; cases mem_product.mp h2 constructor <;> refine UniqueMul.of_mulHom_image f hf ((UniqueMul.iff_card_le_one ?_ ?_).mpr <| (card_filter_le _ _).trans hc') <;> apply mem_image_of_mem <;> assumption @[to_additive] theorem of_injective_mulHom (f : H →ₙ* G) (hf : Function.Injective f) (_ : TwoUniqueProds G) : TwoUniqueProds H := of_mulHom f (fun _ _ _ _ _ ↦ .imp (hf ·) (hf ·)) /-- `TwoUniqueProd` is preserved under multiplicative equivalences. -/ @[to_additive "`TwoUniqueSums` is preserved under additive equivalences."] theorem _root_.MulEquiv.twoUniqueProds_iff (f : G ≃* H) : TwoUniqueProds G ↔ TwoUniqueProds H := ⟨of_injective_mulHom f.symm f.symm.injective, of_injective_mulHom f f.injective⟩ @[to_additive] instance instForall {ι} (G : ι → Type*) [∀ i, Mul (G i)] [∀ i, TwoUniqueProds (G i)] : TwoUniqueProds (∀ i, G i) where uniqueMul_of_one_lt_card {A} := by classical let _ := isWellFounded_ssubset (α := ∀ i, G i) -- why need this? apply IsWellFounded.induction (· ⊂ ·) A; intro A ihA B apply IsWellFounded.induction (· ⊂ ·) B; intro B ihB hc obtain ⟨hA, hB, hc⟩ := Nat.one_lt_mul_iff.mp hc rw [card_pos] at hA hB obtain ⟨i, hc⟩ := exists_or.mpr (hc.imp exists_of_one_lt_card_pi exists_of_one_lt_card_pi) obtain ⟨p1, h1, p2, h2, hne, hi1, hi2⟩ := uniqueMul_of_one_lt_card (Nat.one_lt_mul_iff.mpr ⟨card_pos.2 (hA.image _), card_pos.2 (hB.image _), hc.imp And.left And.left⟩) simp_rw [mem_product, mem_image, ← filter_nonempty_iff] at h1 h2 replace h1 := uniqueMul_of_twoUniqueMul ?_ h1.1 h1.2 on_goal 1 => replace h2 := uniqueMul_of_twoUniqueMul ?_ h2.1 h2.2 · obtain ⟨a1, ha1, b1, hb1, hu1⟩ := h1 obtain ⟨a2, ha2, b2, hb2, hu2⟩ := h2 rw [mem_filter] at ha1 hb1 ha2 hb2 simp_rw [mem_product] refine ⟨(a1, b1), ⟨ha1.1, hb1.1⟩, (a2, b2), ⟨ha2.1, hb2.1⟩, ?_, UniqueMul.of_image_filter (Pi.evalMulHom G i) ha1.2 hb1.2 hi1 hu1, UniqueMul.of_image_filter (Pi.evalMulHom G i) ha2.2 hb2.2 hi2 hu2⟩ contrapose! hne; rw [Prod.mk.inj_iff] at hne ⊢ rw [← ha1.2, ← hb1.2, ← ha2.2, ← hb2.2, hne.1, hne.2]; exact ⟨rfl, rfl⟩ all_goals rcases hc with hc | hc; · exact ihA _ (hc.2 _) · by_cases hA : A.filter (· i = p2.1) = A · rw [hA] exact ihB _ (hc.2 _) · exact ihA _ ((A.filter_subset _).ssubset_of_ne hA) · by_cases hA : A.filter (· i = p1.1) = A · rw [hA] exact ihB _ (hc.2 _) · exact ihA _ ((A.filter_subset _).ssubset_of_ne hA) open ULift in @[to_additive] instance [TwoUniqueProds G] [TwoUniqueProds H] : TwoUniqueProds (G × H) := by have : ∀ b, TwoUniqueProds (I G H b) := Bool.rec ?_ ?_ · exact of_injective_mulHom (downMulHom H) down_injective ‹_› · refine of_injective_mulHom (Prod.upMulHom G H) (fun x y he ↦ Prod.ext ?_ ?_) (TwoUniqueProds.instForall <| I G H) <;> apply up_injective exacts [congr_fun he false, congr_fun he true] · exact of_injective_mulHom (downMulHom G) down_injective ‹_› open MulOpposite in @[to_additive] theorem of_mulOpposite (h : TwoUniqueProds Gᵐᵒᵖ) : TwoUniqueProds G where uniqueMul_of_one_lt_card hc := by let f : G ↪ Gᵐᵒᵖ := ⟨op, op_injective⟩ rw [← card_map f, ← card_map f, mul_comm] at hc obtain ⟨p1, h1, p2, h2, hne, hu1, hu2⟩ := h.uniqueMul_of_one_lt_card hc simp_rw [mem_product] at h1 h2 ⊢ refine ⟨(_, _), ⟨?_, ?_⟩, (_, _), ⟨?_, ?_⟩, ?_, hu1.of_mulOpposite, hu2.of_mulOpposite⟩ pick_goal 5 · contrapose! hne; rw [Prod.ext_iff] at hne ⊢ exact ⟨unop_injective hne.2, unop_injective hne.1⟩ all_goals apply (mem_map' f).mp exacts [h1.2, h1.1, h2.2, h2.1] @[to_additive] instance [h : TwoUniqueProds G] : TwoUniqueProds Gᵐᵒᵖ := of_mulOpposite <| (MulEquiv.opOp G).twoUniqueProds_iff.mp h -- see Note [lower instance priority] /-- This instance asserts that if `G` has a right-cancellative multiplication, a linear order, and multiplication is strictly monotone w.r.t. the second argument, then `G` has `TwoUniqueProds`. -/ @[to_additive "This instance asserts that if `G` has a right-cancellative addition, a linear order, and addition is strictly monotone w.r.t. the second argument, then `G` has `TwoUniqueSums`." ] instance (priority := 100) of_covariant_right [IsRightCancelMul G] [LinearOrder G] [CovariantClass G G (· * ·) (· < ·)] : TwoUniqueProds G where uniqueMul_of_one_lt_card {A B} hc := by obtain ⟨hA, hB, -⟩ := Nat.one_lt_mul_iff.mp hc rw [card_pos] at hA hB rw [← card_product] at hc obtain ⟨a0, ha0, b0, hb0, he0⟩ := mem_mul.mp (max'_mem _ <| hA.mul hB) obtain ⟨a1, ha1, b1, hb1, he1⟩ := mem_mul.mp (min'_mem _ <| hA.mul hB) have : UniqueMul A B a0 b0 := by intro a b ha hb he obtain hl | rfl | hl := lt_trichotomy b b0 · exact ((he0 ▸ he ▸ mul_lt_mul_left' hl a).not_le <| le_max' _ _ <| mul_mem_mul ha hb0).elim · exact ⟨mul_right_cancel he, rfl⟩ · exact ((he0 ▸ mul_lt_mul_left' hl a0).not_le <| le_max' _ _ <| mul_mem_mul ha0 hb).elim refine ⟨_, mk_mem_product ha0 hb0, _, mk_mem_product ha1 hb1, fun he ↦ ?_, this, ?_⟩ · rw [Prod.mk.inj_iff] at he; rw [he.1, he.2, he1] at he0 obtain ⟨⟨a2, b2⟩, h2, hne⟩ := exists_ne_of_one_lt_card hc (a0, b0) rw [mem_product] at h2 refine (min'_lt_max' _ (mul_mem_mul ha0 hb0) (mul_mem_mul h2.1 h2.2) fun he ↦ hne ?_).ne he0 exact Prod.ext_iff.mpr (this h2.1 h2.2 he.symm) · intro a b ha hb he obtain hl | rfl | hl := lt_trichotomy b b1 · exact ((he1 ▸ mul_lt_mul_left' hl a1).not_le <| min'_le _ _ <| mul_mem_mul ha1 hb).elim · exact ⟨mul_right_cancel he, rfl⟩ · exact ((he1 ▸ he ▸ mul_lt_mul_left' hl a).not_le <| min'_le _ _ <| mul_mem_mul ha hb1).elim open MulOpposite in -- see Note [lower instance priority] /-- This instance asserts that if `G` has a left-cancellative multiplication, a linear order, and multiplication is strictly monotone w.r.t. the first argument, then `G` has `TwoUniqueProds`. -/ @[to_additive "This instance asserts that if `G` has a left-cancellative addition, a linear order, and addition is strictly monotone w.r.t. the first argument, then `G` has `TwoUniqueSums`." ] instance (priority := 100) of_covariant_left [IsLeftCancelMul G] [LinearOrder G] [CovariantClass G G (Function.swap (· * ·)) (· < ·)] : TwoUniqueProds G := let _ := LinearOrder.lift' (unop : Gᵐᵒᵖ → G) unop_injective let _ : CovariantClass Gᵐᵒᵖ Gᵐᵒᵖ (· * ·) (· < ·) := { elim := fun _ _ _ bc ↦ mul_lt_mul_right' (α := G) bc (unop _) } of_mulOpposite of_covariant_right end TwoUniqueProds @[deprecated (since := "2024-02-04")] alias UniqueProds.mulHom_image_of_injective := UniqueProds.of_injective_mulHom @[deprecated (since := "2024-02-04")] alias UniqueSums.addHom_image_of_injective := UniqueSums.of_injective_addHom @[deprecated (since := "2024-02-04")] alias UniqueProds.mulHom_image_iff := MulEquiv.uniqueProds_iff @[deprecated (since := "2024-02-04")] alias UniqueSums.addHom_image_iff := AddEquiv.uniqueSums_iff @[deprecated (since := "2024-02-04")] alias TwoUniqueProds.mulHom_image_of_injective := TwoUniqueProds.of_injective_mulHom @[deprecated (since := "2024-02-04")] alias TwoUniqueSums.addHom_image_of_injective := TwoUniqueSums.of_injective_addHom @[deprecated (since := "2024-02-04")] alias TwoUniqueProds.mulHom_image_iff := MulEquiv.twoUniqueProds_iff @[deprecated (since := "2024-02-04")] alias TwoUniqueSums.addHom_image_iff := AddEquiv.twoUniqueSums_iff instance {ι} (G : ι → Type*) [∀ i, AddZeroClass (G i)] [∀ i, TwoUniqueSums (G i)] : TwoUniqueSums (Π₀ i, G i) := TwoUniqueSums.of_injective_addHom DFinsupp.coeFnAddMonoidHom.toAddHom DFunLike.coe_injective inferInstance instance {ι G} [AddZeroClass G] [TwoUniqueSums G] : TwoUniqueSums (ι →₀ G) := TwoUniqueSums.of_injective_addHom Finsupp.coeFnAddHom.toAddHom DFunLike.coe_injective inferInstance /-- Any `ℚ`-vector space has `TwoUniqueSums`, because it is isomorphic to some `(Basis.ofVectorSpaceIndex ℚ G) →₀ ℚ` by choosing a basis, and `ℚ` already has `TwoUniqueSums` because it's ordered. -/ instance [AddCommGroup G] [Module ℚ G] : TwoUniqueSums G := TwoUniqueSums.of_injective_addHom _ (Basis.ofVectorSpace ℚ G).repr.injective inferInstance /-- Any `FreeMonoid` has the `TwoUniqueProds` property. -/ instance FreeMonoid.instTwoUniqueProds {κ : Type*} : TwoUniqueProds (FreeMonoid κ) := .of_mulHom ⟨Multiplicative.ofAdd ∘ List.length, fun _ _ ↦ congr_arg _ (List.length_append _ _)⟩ (fun _ _ _ _ h h' ↦ List.append_inj h <| Equiv.injective Multiplicative.ofAdd h'.1) /-- Any `FreeAddMonoid` has the `TwoUniqueSums` property. -/ instance FreeAddMonoid.instTwoUniqueSums {κ : Type*} : TwoUniqueSums (FreeAddMonoid κ) := .of_addHom ⟨_, List.length_append⟩ (fun _ _ _ _ h h' ↦ List.append_inj h h'.1)
Algebra\Group\Units.lean
/- Copyright (c) 2017 Kenny Lau. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Kenny Lau, Mario Carneiro, Johannes Hölzl, Chris Hughes, Jens Wagemaker, Jon Eugster -/ import Mathlib.Algebra.Group.Basic import Mathlib.Algebra.Group.Commute.Defs import Mathlib.Logic.Unique import Mathlib.Tactic.Nontriviality import Mathlib.Tactic.Lift import Mathlib.Tactic.Subsingleton /-! # Units (i.e., invertible elements) of a monoid An element of a `Monoid` is a unit if it has a two-sided inverse. ## Main declarations * `Units M`: the group of units (i.e., invertible elements) of a monoid. * `IsUnit x`: a predicate asserting that `x` is a unit (i.e., invertible element) of a monoid. For both declarations, there is an additive counterpart: `AddUnits` and `IsAddUnit`. See also `Prime`, `Associated`, and `Irreducible` in `Mathlib.Algebra.Associated`. ## Notation We provide `Mˣ` as notation for `Units M`, resembling the notation $R^{\times}$ for the units of a ring, which is common in mathematics. ## TODO The results here should be used to golf the basic `Group` lemmas. -/ assert_not_exists Multiplicative assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered open Function universe u variable {α : Type u} /-- Units of a `Monoid`, bundled version. Notation: `αˣ`. An element of a `Monoid` is a unit if it has a two-sided inverse. This version bundles the inverse element so that it can be computed. For a predicate see `IsUnit`. -/ structure Units (α : Type u) [Monoid α] where /-- The underlying value in the base `Monoid`. -/ val : α /-- The inverse value of `val` in the base `Monoid`. -/ inv : α /-- `inv` is the right inverse of `val` in the base `Monoid`. -/ val_inv : val * inv = 1 /-- `inv` is the left inverse of `val` in the base `Monoid`. -/ inv_val : inv * val = 1 attribute [coe] Units.val @[inherit_doc] postfix:1024 "ˣ" => Units -- We don't provide notation for the additive version, because its use is somewhat rare. /-- Units of an `AddMonoid`, bundled version. An element of an `AddMonoid` is a unit if it has a two-sided additive inverse. This version bundles the inverse element so that it can be computed. For a predicate see `isAddUnit`. -/ structure AddUnits (α : Type u) [AddMonoid α] where /-- The underlying value in the base `AddMonoid`. -/ val : α /-- The additive inverse value of `val` in the base `AddMonoid`. -/ neg : α /-- `neg` is the right additive inverse of `val` in the base `AddMonoid`. -/ val_neg : val + neg = 0 /-- `neg` is the left additive inverse of `val` in the base `AddMonoid`. -/ neg_val : neg + val = 0 attribute [to_additive] Units attribute [coe] AddUnits.val section HasElem @[to_additive] theorem unique_one {α : Type*} [Unique α] [One α] : default = (1 : α) := Unique.default_eq 1 end HasElem namespace Units section Monoid variable [Monoid α] -- Porting note: unclear whether this should be a `CoeHead` or `CoeTail` /-- A unit can be interpreted as a term in the base `Monoid`. -/ @[to_additive "An additive unit can be interpreted as a term in the base `AddMonoid`."] instance : CoeHead αˣ α := ⟨val⟩ /-- The inverse of a unit in a `Monoid`. -/ @[to_additive "The additive inverse of an additive unit in an `AddMonoid`."] instance instInv : Inv αˣ := ⟨fun u => ⟨u.2, u.1, u.4, u.3⟩⟩ attribute [instance] AddUnits.instNeg /- porting note: the result of these definitions is syntactically equal to `Units.val` because of the way coercions work in Lean 4, so there is no need for these custom `simp` projections. -/ /-- See Note [custom simps projection] -/ @[to_additive "See Note [custom simps projection]"] def Simps.val_inv (u : αˣ) : α := ↑(u⁻¹) initialize_simps_projections Units (as_prefix val, val_inv → null, inv → val_inv, as_prefix val_inv) initialize_simps_projections AddUnits (as_prefix val, val_neg → null, neg → val_neg, as_prefix val_neg) -- Porting note: removed `simp` tag because of the tautology @[to_additive] theorem val_mk (a : α) (b h₁ h₂) : ↑(Units.mk a b h₁ h₂) = a := rfl @[to_additive (attr := ext)] theorem ext : Function.Injective (val : αˣ → α) | ⟨v, i₁, vi₁, iv₁⟩, ⟨v', i₂, vi₂, iv₂⟩, e => by simp only at e; subst v'; congr simpa only [iv₂, vi₁, one_mul, mul_one] using mul_assoc i₂ v i₁ @[to_additive (attr := norm_cast)] theorem eq_iff {a b : αˣ} : (a : α) = b ↔ a = b := ext.eq_iff /-- Units have decidable equality if the base `Monoid` has decidable equality. -/ @[to_additive "Additive units have decidable equality if the base `AddMonoid` has deciable equality."] instance [DecidableEq α] : DecidableEq αˣ := fun _ _ => decidable_of_iff' _ Units.ext_iff @[to_additive (attr := simp)] theorem mk_val (u : αˣ) (y h₁ h₂) : mk (u : α) y h₁ h₂ = u := ext rfl /-- Copy a unit, adjusting definition equalities. -/ @[to_additive (attr := simps) "Copy an `AddUnit`, adjusting definitional equalities."] def copy (u : αˣ) (val : α) (hv : val = u) (inv : α) (hi : inv = ↑u⁻¹) : αˣ := { val, inv, inv_val := hv.symm ▸ hi.symm ▸ u.inv_val, val_inv := hv.symm ▸ hi.symm ▸ u.val_inv } @[to_additive] theorem copy_eq (u : αˣ) (val hv inv hi) : u.copy val hv inv hi = u := ext hv /-- Units of a monoid have an induced multiplication. -/ @[to_additive "Additive units of an additive monoid have an induced addition."] instance : Mul αˣ where mul u₁ u₂ := ⟨u₁.val * u₂.val, u₂.inv * u₁.inv, by rw [mul_assoc, ← mul_assoc u₂.val, val_inv, one_mul, val_inv], by rw [mul_assoc, ← mul_assoc u₁.inv, inv_val, one_mul, inv_val]⟩ /-- Units of a monoid have a unit -/ @[to_additive "Additive units of an additive monoid have a zero."] instance : One αˣ where one := ⟨1, 1, one_mul 1, one_mul 1⟩ /-- Units of a monoid have a multiplication and multiplicative identity. -/ @[to_additive "Additive units of an additive monoid have an addition and an additive identity."] instance instMulOneClass : MulOneClass αˣ where one_mul u := ext <| one_mul (u : α) mul_one u := ext <| mul_one (u : α) /-- Units of a monoid are inhabited because `1` is a unit. -/ @[to_additive "Additive units of an additive monoid are inhabited because `0` is an additive unit."] instance : Inhabited αˣ := ⟨1⟩ /-- Units of a monoid have a representation of the base value in the `Monoid`. -/ @[to_additive "Additive units of an additive monoid have a representation of the base value in the `AddMonoid`."] instance [Repr α] : Repr αˣ := ⟨reprPrec ∘ val⟩ variable (a b c : αˣ) {u : αˣ} @[to_additive (attr := simp, norm_cast)] theorem val_mul : (↑(a * b) : α) = a * b := rfl @[to_additive (attr := simp, norm_cast)] theorem val_one : ((1 : αˣ) : α) = 1 := rfl @[to_additive (attr := simp, norm_cast)] theorem val_eq_one {a : αˣ} : (a : α) = 1 ↔ a = 1 := by rw [← Units.val_one, eq_iff] @[to_additive (attr := simp)] theorem inv_mk (x y : α) (h₁ h₂) : (mk x y h₁ h₂)⁻¹ = mk y x h₂ h₁ := rfl -- Porting note: coercions are now eagerly elaborated, so no need for `val_eq_coe` @[to_additive (attr := simp)] theorem inv_eq_val_inv : a.inv = ((a⁻¹ : αˣ) : α) := rfl @[to_additive (attr := simp)] theorem inv_mul : (↑a⁻¹ * a : α) = 1 := inv_val _ @[to_additive (attr := simp)] theorem mul_inv : (a * ↑a⁻¹ : α) = 1 := val_inv _ @[to_additive] lemma commute_coe_inv : Commute (a : α) ↑a⁻¹ := by rw [Commute, SemiconjBy, inv_mul, mul_inv] @[to_additive] lemma commute_inv_coe : Commute ↑a⁻¹ (a : α) := a.commute_coe_inv.symm @[to_additive] theorem inv_mul_of_eq {a : α} (h : ↑u = a) : ↑u⁻¹ * a = 1 := by rw [← h, u.inv_mul] @[to_additive] theorem mul_inv_of_eq {a : α} (h : ↑u = a) : a * ↑u⁻¹ = 1 := by rw [← h, u.mul_inv] @[to_additive (attr := simp)] theorem mul_inv_cancel_left (a : αˣ) (b : α) : (a : α) * (↑a⁻¹ * b) = b := by rw [← mul_assoc, mul_inv, one_mul] @[to_additive (attr := simp)] theorem inv_mul_cancel_left (a : αˣ) (b : α) : (↑a⁻¹ : α) * (a * b) = b := by rw [← mul_assoc, inv_mul, one_mul] @[to_additive (attr := simp)] theorem mul_inv_cancel_right (a : α) (b : αˣ) : a * b * ↑b⁻¹ = a := by rw [mul_assoc, mul_inv, mul_one] @[to_additive (attr := simp)] theorem inv_mul_cancel_right (a : α) (b : αˣ) : a * ↑b⁻¹ * b = a := by rw [mul_assoc, inv_mul, mul_one] @[to_additive (attr := simp)] theorem mul_right_inj (a : αˣ) {b c : α} : (a : α) * b = a * c ↔ b = c := ⟨fun h => by simpa only [inv_mul_cancel_left] using congr_arg (fun x : α => ↑(a⁻¹ : αˣ) * x) h, congr_arg _⟩ @[to_additive (attr := simp)] theorem mul_left_inj (a : αˣ) {b c : α} : b * a = c * a ↔ b = c := ⟨fun h => by simpa only [mul_inv_cancel_right] using congr_arg (fun x : α => x * ↑(a⁻¹ : αˣ)) h, congr_arg (· * a.val)⟩ @[to_additive] theorem eq_mul_inv_iff_mul_eq {a b : α} : a = b * ↑c⁻¹ ↔ a * c = b := ⟨fun h => by rw [h, inv_mul_cancel_right], fun h => by rw [← h, mul_inv_cancel_right]⟩ @[to_additive] theorem eq_inv_mul_iff_mul_eq {a c : α} : a = ↑b⁻¹ * c ↔ ↑b * a = c := ⟨fun h => by rw [h, mul_inv_cancel_left], fun h => by rw [← h, inv_mul_cancel_left]⟩ @[to_additive] theorem inv_mul_eq_iff_eq_mul {b c : α} : ↑a⁻¹ * b = c ↔ b = a * c := ⟨fun h => by rw [← h, mul_inv_cancel_left], fun h => by rw [h, inv_mul_cancel_left]⟩ @[to_additive] theorem mul_inv_eq_iff_eq_mul {a c : α} : a * ↑b⁻¹ = c ↔ a = c * b := ⟨fun h => by rw [← h, inv_mul_cancel_right], fun h => by rw [h, mul_inv_cancel_right]⟩ -- Porting note: have to explicitly type annotate the 1 @[to_additive] protected theorem inv_eq_of_mul_eq_one_left {a : α} (h : a * u = 1) : ↑u⁻¹ = a := calc ↑u⁻¹ = (1 : α) * ↑u⁻¹ := by rw [one_mul] _ = a := by rw [← h, mul_inv_cancel_right] -- Porting note: have to explicitly type annotate the 1 @[to_additive] protected theorem inv_eq_of_mul_eq_one_right {a : α} (h : ↑u * a = 1) : ↑u⁻¹ = a := calc ↑u⁻¹ = ↑u⁻¹ * (1 : α) := by rw [mul_one] _ = a := by rw [← h, inv_mul_cancel_left] @[to_additive] protected theorem eq_inv_of_mul_eq_one_left {a : α} (h : ↑u * a = 1) : a = ↑u⁻¹ := (Units.inv_eq_of_mul_eq_one_right h).symm @[to_additive] protected theorem eq_inv_of_mul_eq_one_right {a : α} (h : a * u = 1) : a = ↑u⁻¹ := (Units.inv_eq_of_mul_eq_one_left h).symm @[to_additive] instance instMonoid : Monoid αˣ := { (inferInstance : MulOneClass αˣ) with mul_assoc := fun _ _ _ => ext <| mul_assoc _ _ _, npow := fun n a ↦ { val := a ^ n inv := a⁻¹ ^ n val_inv := by rw [← a.commute_coe_inv.mul_pow]; simp inv_val := by rw [← a.commute_inv_coe.mul_pow]; simp } npow_zero := fun a ↦ by ext; simp npow_succ := fun n a ↦ by ext; simp [pow_succ] } /-- Units of a monoid have division -/ @[to_additive "Additive units of an additive monoid have subtraction."] instance : Div αˣ where div := fun a b ↦ { val := a * b⁻¹ inv := b * a⁻¹ val_inv := by rw [mul_assoc, inv_mul_cancel_left, mul_inv] inv_val := by rw [mul_assoc, inv_mul_cancel_left, mul_inv] } /-- Units of a monoid form a `DivInvMonoid`. -/ @[to_additive "Additive units of an additive monoid form a `SubNegMonoid`."] instance instDivInvMonoid : DivInvMonoid αˣ where zpow := fun n a ↦ match n, a with | Int.ofNat n, a => a ^ n | Int.negSucc n, a => (a ^ n.succ)⁻¹ zpow_zero' := fun a ↦ by simp zpow_succ' := fun n a ↦ by simp [pow_succ] zpow_neg' := fun n a ↦ by simp /-- Units of a monoid form a group. -/ @[to_additive "Additive units of an additive monoid form an additive group."] instance instGroup : Group αˣ where mul_left_inv := fun u => ext u.inv_val /-- Units of a commutative monoid form a commutative group. -/ @[to_additive "Additive units of an additive commutative monoid form an additive commutative group."] instance instCommGroupUnits {α} [CommMonoid α] : CommGroup αˣ where mul_comm := fun _ _ => ext <| mul_comm _ _ @[to_additive (attr := simp, norm_cast)] lemma val_pow_eq_pow_val (n : ℕ) : ↑(a ^ n) = (a ^ n : α) := rfl @[to_additive (attr := simp)] theorem mul_inv_eq_one {a : α} : a * ↑u⁻¹ = 1 ↔ a = u := ⟨inv_inv u ▸ Units.eq_inv_of_mul_eq_one_right, fun h => mul_inv_of_eq h.symm⟩ @[to_additive (attr := simp)] theorem inv_mul_eq_one {a : α} : ↑u⁻¹ * a = 1 ↔ ↑u = a := ⟨inv_inv u ▸ Units.inv_eq_of_mul_eq_one_right, inv_mul_of_eq⟩ @[to_additive] theorem mul_eq_one_iff_eq_inv {a : α} : a * u = 1 ↔ a = ↑u⁻¹ := by rw [← mul_inv_eq_one, inv_inv] @[to_additive] theorem mul_eq_one_iff_inv_eq {a : α} : ↑u * a = 1 ↔ ↑u⁻¹ = a := by rw [← inv_mul_eq_one, inv_inv] @[to_additive] theorem inv_unique {u₁ u₂ : αˣ} (h : (↑u₁ : α) = ↑u₂) : (↑u₁⁻¹ : α) = ↑u₂⁻¹ := Units.inv_eq_of_mul_eq_one_right <| by rw [h, u₂.mul_inv] end Monoid section DivisionMonoid variable [DivisionMonoid α] @[to_additive (attr := simp, norm_cast)] lemma val_inv_eq_inv_val (u : αˣ) : ↑u⁻¹ = (u⁻¹ : α) := Eq.symm <| inv_eq_of_mul_eq_one_right u.mul_inv @[to_additive (attr := simp, norm_cast)] lemma val_div_eq_div_val : ∀ u₁ u₂ : αˣ, ↑(u₁ / u₂) = (u₁ / u₂ : α) := by simp [div_eq_mul_inv] end DivisionMonoid end Units /-- For `a, b` in a `CommMonoid` such that `a * b = 1`, makes a unit out of `a`. -/ @[to_additive "For `a, b` in an `AddCommMonoid` such that `a + b = 0`, makes an addUnit out of `a`."] def Units.mkOfMulEqOne [CommMonoid α] (a b : α) (hab : a * b = 1) : αˣ := ⟨a, b, hab, (mul_comm b a).trans hab⟩ @[to_additive (attr := simp)] theorem Units.val_mkOfMulEqOne [CommMonoid α] {a b : α} (h : a * b = 1) : (Units.mkOfMulEqOne a b h : α) = a := rfl section Monoid variable [Monoid α] {a b c : α} /-- Partial division. It is defined when the second argument is invertible, and unlike the division operator in `DivisionRing` it is not totalized at zero. -/ def divp (a : α) (u : Units α) : α := a * (u⁻¹ : αˣ) @[inherit_doc] infixl:70 " /ₚ " => divp @[simp] theorem divp_self (u : αˣ) : (u : α) /ₚ u = 1 := Units.mul_inv _ @[simp] theorem divp_one (a : α) : a /ₚ 1 = a := mul_one _ theorem divp_assoc (a b : α) (u : αˣ) : a * b /ₚ u = a * (b /ₚ u) := mul_assoc _ _ _ /-- `field_simp` needs the reverse direction of `divp_assoc` to move all `/ₚ` to the right. -/ @[field_simps] theorem divp_assoc' (x y : α) (u : αˣ) : x * (y /ₚ u) = x * y /ₚ u := (divp_assoc _ _ _).symm @[simp] theorem divp_inv (u : αˣ) : a /ₚ u⁻¹ = a * u := rfl @[simp] theorem divp_mul_cancel (a : α) (u : αˣ) : a /ₚ u * u = a := (mul_assoc _ _ _).trans <| by rw [Units.inv_mul, mul_one] @[simp] theorem mul_divp_cancel (a : α) (u : αˣ) : a * u /ₚ u = a := (mul_assoc _ _ _).trans <| by rw [Units.mul_inv, mul_one] @[simp] theorem divp_left_inj (u : αˣ) {a b : α} : a /ₚ u = b /ₚ u ↔ a = b := Units.mul_left_inj _ @[field_simps] theorem divp_divp_eq_divp_mul (x : α) (u₁ u₂ : αˣ) : x /ₚ u₁ /ₚ u₂ = x /ₚ (u₂ * u₁) := by simp only [divp, mul_inv_rev, Units.val_mul, mul_assoc] /- Porting note: to match the mathlib3 behavior, this needs to have higher simp priority than eq_divp_iff_mul_eq. -/ @[field_simps 1010] theorem divp_eq_iff_mul_eq {x : α} {u : αˣ} {y : α} : x /ₚ u = y ↔ y * u = x := u.mul_left_inj.symm.trans <| by rw [divp_mul_cancel]; exact ⟨Eq.symm, Eq.symm⟩ @[field_simps] theorem eq_divp_iff_mul_eq {x : α} {u : αˣ} {y : α} : x = y /ₚ u ↔ x * u = y := by rw [eq_comm, divp_eq_iff_mul_eq] theorem divp_eq_one_iff_eq {a : α} {u : αˣ} : a /ₚ u = 1 ↔ a = u := (Units.mul_left_inj u).symm.trans <| by rw [divp_mul_cancel, one_mul] @[simp] theorem one_divp (u : αˣ) : 1 /ₚ u = ↑u⁻¹ := one_mul _ /-- Used for `field_simp` to deal with inverses of units. -/ @[field_simps] theorem inv_eq_one_divp (u : αˣ) : ↑u⁻¹ = 1 /ₚ u := by rw [one_divp] /-- Used for `field_simp` to deal with inverses of units. This form of the lemma is essential since `field_simp` likes to use `inv_eq_one_div` to rewrite `↑u⁻¹ = ↑(1 / u)`. -/ @[field_simps] theorem inv_eq_one_divp' (u : αˣ) : ((1 / u : αˣ) : α) = 1 /ₚ u := by rw [one_div, one_divp] /-- `field_simp` moves division inside `αˣ` to the right, and this lemma lifts the calculation to `α`. -/ @[field_simps] theorem val_div_eq_divp (u₁ u₂ : αˣ) : ↑(u₁ / u₂) = ↑u₁ /ₚ u₂ := by rw [divp, division_def, Units.val_mul] end Monoid section CommMonoid variable [CommMonoid α] @[field_simps] theorem divp_mul_eq_mul_divp (x y : α) (u : αˣ) : x /ₚ u * y = x * y /ₚ u := by rw [divp, divp, mul_right_comm] -- Theoretically redundant as `field_simp` lemma. @[field_simps] theorem divp_eq_divp_iff {x y : α} {ux uy : αˣ} : x /ₚ ux = y /ₚ uy ↔ x * uy = y * ux := by rw [divp_eq_iff_mul_eq, divp_mul_eq_mul_divp, divp_eq_iff_mul_eq] -- Theoretically redundant as `field_simp` lemma. @[field_simps] theorem divp_mul_divp (x y : α) (ux uy : αˣ) : x /ₚ ux * (y /ₚ uy) = x * y /ₚ (ux * uy) := by rw [divp_mul_eq_mul_divp, divp_assoc', divp_divp_eq_divp_mul] variable [Subsingleton αˣ] {a b : α} @[to_additive] theorem eq_one_of_mul_right (h : a * b = 1) : a = 1 := congr_arg Units.inv <| Subsingleton.elim (Units.mk _ _ (by rwa [mul_comm]) h) 1 @[to_additive] theorem eq_one_of_mul_left (h : a * b = 1) : b = 1 := congr_arg Units.inv <| Subsingleton.elim (Units.mk _ _ h <| by rwa [mul_comm]) 1 @[to_additive (attr := simp)] theorem mul_eq_one : a * b = 1 ↔ a = 1 ∧ b = 1 := ⟨fun h => ⟨eq_one_of_mul_right h, eq_one_of_mul_left h⟩, by rintro ⟨rfl, rfl⟩ exact mul_one _⟩ end CommMonoid /-! # `IsUnit` predicate -/ section IsUnit variable {M : Type*} {N : Type*} /-- An element `a : M` of a `Monoid` is a unit if it has a two-sided inverse. The actual definition says that `a` is equal to some `u : Mˣ`, where `Mˣ` is a bundled version of `IsUnit`. -/ @[to_additive "An element `a : M` of an `AddMonoid` is an `AddUnit` if it has a two-sided additive inverse. The actual definition says that `a` is equal to some `u : AddUnits M`, where `AddUnits M` is a bundled version of `IsAddUnit`."] def IsUnit [Monoid M] (a : M) : Prop := ∃ u : Mˣ, (u : M) = a /-- See `isUnit_iff_exists_and_exists` for a similar lemma with two existentials. -/ @[to_additive "See `isAddUnit_iff_exists_and_exists` for a similar lemma with two existentials."] lemma isUnit_iff_exists [Monoid M] {x : M} : IsUnit x ↔ ∃ b, x * b = 1 ∧ b * x = 1 := by refine ⟨fun ⟨u, hu⟩ => ?_, fun ⟨b, h1b, h2b⟩ => ⟨⟨x, b, h1b, h2b⟩, rfl⟩⟩ subst x exact ⟨u.inv, u.val_inv, u.inv_val⟩ /-- See `isUnit_iff_exists` for a similar lemma with one existential. -/ @[to_additive "See `isAddUnit_iff_exists` for a similar lemma with one existential."] theorem isUnit_iff_exists_and_exists [Monoid M] {a : M} : IsUnit a ↔ (∃ b, a * b = 1) ∧ (∃ c, c * a = 1) := isUnit_iff_exists.trans ⟨fun ⟨b, hba, hab⟩ => ⟨⟨b, hba⟩, ⟨b, hab⟩⟩, fun ⟨⟨b, hb⟩, ⟨_, hc⟩⟩ => ⟨b, hb, left_inv_eq_right_inv hc hb ▸ hc⟩⟩ @[to_additive (attr := nontriviality)] theorem isUnit_of_subsingleton [Monoid M] [Subsingleton M] (a : M) : IsUnit a := ⟨⟨a, a, by subsingleton, by subsingleton⟩, rfl⟩ @[to_additive] instance [Monoid M] : CanLift M Mˣ Units.val IsUnit := { prf := fun _ ↦ id } /-- A subsingleton `Monoid` has a unique unit. -/ @[to_additive "A subsingleton `AddMonoid` has a unique additive unit."] instance [Monoid M] [Subsingleton M] : Unique Mˣ where uniq _ := Units.val_eq_one.mp (by subsingleton) @[to_additive (attr := simp)] protected theorem Units.isUnit [Monoid M] (u : Mˣ) : IsUnit (u : M) := ⟨u, rfl⟩ @[to_additive (attr := simp)] theorem isUnit_one [Monoid M] : IsUnit (1 : M) := ⟨1, rfl⟩ @[to_additive] theorem isUnit_of_mul_eq_one [CommMonoid M] (a b : M) (h : a * b = 1) : IsUnit a := ⟨Units.mkOfMulEqOne a b h, rfl⟩ @[to_additive] theorem isUnit_of_mul_eq_one_right [CommMonoid M] (a b : M) (h : a * b = 1) : IsUnit b := by rw [mul_comm] at h exact isUnit_of_mul_eq_one b a h section Monoid variable [Monoid M] {a b : M} @[to_additive IsAddUnit.exists_neg] lemma IsUnit.exists_right_inv (h : IsUnit a) : ∃ b, a * b = 1 := by rcases h with ⟨⟨a, b, hab, _⟩, rfl⟩ exact ⟨b, hab⟩ @[to_additive IsAddUnit.exists_neg'] lemma IsUnit.exists_left_inv {a : M} (h : IsUnit a) : ∃ b, b * a = 1 := by rcases h with ⟨⟨a, b, _, hba⟩, rfl⟩ exact ⟨b, hba⟩ @[to_additive] lemma IsUnit.mul : IsUnit a → IsUnit b → IsUnit (a * b) := by rintro ⟨x, rfl⟩ ⟨y, rfl⟩; exact ⟨x * y, rfl⟩ @[to_additive] lemma IsUnit.pow (n : ℕ) : IsUnit a → IsUnit (a ^ n) := by rintro ⟨u, rfl⟩; exact ⟨u ^ n, rfl⟩ theorem units_eq_one [Unique Mˣ] (u : Mˣ) : u = 1 := by subsingleton @[to_additive] lemma isUnit_iff_eq_one [Unique Mˣ] {x : M} : IsUnit x ↔ x = 1 := ⟨fun ⟨u, hu⟩ ↦ by rw [← hu, Subsingleton.elim u 1, Units.val_one], fun h ↦ h ▸ isUnit_one⟩ end Monoid @[to_additive] theorem isUnit_iff_exists_inv [CommMonoid M] {a : M} : IsUnit a ↔ ∃ b, a * b = 1 := ⟨fun h => h.exists_right_inv, fun ⟨b, hab⟩ => isUnit_of_mul_eq_one _ b hab⟩ @[to_additive] theorem isUnit_iff_exists_inv' [CommMonoid M] {a : M} : IsUnit a ↔ ∃ b, b * a = 1 := by simp [isUnit_iff_exists_inv, mul_comm] /-- Multiplication by a `u : Mˣ` on the right doesn't affect `IsUnit`. -/ @[to_additive (attr := simp) "Addition of a `u : AddUnits M` on the right doesn't affect `IsAddUnit`."] theorem Units.isUnit_mul_units [Monoid M] (a : M) (u : Mˣ) : IsUnit (a * u) ↔ IsUnit a := Iff.intro (fun ⟨v, hv⟩ => by have : IsUnit (a * ↑u * ↑u⁻¹) := by exists v * u⁻¹; rw [← hv, Units.val_mul] rwa [mul_assoc, Units.mul_inv, mul_one] at this) fun v => v.mul u.isUnit /-- Multiplication by a `u : Mˣ` on the left doesn't affect `IsUnit`. -/ @[to_additive (attr := simp) "Addition of a `u : AddUnits M` on the left doesn't affect `IsAddUnit`."] theorem Units.isUnit_units_mul {M : Type*} [Monoid M] (u : Mˣ) (a : M) : IsUnit (↑u * a) ↔ IsUnit a := Iff.intro (fun ⟨v, hv⟩ => by have : IsUnit (↑u⁻¹ * (↑u * a)) := by exists u⁻¹ * v; rw [← hv, Units.val_mul] rwa [← mul_assoc, Units.inv_mul, one_mul] at this) u.isUnit.mul @[to_additive] theorem isUnit_of_mul_isUnit_left [CommMonoid M] {x y : M} (hu : IsUnit (x * y)) : IsUnit x := let ⟨z, hz⟩ := isUnit_iff_exists_inv.1 hu isUnit_iff_exists_inv.2 ⟨y * z, by rwa [← mul_assoc]⟩ @[to_additive] theorem isUnit_of_mul_isUnit_right [CommMonoid M] {x y : M} (hu : IsUnit (x * y)) : IsUnit y := @isUnit_of_mul_isUnit_left _ _ y x <| by rwa [mul_comm] namespace IsUnit @[to_additive (attr := simp)] theorem mul_iff [CommMonoid M] {x y : M} : IsUnit (x * y) ↔ IsUnit x ∧ IsUnit y := ⟨fun h => ⟨isUnit_of_mul_isUnit_left h, isUnit_of_mul_isUnit_right h⟩, fun h => IsUnit.mul h.1 h.2⟩ section Monoid variable [Monoid M] {a b c : M} /-- The element of the group of units, corresponding to an element of a monoid which is a unit. When `α` is a `DivisionMonoid`, use `IsUnit.unit'` instead. -/ protected noncomputable def unit (h : IsUnit a) : Mˣ := (Classical.choose h).copy a (Classical.choose_spec h).symm _ rfl -- Porting note: `to_additive` doesn't carry over `noncomputable` so we make an explicit defn /-- "The element of the additive group of additive units, corresponding to an element of an additive monoid which is an additive unit. When `α` is a `SubtractionMonoid`, use `IsAddUnit.addUnit'` instead. -/ protected noncomputable def _root_.IsAddUnit.addUnit [AddMonoid N] {a : N} (h : IsAddUnit a) : AddUnits N := (Classical.choose h).copy a (Classical.choose_spec h).symm _ rfl attribute [to_additive existing] IsUnit.unit @[to_additive (attr := simp)] theorem unit_of_val_units {a : Mˣ} (h : IsUnit (a : M)) : h.unit = a := Units.ext <| rfl @[to_additive (attr := simp)] theorem unit_spec (h : IsUnit a) : ↑h.unit = a := rfl @[to_additive (attr := simp)] theorem unit_one (h : IsUnit (1 : M)) : h.unit = 1 := Units.eq_iff.1 rfl @[to_additive (attr := simp)] theorem val_inv_mul (h : IsUnit a) : ↑h.unit⁻¹ * a = 1 := Units.mul_inv _ @[to_additive (attr := simp)] theorem mul_val_inv (h : IsUnit a) : a * ↑h.unit⁻¹ = 1 := by rw [← h.unit.mul_inv]; congr /-- `IsUnit x` is decidable if we can decide if `x` comes from `Mˣ`. -/ @[to_additive "`IsAddUnit x` is decidable if we can decide if `x` comes from `AddUnits M`."] instance (x : M) [h : Decidable (∃ u : Mˣ, ↑u = x)] : Decidable (IsUnit x) := h @[to_additive] theorem mul_left_inj (h : IsUnit a) : b * a = c * a ↔ b = c := let ⟨u, hu⟩ := h hu ▸ u.mul_left_inj @[to_additive] theorem mul_right_inj (h : IsUnit a) : a * b = a * c ↔ b = c := let ⟨u, hu⟩ := h hu ▸ u.mul_right_inj @[to_additive] protected theorem mul_left_cancel (h : IsUnit a) : a * b = a * c → b = c := h.mul_right_inj.1 @[to_additive] protected theorem mul_right_cancel (h : IsUnit b) : a * b = c * b → a = c := h.mul_left_inj.1 @[to_additive] protected theorem mul_right_injective (h : IsUnit a) : Injective (a * ·) := fun _ _ => h.mul_left_cancel @[to_additive] protected theorem mul_left_injective (h : IsUnit b) : Injective (· * b) := fun _ _ => h.mul_right_cancel @[to_additive] theorem isUnit_iff_mulLeft_bijective {a : M} : IsUnit a ↔ Function.Bijective (a * ·) := ⟨fun h ↦ ⟨h.mul_right_injective, fun y ↦ ⟨h.unit⁻¹ * y, by simp [← mul_assoc]⟩⟩, fun h ↦ ⟨⟨a, _, (h.2 1).choose_spec, h.1 (by simpa [mul_assoc] using congr_arg (· * a) (h.2 1).choose_spec)⟩, rfl⟩⟩ @[to_additive] theorem isUnit_iff_mulRight_bijective {a : M} : IsUnit a ↔ Function.Bijective (· * a) := ⟨fun h ↦ ⟨h.mul_left_injective, fun y ↦ ⟨y * h.unit⁻¹, by simp [mul_assoc]⟩⟩, fun h ↦ ⟨⟨a, _, h.1 (by simpa [mul_assoc] using congr_arg (a * ·) (h.2 1).choose_spec), (h.2 1).choose_spec⟩, rfl⟩⟩ end Monoid section DivisionMonoid variable [DivisionMonoid α] {a b c : α} @[to_additive (attr := simp)] protected theorem inv_mul_cancel : IsUnit a → a⁻¹ * a = 1 := by rintro ⟨u, rfl⟩ rw [← Units.val_inv_eq_inv_val, Units.inv_mul] @[to_additive (attr := simp)] protected theorem mul_inv_cancel : IsUnit a → a * a⁻¹ = 1 := by rintro ⟨u, rfl⟩ rw [← Units.val_inv_eq_inv_val, Units.mul_inv] /-- The element of the group of units, corresponding to an element of a monoid which is a unit. As opposed to `IsUnit.unit`, the inverse is computable and comes from the inversion on `α`. This is useful to transfer properties of inversion in `Units α` to `α`. See also `toUnits`. -/ @[to_additive (attr := simps val ) "The element of the additive group of additive units, corresponding to an element of an additive monoid which is an additive unit. As opposed to `IsAddUnit.addUnit`, the negation is computable and comes from the negation on `α`. This is useful to transfer properties of negation in `AddUnits α` to `α`. See also `toAddUnits`."] def unit' (h : IsUnit a) : αˣ := ⟨a, a⁻¹, h.mul_inv_cancel, h.inv_mul_cancel⟩ -- Porting note (#11215): TODO: `simps val_inv` fails @[to_additive] lemma val_inv_unit' (h : IsUnit a) : ↑(h.unit'⁻¹) = a⁻¹ := rfl @[to_additive (attr := simp)] protected lemma mul_inv_cancel_left (h : IsUnit a) : ∀ b, a * (a⁻¹ * b) = b := h.unit'.mul_inv_cancel_left @[to_additive (attr := simp)] protected lemma inv_mul_cancel_left (h : IsUnit a) : ∀ b, a⁻¹ * (a * b) = b := h.unit'.inv_mul_cancel_left @[to_additive (attr := simp)] protected lemma mul_inv_cancel_right (h : IsUnit b) (a : α) : a * b * b⁻¹ = a := h.unit'.mul_inv_cancel_right _ @[to_additive (attr := simp)] protected lemma inv_mul_cancel_right (h : IsUnit b) (a : α) : a * b⁻¹ * b = a := h.unit'.inv_mul_cancel_right _ @[to_additive] protected lemma div_self (h : IsUnit a) : a / a = 1 := by rw [div_eq_mul_inv, h.mul_inv_cancel] @[to_additive] protected lemma eq_mul_inv_iff_mul_eq (h : IsUnit c) : a = b * c⁻¹ ↔ a * c = b := h.unit'.eq_mul_inv_iff_mul_eq @[to_additive] protected lemma eq_inv_mul_iff_mul_eq (h : IsUnit b) : a = b⁻¹ * c ↔ b * a = c := h.unit'.eq_inv_mul_iff_mul_eq @[to_additive] protected lemma inv_mul_eq_iff_eq_mul (h : IsUnit a) : a⁻¹ * b = c ↔ b = a * c := h.unit'.inv_mul_eq_iff_eq_mul @[to_additive] protected lemma mul_inv_eq_iff_eq_mul (h : IsUnit b) : a * b⁻¹ = c ↔ a = c * b := h.unit'.mul_inv_eq_iff_eq_mul @[to_additive] protected lemma mul_inv_eq_one (h : IsUnit b) : a * b⁻¹ = 1 ↔ a = b := @Units.mul_inv_eq_one _ _ h.unit' _ @[to_additive] protected lemma inv_mul_eq_one (h : IsUnit a) : a⁻¹ * b = 1 ↔ a = b := @Units.inv_mul_eq_one _ _ h.unit' _ @[to_additive] protected lemma mul_eq_one_iff_eq_inv (h : IsUnit b) : a * b = 1 ↔ a = b⁻¹ := @Units.mul_eq_one_iff_eq_inv _ _ h.unit' _ @[to_additive] protected lemma mul_eq_one_iff_inv_eq (h : IsUnit a) : a * b = 1 ↔ a⁻¹ = b := @Units.mul_eq_one_iff_inv_eq _ _ h.unit' _ @[to_additive (attr := simp)] protected lemma div_mul_cancel (h : IsUnit b) (a : α) : a / b * b = a := by rw [div_eq_mul_inv, h.inv_mul_cancel_right] @[to_additive (attr := simp)] protected lemma mul_div_cancel_right (h : IsUnit b) (a : α) : a * b / b = a := by rw [div_eq_mul_inv, h.mul_inv_cancel_right] @[to_additive] protected lemma mul_one_div_cancel (h : IsUnit a) : a * (1 / a) = 1 := by simp [h] @[to_additive] protected lemma one_div_mul_cancel (h : IsUnit a) : 1 / a * a = 1 := by simp [h] @[to_additive] lemma inv (h : IsUnit a) : IsUnit a⁻¹ := by obtain ⟨u, hu⟩ := h rw [← hu, ← Units.val_inv_eq_inv_val] exact Units.isUnit _ @[to_additive] lemma div (ha : IsUnit a) (hb : IsUnit b) : IsUnit (a / b) := by rw [div_eq_mul_inv]; exact ha.mul hb.inv @[to_additive] protected lemma div_left_inj (h : IsUnit c) : a / c = b / c ↔ a = b := by simp only [div_eq_mul_inv] exact Units.mul_left_inj h.inv.unit' @[to_additive] protected lemma div_eq_iff (h : IsUnit b) : a / b = c ↔ a = c * b := by rw [div_eq_mul_inv, h.mul_inv_eq_iff_eq_mul] @[to_additive] protected lemma eq_div_iff (h : IsUnit c) : a = b / c ↔ a * c = b := by rw [div_eq_mul_inv, h.eq_mul_inv_iff_mul_eq] @[to_additive] protected lemma div_eq_of_eq_mul (h : IsUnit b) : a = c * b → a / b = c := h.div_eq_iff.2 @[to_additive] protected lemma eq_div_of_mul_eq (h : IsUnit c) : a * c = b → a = b / c := h.eq_div_iff.2 @[to_additive] protected lemma div_eq_one_iff_eq (h : IsUnit b) : a / b = 1 ↔ a = b := ⟨eq_of_div_eq_one, fun hab => hab.symm ▸ h.div_self⟩ @[to_additive] protected lemma div_mul_cancel_right (h : IsUnit b) (a : α) : b / (a * b) = a⁻¹ := by rw [div_eq_mul_inv, mul_inv_rev, h.mul_inv_cancel_left] @[to_additive] protected lemma div_mul_left (h : IsUnit b) : b / (a * b) = 1 / a := by rw [h.div_mul_cancel_right, one_div] @[to_additive] protected lemma mul_div_mul_right (h : IsUnit c) (a b : α) : a * c / (b * c) = a / b := by simp only [div_eq_mul_inv, mul_inv_rev, mul_assoc, h.mul_inv_cancel_left] @[to_additive] protected lemma mul_mul_div (a : α) (h : IsUnit b) : a * b * (1 / b) = a := by simp [h] end DivisionMonoid section DivisionCommMonoid variable [DivisionCommMonoid α] {a b c d : α} @[to_additive] protected lemma div_mul_cancel_left (h : IsUnit a) (b : α) : a / (a * b) = b⁻¹ := by rw [mul_comm, h.div_mul_cancel_right] @[to_additive] protected lemma div_mul_right (h : IsUnit a) (b : α) : a / (a * b) = 1 / b := by rw [mul_comm, h.div_mul_left] @[to_additive] protected lemma mul_div_cancel_left (h : IsUnit a) (b : α) : a * b / a = b := by rw [mul_comm, h.mul_div_cancel_right] @[to_additive] protected lemma mul_div_cancel (h : IsUnit a) (b : α) : a * (b / a) = b := by rw [mul_comm, h.div_mul_cancel] @[to_additive] protected lemma mul_div_mul_left (h : IsUnit c) (a b : α) : c * a / (c * b) = a / b := by rw [mul_comm c, mul_comm c, h.mul_div_mul_right] @[to_additive] protected lemma mul_eq_mul_of_div_eq_div (hb : IsUnit b) (hd : IsUnit d) (a c : α) (h : a / b = c / d) : a * d = c * b := by rw [← mul_one a, ← hb.div_self, ← mul_comm_div, h, div_mul_eq_mul_div, hd.div_mul_cancel] @[to_additive] protected lemma div_eq_div_iff (hb : IsUnit b) (hd : IsUnit d) : a / b = c / d ↔ a * d = c * b := by rw [← (hb.mul hd).mul_left_inj, ← mul_assoc, hb.div_mul_cancel, ← mul_assoc, mul_right_comm, hd.div_mul_cancel] @[to_additive] protected lemma div_div_cancel (h : IsUnit a) : a / (a / b) = b := by rw [div_div_eq_mul_div, h.mul_div_cancel_left] @[to_additive] protected lemma div_div_cancel_left (h : IsUnit a) : a / b / a = b⁻¹ := by rw [div_eq_mul_inv, div_eq_mul_inv, mul_right_comm, h.mul_inv_cancel, one_mul] end DivisionCommMonoid end IsUnit @[field_simps] lemma divp_eq_div [DivisionMonoid α] (a : α) (u : αˣ) : a /ₚ u = a / u := by rw [div_eq_mul_inv, divp, u.val_inv_eq_inv_val] @[to_additive] lemma Group.isUnit [Group α] (a : α) : IsUnit a := ⟨⟨a, a⁻¹, mul_inv_self _, inv_mul_self _⟩, rfl⟩ -- namespace end IsUnit -- section section NoncomputableDefs variable {M : Type*} /-- Constructs an inv operation for a `Monoid` consisting only of units. -/ noncomputable def invOfIsUnit [Monoid M] (h : ∀ a : M, IsUnit a) : Inv M where inv := fun a => ↑(h a).unit⁻¹ /-- Constructs a `Group` structure on a `Monoid` consisting only of units. -/ noncomputable def groupOfIsUnit [hM : Monoid M] (h : ∀ a : M, IsUnit a) : Group M := { hM with toInv := invOfIsUnit h, mul_left_inv := fun a => by change ↑(h a).unit⁻¹ * a = 1 rw [Units.inv_mul_eq_iff_eq_mul, (h a).unit_spec, mul_one] } /-- Constructs a `CommGroup` structure on a `CommMonoid` consisting only of units. -/ noncomputable def commGroupOfIsUnit [hM : CommMonoid M] (h : ∀ a : M, IsUnit a) : CommGroup M := { hM with toInv := invOfIsUnit h, mul_left_inv := fun a => by change ↑(h a).unit⁻¹ * a = 1 rw [Units.inv_mul_eq_iff_eq_mul, (h a).unit_spec, mul_one] } end NoncomputableDefs attribute [deprecated div_mul_cancel_right (since := "2024-03-20")] IsUnit.div_mul_left attribute [deprecated sub_add_cancel_right (since := "2024-03-20")] IsAddUnit.sub_add_left attribute [deprecated div_mul_cancel_left (since := "2024-03-20")] IsUnit.div_mul_right attribute [deprecated sub_add_cancel_left (since := "2024-03-20")] IsAddUnit.sub_add_right -- The names `IsUnit.mul_div_cancel` and `IsAddUnit.add_sub_cancel` have been reused -- @[deprecated (since := "2024-03-20")] alias IsUnit.mul_div_cancel := IsUnit.mul_div_cancel_right -- @[deprecated (since := "2024-03-20")] -- alias IsAddUnit.add_sub_cancel := IsAddUnit.add_sub_cancel_right @[deprecated (since := "2024-03-20")] alias IsUnit.mul_div_cancel' := IsUnit.mul_div_cancel @[deprecated (since := "2024-03-20")] alias IsAddUnit.add_sub_cancel' := IsAddUnit.add_sub_cancel
Algebra\Group\ZeroOne.lean
/- Copyright (c) 2021 Gabriel Ebner. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Gabriel Ebner, Mario Carneiro -/ import Mathlib.Tactic.ToAdditive /-! ## Classes for `Zero` and `One` -/ class Zero.{u} (α : Type u) where zero : α instance (priority := 300) Zero.toOfNat0 {α} [Zero α] : OfNat α (nat_lit 0) where ofNat := ‹Zero α›.1 instance (priority := 200) Zero.ofOfNat0 {α} [OfNat α (nat_lit 0)] : Zero α where zero := 0 universe u @[to_additive] class One (α : Type u) where one : α @[to_additive existing Zero.toOfNat0] instance (priority := 300) One.toOfNat1 {α} [One α] : OfNat α (nat_lit 1) where ofNat := ‹One α›.1 @[to_additive existing Zero.ofOfNat0, to_additive_change_numeral 2] instance (priority := 200) One.ofOfNat1 {α} [OfNat α (nat_lit 1)] : One α where one := 1 attribute [to_additive_change_numeral 2] OfNat OfNat.ofNat
Algebra\Group\Action\Basic.lean
/- Copyright (c) 2018 Chris Hughes. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Chris Hughes -/ import Mathlib.Algebra.Group.Action.Units import Mathlib.Algebra.Group.Invertible.Basic import Mathlib.GroupTheory.Perm.Basic /-! # More lemmas about group actions This file contains lemmas about group actions that require more imports than `Mathlib.Algebra.Group.Action.Defs` offers. -/ assert_not_exists MonoidWithZero variable {α β γ : Type*} section MulAction section Group variable [Group α] [MulAction α β] /-- Given an action of a group `α` on `β`, each `g : α` defines a permutation of `β`. -/ @[to_additive (attr := simps)] def MulAction.toPerm (a : α) : Equiv.Perm β := ⟨fun x => a • x, fun x => a⁻¹ • x, inv_smul_smul a, smul_inv_smul a⟩ /-- Given an action of an additive group `α` on `β`, each `g : α` defines a permutation of `β`. -/ add_decl_doc AddAction.toPerm /-- `MulAction.toPerm` is injective on faithful actions. -/ @[to_additive "`AddAction.toPerm` is injective on faithful actions."] lemma MulAction.toPerm_injective [FaithfulSMul α β] : Function.Injective (MulAction.toPerm : α → Equiv.Perm β) := (show Function.Injective (Equiv.toFun ∘ MulAction.toPerm) from smul_left_injective').of_comp variable (α) (β) /-- Given an action of a group `α` on a set `β`, each `g : α` defines a permutation of `β`. -/ @[simps] def MulAction.toPermHom : α →* Equiv.Perm β where toFun := MulAction.toPerm map_one' := Equiv.ext <| one_smul α map_mul' u₁ u₂ := Equiv.ext <| mul_smul (u₁ : α) u₂ /-- Given an action of an additive group `α` on a set `β`, each `g : α` defines a permutation of `β`. -/ @[simps!] def AddAction.toPermHom (α : Type*) [AddGroup α] [AddAction α β] : α →+ Additive (Equiv.Perm β) := MonoidHom.toAdditive'' <| MulAction.toPermHom (Multiplicative α) β /-- The tautological action by `Equiv.Perm α` on `α`. This generalizes `Function.End.applyMulAction`. -/ instance Equiv.Perm.applyMulAction (α : Type*) : MulAction (Equiv.Perm α) α where smul f a := f a one_smul _ := rfl mul_smul _ _ _ := rfl @[simp] protected lemma Equiv.Perm.smul_def {α : Type*} (f : Equiv.Perm α) (a : α) : f • a = f a := rfl /-- `Equiv.Perm.applyMulAction` is faithful. -/ instance Equiv.Perm.applyFaithfulSMul (α : Type*) : FaithfulSMul (Equiv.Perm α) α := ⟨Equiv.ext⟩ variable {α} {β} @[to_additive] protected lemma MulAction.bijective (g : α) : Function.Bijective (g • · : β → β) := (MulAction.toPerm g).bijective @[to_additive] protected lemma MulAction.injective (g : α) : Function.Injective (g • · : β → β) := (MulAction.bijective g).injective @[to_additive] protected lemma MulAction.surjective (g : α) : Function.Surjective (g • · : β → β) := (MulAction.bijective g).surjective @[to_additive] lemma smul_left_cancel (g : α) {x y : β} (h : g • x = g • y) : x = y := MulAction.injective g h @[to_additive (attr := simp)] lemma smul_left_cancel_iff (g : α) {x y : β} : g • x = g • y ↔ x = y := (MulAction.injective g).eq_iff @[to_additive] lemma smul_eq_iff_eq_inv_smul (g : α) {x y : β} : g • x = y ↔ x = g⁻¹ • y := (MulAction.toPerm g).apply_eq_iff_eq_symm_apply end Group section Monoid variable [Monoid α] [MulAction α β] (c : α) (x y : β) [Invertible c] @[simp] lemma invOf_smul_smul : ⅟c • c • x = x := inv_smul_smul (unitOfInvertible c) _ @[simp] lemma smul_invOf_smul : c • (⅟ c • x) = x := smul_inv_smul (unitOfInvertible c) _ variable {c x y} lemma invOf_smul_eq_iff : ⅟c • x = y ↔ x = c • y := inv_smul_eq_iff (g := unitOfInvertible c) lemma smul_eq_iff_eq_invOf_smul : c • x = y ↔ x = ⅟c • y := smul_eq_iff_eq_inv_smul (g := unitOfInvertible c) end Monoid end MulAction section Arrow /-- If `G` acts on `A`, then it acts also on `A → B`, by `(g • F) a = F (g⁻¹ • a)`. -/ @[to_additive (attr := simps) arrowAddAction "If `G` acts on `A`, then it acts also on `A → B`, by `(g +ᵥ F) a = F (g⁻¹ +ᵥ a)`"] def arrowAction {G A B : Type*} [DivisionMonoid G] [MulAction G A] : MulAction G (A → B) where smul g F a := F (g⁻¹ • a) one_smul f := by show (fun x => f ((1 : G)⁻¹ • x)) = f simp only [inv_one, one_smul] mul_smul x y f := by show (fun a => f ((x*y)⁻¹ • a)) = (fun a => f (y⁻¹ • x⁻¹ • a)) simp only [mul_smul, mul_inv_rev] end Arrow namespace IsUnit variable [Monoid α] [MulAction α β] @[to_additive] lemma smul_left_cancel {a : α} (ha : IsUnit a) {x y : β} : a • x = a • y ↔ x = y := let ⟨u, hu⟩ := ha hu ▸ smul_left_cancel_iff u end IsUnit section SMul variable [Group α] [Monoid β] [MulAction α β] [SMulCommClass α β β] [IsScalarTower α β β] @[simp] lemma isUnit_smul_iff (g : α) (m : β) : IsUnit (g • m) ↔ IsUnit m := ⟨fun h => inv_smul_smul g m ▸ h.smul g⁻¹, IsUnit.smul g⟩ end SMul
Algebra\Group\Action\Defs.lean
/- Copyright (c) 2018 Chris Hughes. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Chris Hughes, Yury Kudryashov -/ import Mathlib.Algebra.Group.Commute.Defs import Mathlib.Algebra.Group.TypeTags import Mathlib.Algebra.Opposites import Mathlib.Logic.Embedding.Basic /-! # Definitions of group actions This file defines a hierarchy of group action type-classes on top of the previously defined notation classes `SMul` and its additive version `VAdd`: * `MulAction M α` and its additive version `AddAction G P` are typeclasses used for actions of multiplicative and additive monoids and groups; they extend notation classes `SMul` and `VAdd` that are defined in `Algebra.Group.Defs`; * `DistribMulAction M A` is a typeclass for an action of a multiplicative monoid on an additive monoid such that `a • (b + c) = a • b + a • c` and `a • 0 = 0`. The hierarchy is extended further by `Module`, defined elsewhere. Also provided are typeclasses for faithful and transitive actions, and typeclasses regarding the interaction of different group actions, * `SMulCommClass M N α` and its additive version `VAddCommClass M N α`; * `IsScalarTower M N α` and its additive version `VAddAssocClass M N α`; * `IsCentralScalar M α` and its additive version `IsCentralVAdd M N α`. ## Notation - `a • b` is used as notation for `SMul.smul a b`. - `a +ᵥ b` is used as notation for `VAdd.vadd a b`. ## Implementation details This file should avoid depending on other parts of `GroupTheory`, to avoid import cycles. More sophisticated lemmas belong in `GroupTheory.GroupAction`. ## Tags group action -/ assert_not_exists MonoidWithZero open Function (Injective Surjective) variable {M N G H A B α β γ δ : Type*} /-! ### Faithful actions -/ /-- Typeclass for faithful actions. -/ class FaithfulVAdd (G : Type*) (P : Type*) [VAdd G P] : Prop where /-- Two elements `g₁` and `g₂` are equal whenever they act in the same way on all points. -/ eq_of_vadd_eq_vadd : ∀ {g₁ g₂ : G}, (∀ p : P, g₁ +ᵥ p = g₂ +ᵥ p) → g₁ = g₂ /-- Typeclass for faithful actions. -/ @[to_additive] class FaithfulSMul (M : Type*) (α : Type*) [SMul M α] : Prop where /-- Two elements `m₁` and `m₂` are equal whenever they act in the same way on all points. -/ eq_of_smul_eq_smul : ∀ {m₁ m₂ : M}, (∀ a : α, m₁ • a = m₂ • a) → m₁ = m₂ export FaithfulSMul (eq_of_smul_eq_smul) export FaithfulVAdd (eq_of_vadd_eq_vadd) @[to_additive] lemma smul_left_injective' [SMul M α] [FaithfulSMul M α] : Injective ((· • ·) : M → α → α) := fun _ _ h ↦ FaithfulSMul.eq_of_smul_eq_smul (congr_fun h) -- see Note [lower instance priority] /-- See also `Monoid.toMulAction` and `MulZeroClass.toSMulWithZero`. -/ @[to_additive "See also `AddMonoid.toAddAction`"] instance (priority := 910) Mul.toSMul (α : Type*) [Mul α] : SMul α α := ⟨(· * ·)⟩ @[to_additive (attr := simp)] lemma smul_eq_mul (α : Type*) [Mul α] {a a' : α} : a • a' = a * a' := rfl /-- `Monoid.toMulAction` is faithful on cancellative monoids. -/ @[to_additive " `AddMonoid.toAddAction` is faithful on additive cancellative monoids. "] instance RightCancelMonoid.faithfulSMul [RightCancelMonoid α] : FaithfulSMul α α := ⟨fun h ↦ mul_right_cancel (h 1)⟩ /-- Type class for additive monoid actions. -/ class AddAction (G : Type*) (P : Type*) [AddMonoid G] extends VAdd G P where /-- Zero is a neutral element for `+ᵥ` -/ protected zero_vadd : ∀ p : P, (0 : G) +ᵥ p = p /-- Associativity of `+` and `+ᵥ` -/ add_vadd : ∀ (g₁ g₂ : G) (p : P), g₁ + g₂ +ᵥ p = g₁ +ᵥ (g₂ +ᵥ p) /-- Typeclass for multiplicative actions by monoids. This generalizes group actions. -/ @[to_additive (attr := ext)] class MulAction (α : Type*) (β : Type*) [Monoid α] extends SMul α β where /-- One is the neutral element for `•` -/ protected one_smul : ∀ b : β, (1 : α) • b = b /-- Associativity of `•` and `*` -/ mul_smul : ∀ (x y : α) (b : β), (x * y) • b = x • y • b /-! ### (Pre)transitive action `M` acts pretransitively on `α` if for any `x y` there is `g` such that `g • x = y` (or `g +ᵥ x = y` for an additive action). A transitive action should furthermore have `α` nonempty. In this section we define typeclasses `MulAction.IsPretransitive` and `AddAction.IsPretransitive` and provide `MulAction.exists_smul_eq`/`AddAction.exists_vadd_eq`, `MulAction.surjective_smul`/`AddAction.surjective_vadd` as public interface to access this property. We do not provide typeclasses `*Action.IsTransitive`; users should assume `[MulAction.IsPretransitive M α] [Nonempty α]` instead. -/ /-- `M` acts pretransitively on `α` if for any `x y` there is `g` such that `g +ᵥ x = y`. A transitive action should furthermore have `α` nonempty. -/ class AddAction.IsPretransitive (M α : Type*) [VAdd M α] : Prop where /-- There is `g` such that `g +ᵥ x = y`. -/ exists_vadd_eq : ∀ x y : α, ∃ g : M, g +ᵥ x = y /-- `M` acts pretransitively on `α` if for any `x y` there is `g` such that `g • x = y`. A transitive action should furthermore have `α` nonempty. -/ @[to_additive] class MulAction.IsPretransitive (M α : Type*) [SMul M α] : Prop where /-- There is `g` such that `g • x = y`. -/ exists_smul_eq : ∀ x y : α, ∃ g : M, g • x = y namespace MulAction variable (M) [SMul M α] [IsPretransitive M α] @[to_additive] lemma exists_smul_eq (x y : α) : ∃ m : M, m • x = y := IsPretransitive.exists_smul_eq x y @[to_additive] lemma surjective_smul (x : α) : Surjective fun c : M ↦ c • x := exists_smul_eq M x /-- The regular action of a group on itself is transitive. -/ @[to_additive "The regular action of a group on itself is transitive."] instance Regular.isPretransitive [Group G] : IsPretransitive G G := ⟨fun x y ↦ ⟨y * x⁻¹, inv_mul_cancel_right _ _⟩⟩ end MulAction /-! ### Scalar tower and commuting actions -/ /-- A typeclass mixin saying that two additive actions on the same space commute. -/ class VAddCommClass (M N α : Type*) [VAdd M α] [VAdd N α] : Prop where /-- `+ᵥ` is left commutative -/ vadd_comm : ∀ (m : M) (n : N) (a : α), m +ᵥ (n +ᵥ a) = n +ᵥ (m +ᵥ a) /-- A typeclass mixin saying that two multiplicative actions on the same space commute. -/ @[to_additive] class SMulCommClass (M N α : Type*) [SMul M α] [SMul N α] : Prop where /-- `•` is left commutative -/ smul_comm : ∀ (m : M) (n : N) (a : α), m • n • a = n • m • a export MulAction (mul_smul) export AddAction (add_vadd) export SMulCommClass (smul_comm) export VAddCommClass (vadd_comm) library_note "bundled maps over different rings"/-- Frequently, we find ourselves wanting to express a bilinear map `M →ₗ[R] N →ₗ[R] P` or an equivalence between maps `(M →ₗ[R] N) ≃ₗ[R] (M' →ₗ[R] N')` where the maps have an associated ring `R`. Unfortunately, using definitions like these requires that `R` satisfy `CommSemiring R`, and not just `Semiring R`. Using `M →ₗ[R] N →+ P` and `(M →ₗ[R] N) ≃+ (M' →ₗ[R] N')` avoids this problem, but throws away structure that is useful for when we _do_ have a commutative (semi)ring. To avoid making this compromise, we instead state these definitions as `M →ₗ[R] N →ₗ[S] P` or `(M →ₗ[R] N) ≃ₗ[S] (M' →ₗ[R] N')` and require `SMulCommClass S R` on the appropriate modules. When the caller has `CommSemiring R`, they can set `S = R` and `smulCommClass_self` will populate the instance. If the caller only has `Semiring R` they can still set either `R = ℕ` or `S = ℕ`, and `AddCommMonoid.nat_smulCommClass` or `AddCommMonoid.nat_smulCommClass'` will populate the typeclass, which is still sufficient to recover a `≃+` or `→+` structure. An example of where this is used is `LinearMap.prod_equiv`. -/ /-- Commutativity of actions is a symmetric relation. This lemma can't be an instance because this would cause a loop in the instance search graph. -/ @[to_additive] lemma SMulCommClass.symm (M N α : Type*) [SMul M α] [SMul N α] [SMulCommClass M N α] : SMulCommClass N M α where smul_comm a' a b := (smul_comm a a' b).symm /-- Commutativity of additive actions is a symmetric relation. This lemma can't be an instance because this would cause a loop in the instance search graph. -/ add_decl_doc VAddCommClass.symm @[to_additive] lemma Function.Injective.smulCommClass [SMul M α] [SMul N α] [SMul M β] [SMul N β] [SMulCommClass M N β] {f : α → β} (hf : Injective f) (h₁ : ∀ (c : M) x, f (c • x) = c • f x) (h₂ : ∀ (c : N) x, f (c • x) = c • f x) : SMulCommClass M N α where smul_comm c₁ c₂ x := hf <| by simp only [h₁, h₂, smul_comm c₁ c₂ (f x)] @[to_additive] lemma Function.Surjective.smulCommClass [SMul M α] [SMul N α] [SMul M β] [SMul N β] [SMulCommClass M N α] {f : α → β} (hf : Surjective f) (h₁ : ∀ (c : M) x, f (c • x) = c • f x) (h₂ : ∀ (c : N) x, f (c • x) = c • f x) : SMulCommClass M N β where smul_comm c₁ c₂ := hf.forall.2 fun x ↦ by simp only [← h₁, ← h₂, smul_comm c₁ c₂ x] @[to_additive] instance smulCommClass_self (M α : Type*) [CommMonoid M] [MulAction M α] : SMulCommClass M M α where smul_comm a a' b := by rw [← mul_smul, mul_comm, mul_smul] /-- An instance of `VAddAssocClass M N α` states that the additive action of `M` on `α` is determined by the additive actions of `M` on `N` and `N` on `α`. -/ class VAddAssocClass (M N α : Type*) [VAdd M N] [VAdd N α] [VAdd M α] : Prop where /-- Associativity of `+ᵥ` -/ vadd_assoc : ∀ (x : M) (y : N) (z : α), x +ᵥ y +ᵥ z = x +ᵥ (y +ᵥ z) /-- An instance of `IsScalarTower M N α` states that the multiplicative action of `M` on `α` is determined by the multiplicative actions of `M` on `N` and `N` on `α`. -/ @[to_additive VAddAssocClass] -- TODO auto-translating class IsScalarTower (M N α : Type*) [SMul M N] [SMul N α] [SMul M α] : Prop where /-- Associativity of `•` -/ smul_assoc : ∀ (x : M) (y : N) (z : α), (x • y) • z = x • y • z @[to_additive (attr := simp)] lemma smul_assoc {M N} [SMul M N] [SMul N α] [SMul M α] [IsScalarTower M N α] (x : M) (y : N) (z : α) : (x • y) • z = x • y • z := IsScalarTower.smul_assoc x y z @[to_additive] instance Semigroup.isScalarTower [Semigroup α] : IsScalarTower α α α := ⟨mul_assoc⟩ /-- A typeclass indicating that the right (aka `AddOpposite`) and left actions by `M` on `α` are equal, that is that `M` acts centrally on `α`. This can be thought of as a version of commutativity for `+ᵥ`. -/ class IsCentralVAdd (M α : Type*) [VAdd M α] [VAdd Mᵃᵒᵖ α] : Prop where /-- The right and left actions of `M` on `α` are equal. -/ op_vadd_eq_vadd : ∀ (m : M) (a : α), AddOpposite.op m +ᵥ a = m +ᵥ a /-- A typeclass indicating that the right (aka `MulOpposite`) and left actions by `M` on `α` are equal, that is that `M` acts centrally on `α`. This can be thought of as a version of commutativity for `•`. -/ @[to_additive] class IsCentralScalar (M α : Type*) [SMul M α] [SMul Mᵐᵒᵖ α] : Prop where /-- The right and left actions of `M` on `α` are equal. -/ op_smul_eq_smul : ∀ (m : M) (a : α), MulOpposite.op m • a = m • a @[to_additive] lemma IsCentralScalar.unop_smul_eq_smul {M α : Type*} [SMul M α] [SMul Mᵐᵒᵖ α] [IsCentralScalar M α] (m : Mᵐᵒᵖ) (a : α) : MulOpposite.unop m • a = m • a := by induction m; exact (IsCentralScalar.op_smul_eq_smul _ a).symm export IsCentralVAdd (op_vadd_eq_vadd unop_vadd_eq_vadd) export IsCentralScalar (op_smul_eq_smul unop_smul_eq_smul) attribute [simp] IsCentralScalar.op_smul_eq_smul -- these instances are very low priority, as there is usually a faster way to find these instances @[to_additive] instance (priority := 50) SMulCommClass.op_left [SMul M α] [SMul Mᵐᵒᵖ α] [IsCentralScalar M α] [SMul N α] [SMulCommClass M N α] : SMulCommClass Mᵐᵒᵖ N α := ⟨fun m n a ↦ by rw [← unop_smul_eq_smul m (n • a), ← unop_smul_eq_smul m a, smul_comm]⟩ @[to_additive] instance (priority := 50) SMulCommClass.op_right [SMul M α] [SMul N α] [SMul Nᵐᵒᵖ α] [IsCentralScalar N α] [SMulCommClass M N α] : SMulCommClass M Nᵐᵒᵖ α := ⟨fun m n a ↦ by rw [← unop_smul_eq_smul n (m • a), ← unop_smul_eq_smul n a, smul_comm]⟩ @[to_additive] instance (priority := 50) IsScalarTower.op_left [SMul M α] [SMul Mᵐᵒᵖ α] [IsCentralScalar M α] [SMul M N] [SMul Mᵐᵒᵖ N] [IsCentralScalar M N] [SMul N α] [IsScalarTower M N α] : IsScalarTower Mᵐᵒᵖ N α where smul_assoc m n a := by rw [← unop_smul_eq_smul m (n • a), ← unop_smul_eq_smul m n, smul_assoc] @[to_additive] instance (priority := 50) IsScalarTower.op_right [SMul M α] [SMul M N] [SMul N α] [SMul Nᵐᵒᵖ α] [IsCentralScalar N α] [IsScalarTower M N α] : IsScalarTower M Nᵐᵒᵖ α where smul_assoc m n a := by rw [← unop_smul_eq_smul n a, ← unop_smul_eq_smul (m • n) a, MulOpposite.unop_smul, smul_assoc] namespace SMul variable [SMul M α] /-- Auxiliary definition for `SMul.comp`, `MulAction.compHom`, `DistribMulAction.compHom`, `Module.compHom`, etc. -/ @[to_additive (attr := simp) " Auxiliary definition for `VAdd.comp`, `AddAction.compHom`, etc. "] def comp.smul (g : N → M) (n : N) (a : α) : α := g n • a variable (α) /-- An action of `M` on `α` and a function `N → M` induces an action of `N` on `α`. -/ -- See note [reducible non-instances] -- Since this is reducible, we make sure to go via -- `SMul.comp.smul` to prevent typeclass inference unfolding too far @[to_additive (attr := reducible) "An additive action of `M` on `α` and a function `N → M` induces an additive action of `N` on `α`."] def comp (g : N → M) : SMul N α where smul := SMul.comp.smul g variable {α} /-- Given a tower of scalar actions `M → α → β`, if we use `SMul.comp` to pull back both of `M`'s actions by a map `g : N → M`, then we obtain a new tower of scalar actions `N → α → β`. This cannot be an instance because it can cause infinite loops whenever the `SMul` arguments are still metavariables. -/ @[to_additive "Given a tower of additive actions `M → α → β`, if we use `SMul.comp` to pull back both of `M`'s actions by a map `g : N → M`, then we obtain a new tower of scalar actions `N → α → β`. This cannot be an instance because it can cause infinite loops whenever the `SMul` arguments are still metavariables."] lemma comp.isScalarTower [SMul M β] [SMul α β] [IsScalarTower M α β] (g : N → M) : by haveI := comp α g; haveI := comp β g; exact IsScalarTower N α β where __ := comp α g __ := comp β g smul_assoc n := smul_assoc (g n) /-- This cannot be an instance because it can cause infinite loops whenever the `SMul` arguments are still metavariables. -/ @[to_additive "This cannot be an instance because it can cause infinite loops whenever the `VAdd` arguments are still metavariables."] lemma comp.smulCommClass [SMul β α] [SMulCommClass M β α] (g : N → M) : haveI := comp α g SMulCommClass N β α where __ := comp α g smul_comm n := smul_comm (g n) /-- This cannot be an instance because it can cause infinite loops whenever the `SMul` arguments are still metavariables. -/ @[to_additive "This cannot be an instance because it can cause infinite loops whenever the `VAdd` arguments are still metavariables."] lemma comp.smulCommClass' [SMul β α] [SMulCommClass β M α] (g : N → M) : haveI := comp α g SMulCommClass β N α where __ := comp α g smul_comm _ n := smul_comm _ (g n) end SMul section /-- Note that the `SMulCommClass α β β` typeclass argument is usually satisfied by `Algebra α β`. -/ @[to_additive] -- Porting note: nolint to_additive_doc lemma mul_smul_comm [Mul β] [SMul α β] [SMulCommClass α β β] (s : α) (x y : β) : x * s • y = s • (x * y) := (smul_comm s x y).symm /-- Note that the `IsScalarTower α β β` typeclass argument is usually satisfied by `Algebra α β`. -/ @[to_additive] -- Porting note: nolint to_additive_doc lemma smul_mul_assoc [Mul β] [SMul α β] [IsScalarTower α β β] (r : α) (x y : β) : r • x * y = r • (x * y) := smul_assoc r x y /-- Note that the `IsScalarTower α β β` typeclass argument is usually satisfied by `Algebra α β`. -/ @[to_additive] lemma smul_div_assoc [DivInvMonoid β] [SMul α β] [IsScalarTower α β β] (r : α) (x y : β) : r • x / y = r • (x / y) := by simp [div_eq_mul_inv, smul_mul_assoc] @[to_additive] lemma smul_smul_smul_comm [SMul α β] [SMul α γ] [SMul β δ] [SMul α δ] [SMul γ δ] [IsScalarTower α β δ] [IsScalarTower α γ δ] [SMulCommClass β γ δ] (a : α) (b : β) (c : γ) (d : δ) : (a • b) • c • d = (a • c) • b • d := by rw [smul_assoc, smul_assoc, smul_comm b] variable [SMul M α] @[to_additive] lemma Commute.smul_right [Mul α] [SMulCommClass M α α] [IsScalarTower M α α] {a b : α} (h : Commute a b) (r : M) : Commute a (r • b) := (mul_smul_comm _ _ _).trans ((congr_arg _ h).trans <| (smul_mul_assoc _ _ _).symm) @[to_additive] lemma Commute.smul_left [Mul α] [SMulCommClass M α α] [IsScalarTower M α α] {a b : α} (h : Commute a b) (r : M) : Commute (r • a) b := (h.symm.smul_right r).symm end section variable [Monoid M] [MulAction M α] @[to_additive] lemma smul_smul (a₁ a₂ : M) (b : α) : a₁ • a₂ • b = (a₁ * a₂) • b := (mul_smul _ _ _).symm variable (M) @[to_additive (attr := simp)] lemma one_smul (b : α) : (1 : M) • b = b := MulAction.one_smul _ /-- `SMul` version of `one_mul_eq_id` -/ @[to_additive "`VAdd` version of `zero_add_eq_id`"] lemma one_smul_eq_id : (((1 : M) • ·) : α → α) = id := funext <| one_smul _ /-- `SMul` version of `comp_mul_left` -/ @[to_additive "`VAdd` version of `comp_add_left`"] lemma comp_smul_left (a₁ a₂ : M) : (a₁ • ·) ∘ (a₂ • ·) = (((a₁ * a₂) • ·) : α → α) := funext fun _ ↦ (mul_smul _ _ _).symm variable {M} /-- Pullback a multiplicative action along an injective map respecting `•`. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "Pullback an additive action along an injective map respecting `+ᵥ`."] protected def Function.Injective.mulAction [SMul M β] (f : β → α) (hf : Injective f) (smul : ∀ (c : M) (x), f (c • x) = c • f x) : MulAction M β where smul := (· • ·) one_smul x := hf <| (smul _ _).trans <| one_smul _ (f x) mul_smul c₁ c₂ x := hf <| by simp only [smul, mul_smul] /-- Pushforward a multiplicative action along a surjective map respecting `•`. See note [reducible non-instances]. -/ @[to_additive (attr := reducible) "Pushforward an additive action along a surjective map respecting `+ᵥ`."] protected def Function.Surjective.mulAction [SMul M β] (f : α → β) (hf : Surjective f) (smul : ∀ (c : M) (x), f (c • x) = c • f x) : MulAction M β where smul := (· • ·) one_smul := by simp [hf.forall, ← smul] mul_smul := by simp [hf.forall, ← smul, mul_smul] /-- Push forward the action of `R` on `M` along a compatible surjective map `f : R →* S`. See also `Function.Surjective.distribMulActionLeft` and `Function.Surjective.moduleLeft`. -/ @[to_additive (attr := reducible) "Push forward the action of `R` on `M` along a compatible surjective map `f : R →+ S`."] def Function.Surjective.mulActionLeft {R S M : Type*} [Monoid R] [MulAction R M] [Monoid S] [SMul S M] (f : R →* S) (hf : Surjective f) (hsmul : ∀ (c) (x : M), f c • x = c • x) : MulAction S M where smul := (· • ·) one_smul b := by rw [← f.map_one, hsmul, one_smul] mul_smul := hf.forall₂.mpr fun a b x ↦ by simp only [← f.map_mul, hsmul, mul_smul] section variable (M) /-- The regular action of a monoid on itself by left multiplication. This is promoted to a module by `Semiring.toModule`. -/ -- see Note [lower instance priority] @[to_additive "The regular action of a monoid on itself by left addition. This is promoted to an `AddTorsor` by `addGroup_is_addTorsor`."] instance (priority := 910) Monoid.toMulAction : MulAction M M where smul := (· * ·) one_smul := one_mul mul_smul := mul_assoc @[to_additive] instance IsScalarTower.left : IsScalarTower M M α where smul_assoc x y z := mul_smul x y z variable {M} /-- Note that the `IsScalarTower M α α` and `SMulCommClass M α α` typeclass arguments are usually satisfied by `Algebra M α`. -/ @[to_additive] -- Porting note: nolint to_additive_doc lemma smul_mul_smul [Mul α] (r s : M) (x y : α) [IsScalarTower M α α] [SMulCommClass M α α] : r • x * s • y = (r * s) • (x * y) := by rw [smul_mul_assoc, mul_smul_comm, ← smul_assoc, smul_eq_mul] section Monoid variable [Monoid N] [MulAction M N] [IsScalarTower M N N] [SMulCommClass M N N] lemma smul_pow (r : M) (x : N) : ∀ n, (r • x) ^ n = r ^ n • x ^ n | 0 => by simp | n + 1 => by rw [pow_succ', smul_pow _ _ n, smul_mul_smul, ← pow_succ', ← pow_succ'] end Monoid section Group variable [Group G] [MulAction G α] {g : G} {a b : α} @[to_additive (attr := simp)] lemma inv_smul_smul (g : G) (a : α) : g⁻¹ • g • a = a := by rw [smul_smul, mul_left_inv, one_smul] @[to_additive (attr := simp)] lemma smul_inv_smul (g : G) (a : α) : g • g⁻¹ • a = a := by rw [smul_smul, mul_right_inv, one_smul] @[to_additive] lemma inv_smul_eq_iff : g⁻¹ • a = b ↔ a = g • b := ⟨fun h ↦ by rw [← h, smul_inv_smul], fun h ↦ by rw [h, inv_smul_smul]⟩ @[to_additive] lemma eq_inv_smul_iff : a = g⁻¹ • b ↔ g • a = b := ⟨fun h ↦ by rw [h, smul_inv_smul], fun h ↦ by rw [← h, inv_smul_smul]⟩ section Mul variable [Mul H] [MulAction G H] [SMulCommClass G H H] [IsScalarTower G H H] {g : G} {a b : H} @[simp] lemma Commute.smul_right_iff : Commute a (g • b) ↔ Commute a b := ⟨fun h ↦ inv_smul_smul g b ▸ h.smul_right g⁻¹, fun h ↦ h.smul_right g⟩ @[simp] lemma Commute.smul_left_iff : Commute (g • a) b ↔ Commute a b := by rw [Commute.symm_iff, Commute.smul_right_iff, Commute.symm_iff] end Mul variable [Group H] [MulAction G H] [SMulCommClass G H H] [IsScalarTower G H H] lemma smul_inv (g : G) (a : H) : (g • a)⁻¹ = g⁻¹ • a⁻¹ := inv_eq_of_mul_eq_one_right $ by rw [smul_mul_smul, mul_right_inv, mul_right_inv, one_smul] lemma smul_zpow (g : G) (a : H) (n : ℤ) : (g • a) ^ n = g ^ n • a ^ n := by cases n <;> simp [smul_pow, smul_inv] end Group end lemma SMulCommClass.of_commMonoid (A B G : Type*) [CommMonoid G] [SMul A G] [SMul B G] [IsScalarTower A G G] [IsScalarTower B G G] : SMulCommClass A B G where smul_comm r s x := by rw [← one_smul G (s • x), ← smul_assoc, ← one_smul G x, ← smul_assoc s 1 x, smul_comm, smul_assoc, one_smul, smul_assoc, one_smul] namespace MulAction variable (M α) in /-- Embedding of `α` into functions `M → α` induced by a multiplicative action of `M` on `α`. -/ @[to_additive "Embedding of `α` into functions `M → α` induced by an additive action of `M` on `α`."] def toFun : α ↪ M → α := ⟨fun y x ↦ x • y, fun y₁ y₂ H ↦ one_smul M y₁ ▸ one_smul M y₂ ▸ by convert congr_fun H 1⟩ @[to_additive (attr := simp)] lemma toFun_apply (x : M) (y : α) : MulAction.toFun M α y x = x • y := rfl variable (α) /-- A multiplicative action of `M` on `α` and a monoid homomorphism `N → M` induce a multiplicative action of `N` on `α`. See note [reducible non-instances]. -/ @[to_additive (attr := reducible)] def compHom [Monoid N] (g : N →* M) : MulAction N α where smul := SMul.comp.smul g -- Porting note: was `by simp [g.map_one, MulAction.one_smul]` one_smul _ := by simpa [(· • ·)] using MulAction.one_smul .. -- Porting note: was `by simp [g.map_mul, MulAction.mul_smul]` mul_smul _ _ _ := by simpa [(· • ·)] using MulAction.mul_smul .. /-- An additive action of `M` on `α` and an additive monoid homomorphism `N → M` induce an additive action of `N` on `α`. See note [reducible non-instances]. -/ add_decl_doc AddAction.compHom @[to_additive] lemma compHom_smul_def {E F G : Type*} [Monoid E] [Monoid F] [MulAction F G] (f : E →* F) (a : E) (x : G) : letI : MulAction E G := MulAction.compHom _ f a • x = (f a) • x := rfl /-- If an action is transitive, then composing this action with a surjective homomorphism gives again a transitive action. -/ @[to_additive] lemma isPretransitive_compHom {E F G : Type*} [Monoid E] [Monoid F] [MulAction F G] [IsPretransitive F G] {f : E →* F} (hf : Surjective f) : letI : MulAction E G := MulAction.compHom _ f IsPretransitive E G := by let _ : MulAction E G := MulAction.compHom _ f refine ⟨fun x y ↦ ?_⟩ obtain ⟨m, rfl⟩ : ∃ m : F, m • x = y := exists_smul_eq F x y obtain ⟨e, rfl⟩ : ∃ e, f e = m := hf m exact ⟨e, rfl⟩ @[to_additive] lemma IsPretransitive.of_smul_eq {M N α : Type*} [SMul M α] [SMul N α] [IsPretransitive M α] (f : M → N) (hf : ∀ {c : M} {x : α}, f c • x = c • x) : IsPretransitive N α where exists_smul_eq x y := (exists_smul_eq x y).elim fun m h ↦ ⟨f m, hf.trans h⟩ @[to_additive] lemma IsPretransitive.of_compHom {M N α : Type*} [Monoid M] [Monoid N] [MulAction N α] (f : M →* N) [h : letI := compHom α f; IsPretransitive M α] : IsPretransitive N α := letI := compHom α f; h.of_smul_eq f rfl end MulAction end section CompatibleScalar @[to_additive] lemma smul_one_smul {M} (N) [Monoid N] [SMul M N] [MulAction N α] [SMul M α] [IsScalarTower M N α] (x : M) (y : α) : (x • (1 : N)) • y = x • y := by rw [smul_assoc, one_smul] @[to_additive] lemma MulAction.IsPretransitive.of_isScalarTower (M : Type*) {N α : Type*} [Monoid N] [SMul M N] [MulAction N α] [SMul M α] [IsScalarTower M N α] [IsPretransitive M α] : IsPretransitive N α := of_smul_eq (fun x : M ↦ x • 1) (smul_one_smul N _ _) @[to_additive (attr := simp)] lemma smul_one_mul {M N} [MulOneClass N] [SMul M N] [IsScalarTower M N N] (x : M) (y : N) : x • (1 : N) * y = x • y := by rw [smul_mul_assoc, one_mul] @[to_additive (attr := simp)] lemma mul_smul_one {M N} [MulOneClass N] [SMul M N] [SMulCommClass M N N] (x : M) (y : N) : y * x • (1 : N) = x • y := by rw [← smul_eq_mul, ← smul_comm, smul_eq_mul, mul_one] @[to_additive] lemma IsScalarTower.of_smul_one_mul {M N} [Monoid N] [SMul M N] (h : ∀ (x : M) (y : N), x • (1 : N) * y = x • y) : IsScalarTower M N N := ⟨fun x y z ↦ by rw [← h, smul_eq_mul, mul_assoc, h, smul_eq_mul]⟩ @[to_additive] lemma SMulCommClass.of_mul_smul_one {M N} [Monoid N] [SMul M N] (H : ∀ (x : M) (y : N), y * x • (1 : N) = x • y) : SMulCommClass M N N := ⟨fun x y z ↦ by rw [← H x z, smul_eq_mul, ← H, smul_eq_mul, mul_assoc]⟩ /-- If the multiplicative action of `M` on `N` is compatible with multiplication on `N`, then `fun x ↦ x • 1` is a monoid homomorphism from `M` to `N`. -/ @[to_additive (attr := simps) "If the additive action of `M` on `N` is compatible with addition on `N`, then `fun x ↦ x +ᵥ 0` is an additive monoid homomorphism from `M` to `N`."] def MonoidHom.smulOneHom {M N} [Monoid M] [MulOneClass N] [MulAction M N] [IsScalarTower M N N] : M →* N where toFun x := x • (1 : N) map_one' := one_smul _ _ map_mul' x y := by rw [smul_one_mul, smul_smul] /-- A monoid homomorphism between two monoids M and N can be equivalently specified by a multiplicative action of M on N that is compatible with the multiplication on N. -/ @[to_additive "A monoid homomorphism between two additive monoids M and N can be equivalently specified by an additive action of M on N that is compatible with the addition on N."] def monoidHomEquivMulActionIsScalarTower (M N) [Monoid M] [Monoid N] : (M →* N) ≃ {_inst : MulAction M N // IsScalarTower M N N} where toFun f := ⟨MulAction.compHom N f, SMul.comp.isScalarTower _⟩ invFun := fun ⟨_, _⟩ ↦ MonoidHom.smulOneHom left_inv f := MonoidHom.ext fun m ↦ mul_one (f m) right_inv := fun ⟨_, _⟩ ↦ Subtype.ext <| MulAction.ext <| funext₂ <| smul_one_smul N end CompatibleScalar variable (α) /-- The monoid of endomorphisms. Note that this is generalized by `CategoryTheory.End` to categories other than `Type u`. -/ protected def Function.End := α → α instance : Monoid (Function.End α) where one := id mul := (· ∘ ·) mul_assoc f g h := rfl mul_one f := rfl one_mul f := rfl npow n f := f^[n] npow_succ n f := Function.iterate_succ _ _ instance : Inhabited (Function.End α) := ⟨1⟩ variable {α} /-- The tautological action by `Function.End α` on `α`. This is generalized to bundled endomorphisms by: * `Equiv.Perm.applyMulAction` * `AddMonoid.End.applyDistribMulAction` * `AddMonoid.End.applyModule` * `AddAut.applyDistribMulAction` * `MulAut.applyMulDistribMulAction` * `LinearEquiv.applyDistribMulAction` * `LinearMap.applyModule` * `RingHom.applyMulSemiringAction` * `RingAut.applyMulSemiringAction` * `AlgEquiv.applyMulSemiringAction` -/ instance Function.End.applyMulAction : MulAction (Function.End α) α where smul := (· <| ·) one_smul _ := rfl mul_smul _ _ _ := rfl @[simp] lemma Function.End.smul_def (f : Function.End α) (a : α) : f • a = f a := rfl --TODO - This statement should be somethting like `toFun (f * g) = toFun f ∘ toFun g` lemma Function.End.mul_def (f g : Function.End α) : (f * g) = f ∘ g := rfl --TODO - This statement should be somethting like `toFun 1 = id` lemma Function.End.one_def : (1 : Function.End α) = id := rfl /-- `Function.End.applyMulAction` is faithful. -/ instance Function.End.apply_FaithfulSMul : FaithfulSMul (Function.End α) α := ⟨fun {_ _} ↦ funext⟩ /-- The monoid hom representing a monoid action. When `M` is a group, see `MulAction.toPermHom`. -/ def MulAction.toEndHom [Monoid M] [MulAction M α] : M →* Function.End α where toFun := (· • ·) map_one' := funext (one_smul M) map_mul' x y := funext (mul_smul x y) /-- The monoid action induced by a monoid hom to `Function.End α` See note [reducible non-instances]. -/ abbrev MulAction.ofEndHom [Monoid M] (f : M →* Function.End α) : MulAction M α := MulAction.compHom α f /-! ### `Additive`, `Multiplicative` -/ section open Additive Multiplicative instance Additive.vadd [SMul α β] : VAdd (Additive α) β where vadd a := (toMul a • ·) instance Multiplicative.smul [VAdd α β] : SMul (Multiplicative α) β where smul a := (toAdd a +ᵥ ·) @[simp] lemma toMul_smul [SMul α β] (a) (b : β) : (toMul a : α) • b = a +ᵥ b := rfl @[simp] lemma ofMul_vadd [SMul α β] (a : α) (b : β) : ofMul a +ᵥ b = a • b := rfl @[simp] lemma toAdd_vadd [VAdd α β] (a) (b : β) : (toAdd a : α) +ᵥ b = a • b := rfl @[simp] lemma ofAdd_smul [VAdd α β] (a : α) (b : β) : ofAdd a • b = a +ᵥ b := rfl -- Porting note: I don't know why `one_smul` can do without an explicit α and `mul_smul` can't. instance Additive.addAction [Monoid α] [MulAction α β] : AddAction (Additive α) β where zero_vadd := MulAction.one_smul add_vadd := MulAction.mul_smul (α := α) instance Multiplicative.mulAction [AddMonoid α] [AddAction α β] : MulAction (Multiplicative α) β where one_smul := AddAction.zero_vadd mul_smul := AddAction.add_vadd (G := α) instance Additive.addAction_isPretransitive [Monoid α] [MulAction α β] [MulAction.IsPretransitive α β] : AddAction.IsPretransitive (Additive α) β := ⟨@MulAction.exists_smul_eq α _ _ _⟩ instance Multiplicative.mulAction_isPretransitive [AddMonoid α] [AddAction α β] [AddAction.IsPretransitive α β] : MulAction.IsPretransitive (Multiplicative α) β := ⟨@AddAction.exists_vadd_eq α _ _ _⟩ instance Additive.vaddCommClass [SMul α γ] [SMul β γ] [SMulCommClass α β γ] : VAddCommClass (Additive α) (Additive β) γ := ⟨@smul_comm α β _ _ _ _⟩ instance Multiplicative.smulCommClass [VAdd α γ] [VAdd β γ] [VAddCommClass α β γ] : SMulCommClass (Multiplicative α) (Multiplicative β) γ := ⟨@vadd_comm α β _ _ _ _⟩ end /-- The tautological additive action by `Additive (Function.End α)` on `α`. -/ instance AddAction.functionEnd : AddAction (Additive (Function.End α)) α := inferInstance /-- The additive monoid hom representing an additive monoid action. When `M` is a group, see `AddAction.toPermHom`. -/ def AddAction.toEndHom [AddMonoid M] [AddAction M α] : M →+ Additive (Function.End α) := MonoidHom.toAdditive'' MulAction.toEndHom /-- The additive action induced by a hom to `Additive (Function.End α)` See note [reducible non-instances]. -/ abbrev AddAction.ofEndHom [AddMonoid M] (f : M →+ Additive (Function.End α)) : AddAction M α := AddAction.compHom α f
Algebra\Group\Action\Opposite.lean
/- Copyright (c) 2020 Eric Wieser. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Eric Wieser -/ import Mathlib.Algebra.Group.Action.Defs import Mathlib.Algebra.Group.Opposite /-! # Scalar actions on and by `Mᵐᵒᵖ` This file defines the actions on the opposite type `SMul R Mᵐᵒᵖ`, and actions by the opposite type, `SMul Rᵐᵒᵖ M`. Note that `MulOpposite.smul` is provided in an earlier file as it is needed to provide the `AddMonoid.nsmul` and `AddCommGroup.zsmul` fields. ## Notation With `open scoped RightActions`, this provides: * `r •> m` as an alias for `r • m` * `m <• r` as an alias for `MulOpposite.op r • m` * `v +ᵥ> p` as an alias for `v +ᵥ p` * `p <+ᵥ v` as an alias for `AddOpposite.op v +ᵥ p` -/ assert_not_exists MonoidWithZero variable {R M N α : Type*} /-! ### Actions _on_ the opposite type Actions on the opposite type just act on the underlying type. -/ namespace MulOpposite @[to_additive] instance instMulAction [Monoid M] [MulAction M α] : MulAction M αᵐᵒᵖ where one_smul _ := unop_injective <| one_smul _ _ mul_smul _ _ _ := unop_injective <| mul_smul _ _ _ @[to_additive] instance instIsScalarTower [SMul M N] [SMul M α] [SMul N α] [IsScalarTower M N α] : IsScalarTower M N αᵐᵒᵖ where smul_assoc _ _ _ := unop_injective <| smul_assoc _ _ _ @[to_additive] instance instSMulCommClass [SMul M α] [SMul N α] [SMulCommClass M N α] : SMulCommClass M N αᵐᵒᵖ where smul_comm _ _ _ := unop_injective <| smul_comm _ _ _ @[to_additive] instance instIsCentralScalar [SMul M α] [SMul Mᵐᵒᵖ α] [IsCentralScalar M α] : IsCentralScalar M αᵐᵒᵖ where op_smul_eq_smul _ _ := unop_injective <| op_smul_eq_smul _ _ @[to_additive] lemma op_smul_eq_op_smul_op [SMul M α] [SMul Mᵐᵒᵖ α] [IsCentralScalar M α] (r : M) (a : α) : op (r • a) = op r • op a := (op_smul_eq_smul r (op a)).symm @[to_additive] lemma unop_smul_eq_unop_smul_unop [SMul M α] [SMul Mᵐᵒᵖ α] [IsCentralScalar M α] (r : Mᵐᵒᵖ) (a : αᵐᵒᵖ) : unop (r • a) = unop r • unop a := (unop_smul_eq_smul r (unop a)).symm end MulOpposite /-! ### Right actions In this section we establish `SMul αᵐᵒᵖ β` as the canonical spelling of right scalar multiplication of `β` by `α`, and provide convenient notations. -/ namespace RightActions /-- With `open scoped RightActions`, an alternative symbol for left actions, `r • m`. In lemma names this is still called `smul`. -/ scoped notation3:74 r:75 " •> " m:74 => r • m /-- With `open scoped RightActions`, a shorthand for right actions, `op r • m`. In lemma names this is still called `op_smul`. -/ scoped notation3:73 m:73 " <• " r:74 => MulOpposite.op r • m /-- With `open scoped RightActions`, an alternative symbol for left actions, `r • m`. In lemma names this is still called `vadd`. -/ scoped notation3:74 r:75 " +ᵥ> " m:74 => r +ᵥ m /-- With `open scoped RightActions`, a shorthand for right actions, `op r +ᵥ m`. In lemma names this is still called `op_vadd`. -/ scoped notation3:73 m:73 " <+ᵥ " r:74 => AddOpposite.op r +ᵥ m section examples variable {α β : Type*} [SMul α β] [SMul αᵐᵒᵖ β] [VAdd α β] [VAdd αᵃᵒᵖ β] {a a₁ a₂ a₃ a₄ : α} {b : β} -- Left and right actions are just notation around the general `•` and `+ᵥ` notations example : a •> b = a • b := rfl example : b <• a = MulOpposite.op a • b := rfl example : a +ᵥ> b = a +ᵥ b := rfl example : b <+ᵥ a = AddOpposite.op a +ᵥ b := rfl -- Left actions right-associate, right actions left-associate example : a₁ •> a₂ •> b = a₁ •> (a₂ •> b) := rfl example : b <• a₂ <• a₁ = (b <• a₂) <• a₁ := rfl example : a₁ +ᵥ> a₂ +ᵥ> b = a₁ +ᵥ> (a₂ +ᵥ> b) := rfl example : b <+ᵥ a₂ <+ᵥ a₁ = (b <+ᵥ a₂) <+ᵥ a₁ := rfl -- When left and right actions coexist, they associate to the left example : a₁ •> b <• a₂ = (a₁ •> b) <• a₂ := rfl example : a₁ •> a₂ •> b <• a₃ <• a₄ = ((a₁ •> (a₂ •> b)) <• a₃) <• a₄ := rfl example : a₁ +ᵥ> b <+ᵥ a₂ = (a₁ +ᵥ> b) <+ᵥ a₂ := rfl example : a₁ +ᵥ> a₂ +ᵥ> b <+ᵥ a₃ <+ᵥ a₄ = ((a₁ +ᵥ> (a₂ +ᵥ> b)) <+ᵥ a₃) <+ᵥ a₄ := rfl end examples end RightActions section variable {α β : Type*} [Monoid α] [MulAction αᵐᵒᵖ β] open scoped RightActions @[to_additive] lemma op_smul_op_smul (b : β) (a₁ a₂ : α) : b <• a₁ <• a₂ = b <• (a₁ * a₂) := smul_smul _ _ _ @[to_additive] lemma op_smul_mul (b : β) (a₁ a₂ : α) : b <• (a₁ * a₂) = b <• a₁ <• a₂ := mul_smul _ _ _ end /-! ### Actions _by_ the opposite type (right actions) In `Mul.toSMul` in another file, we define the left action `a₁ • a₂ = a₁ * a₂`. For the multiplicative opposite, we define `MulOpposite.op a₁ • a₂ = a₂ * a₁`, with the multiplication reversed. -/ open MulOpposite /-- Like `Mul.toSMul`, but multiplies on the right. See also `Monoid.toOppositeMulAction` and `MonoidWithZero.toOppositeMulActionWithZero`. -/ @[to_additive "Like `Add.toVAdd`, but adds on the right. See also `AddMonoid.toOppositeAddAction`."] instance Mul.toHasOppositeSMul [Mul α] : SMul αᵐᵒᵖ α where smul c x := x * c.unop @[to_additive] lemma op_smul_eq_mul [Mul α] {a a' : α} : op a • a' = a' * a := rfl @[to_additive (attr := simp)] lemma MulOpposite.smul_eq_mul_unop [Mul α] {a : αᵐᵒᵖ} {a' : α} : a • a' = a' * a.unop := rfl /-- The right regular action of a group on itself is transitive. -/ @[to_additive "The right regular action of an additive group on itself is transitive."] instance MulAction.OppositeRegular.isPretransitive {G : Type*} [Group G] : IsPretransitive Gᵐᵒᵖ G := ⟨fun x y => ⟨op (x⁻¹ * y), mul_inv_cancel_left _ _⟩⟩ @[to_additive] instance Semigroup.opposite_smulCommClass [Semigroup α] : SMulCommClass αᵐᵒᵖ α α where smul_comm _ _ _ := mul_assoc _ _ _ @[to_additive] instance Semigroup.opposite_smulCommClass' [Semigroup α] : SMulCommClass α αᵐᵒᵖ α := SMulCommClass.symm _ _ _ @[to_additive] instance CommSemigroup.isCentralScalar [CommSemigroup α] : IsCentralScalar α α where op_smul_eq_smul _ _ := mul_comm _ _ /-- Like `Monoid.toMulAction`, but multiplies on the right. -/ @[to_additive "Like `AddMonoid.toAddAction`, but adds on the right."] instance Monoid.toOppositeMulAction [Monoid α] : MulAction αᵐᵒᵖ α where smul := (· • ·) one_smul := mul_one mul_smul _ _ _ := (mul_assoc _ _ _).symm @[to_additive] instance IsScalarTower.opposite_mid {M N} [Mul N] [SMul M N] [SMulCommClass M N N] : IsScalarTower M Nᵐᵒᵖ N where smul_assoc _ _ _ := mul_smul_comm _ _ _ @[to_additive] instance SMulCommClass.opposite_mid {M N} [Mul N] [SMul M N] [IsScalarTower M N N] : SMulCommClass M Nᵐᵒᵖ N where smul_comm x y z := by induction y using MulOpposite.rec' simp only [smul_mul_assoc, MulOpposite.smul_eq_mul_unop] -- The above instance does not create an unwanted diamond, the two paths to -- `MulAction αᵐᵒᵖ αᵐᵒᵖ` are defeq. example [Monoid α] : Monoid.toMulAction αᵐᵒᵖ = MulOpposite.instMulAction := by with_reducible_and_instances rfl /-- `Monoid.toOppositeMulAction` is faithful on cancellative monoids. -/ @[to_additive "`AddMonoid.toOppositeAddAction` is faithful on cancellative monoids."] instance LeftCancelMonoid.toFaithfulSMul_opposite [LeftCancelMonoid α] : FaithfulSMul αᵐᵒᵖ α where eq_of_smul_eq_smul h := unop_injective <| mul_left_cancel (h 1)
Algebra\Group\Action\Option.lean
/- Copyright (c) 2022 Yaël Dillies. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Yaël Dillies -/ import Mathlib.Algebra.Group.Action.Defs /-! # Option instances for additive and multiplicative actions This file defines instances for additive and multiplicative actions on `Option` type. Scalar multiplication is defined by `a • some b = some (a • b)` and `a • none = none`. ## See also * `Mathlib.Algebra.Group.Action.Pi` * `Mathlib.Algebra.Group.Action.Sigma` * `Mathlib.Algebra.Group.Action.Sum` -/ assert_not_exists MonoidWithZero variable {M N α : Type*} namespace Option section SMul variable [SMul M α] [SMul N α] (a : M) (b : α) (x : Option α) @[to_additive Option.VAdd] instance : SMul M (Option α) := ⟨fun a => Option.map <| (a • ·)⟩ @[to_additive] theorem smul_def : a • x = x.map (a • ·) := rfl @[to_additive (attr := simp)] theorem smul_none : a • (none : Option α) = none := rfl @[to_additive (attr := simp)] theorem smul_some : a • some b = some (a • b) := rfl @[to_additive] instance instIsScalarTowerOfSMul [SMul M N] [IsScalarTower M N α] : IsScalarTower M N (Option α) := ⟨fun a b x => by cases x exacts [rfl, congr_arg some (smul_assoc _ _ _)]⟩ @[to_additive] instance [SMulCommClass M N α] : SMulCommClass M N (Option α) := ⟨fun _ _ => Function.Commute.option_map <| smul_comm _ _⟩ @[to_additive] instance [SMul Mᵐᵒᵖ α] [IsCentralScalar M α] : IsCentralScalar M (Option α) := ⟨fun a x => by cases x exacts [rfl, congr_arg some (op_smul_eq_smul _ _)]⟩ @[to_additive] instance [FaithfulSMul M α] : FaithfulSMul M (Option α) := ⟨fun h => eq_of_smul_eq_smul fun b : α => by injection h (some b)⟩ end SMul instance [Monoid M] [MulAction M α] : MulAction M (Option α) where smul := (· • ·) one_smul b := by cases b exacts [rfl, congr_arg some (one_smul _ _)] mul_smul a₁ a₂ b := by cases b exacts [rfl, congr_arg some (mul_smul _ _ _)] end Option
Algebra\Group\Action\Pi.lean
/- Copyright (c) 2018 Simon Hudon. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Simon Hudon, Patrick Massot -/ import Mathlib.Algebra.Group.Action.Defs import Mathlib.Data.Set.Function /-! # Pi instances for multiplicative actions This file defines instances for `MulAction` and related structures on `Pi` types. ## See also * `Mathlib.Algebra.Group.Action.Option` * `Mathlib.Algebra.Group.Action.Prod` * `Mathlib.Algebra.Group.Action.Sigma` * `Mathlib.Algebra.Group.Action.Sum` -/ assert_not_exists MonoidWithZero variable {ι M N : Type*} {α β γ : ι → Type*} (x y : ∀ i, α i) (i : ι) namespace Pi @[to_additive] instance smul' [∀ i, SMul (α i) (β i)] : SMul (∀ i, α i) (∀ i, β i) where smul s x i := s i • x i @[to_additive (attr := simp)] lemma smul_apply' [∀ i, SMul (α i) (β i)] (s : ∀ i, α i) (x : ∀ i, β i) : (s • x) i = s i • x i := rfl -- Porting note: `to_additive` fails to correctly translate name @[to_additive Pi.vaddAssocClass] instance isScalarTower [SMul M N] [∀ i, SMul N (α i)] [∀ i, SMul M (α i)] [∀ i, IsScalarTower M N (α i)] : IsScalarTower M N (∀ i, α i) where smul_assoc x y z := funext fun i ↦ smul_assoc x y (z i) @[to_additive Pi.vaddAssocClass'] instance isScalarTower' [∀ i, SMul M (α i)] [∀ i, SMul (α i) (β i)] [∀ i, SMul M (β i)] [∀ i, IsScalarTower M (α i) (β i)] : IsScalarTower M (∀ i, α i) (∀ i, β i) where smul_assoc x y z := funext fun i ↦ smul_assoc x (y i) (z i) @[to_additive Pi.vaddAssocClass''] instance isScalarTower'' [∀ i, SMul (α i) (β i)] [∀ i, SMul (β i) (γ i)] [∀ i, SMul (α i) (γ i)] [∀ i, IsScalarTower (α i) (β i) (γ i)] : IsScalarTower (∀ i, α i) (∀ i, β i) (∀ i, γ i) where smul_assoc x y z := funext fun i ↦ smul_assoc (x i) (y i) (z i) @[to_additive] instance smulCommClass [∀ i, SMul M (α i)] [∀ i, SMul N (α i)] [∀ i, SMulCommClass M N (α i)] : SMulCommClass M N (∀ i, α i) where smul_comm x y z := funext fun i ↦ smul_comm x y (z i) @[to_additive] instance smulCommClass' [∀ i, SMul M (β i)] [∀ i, SMul (α i) (β i)] [∀ i, SMulCommClass M (α i) (β i)] : SMulCommClass M (∀ i, α i) (∀ i, β i) := ⟨fun x y z => funext fun i ↦ smul_comm x (y i) (z i)⟩ @[to_additive] instance smulCommClass'' [∀ i, SMul (β i) (γ i)] [∀ i, SMul (α i) (γ i)] [∀ i, SMulCommClass (α i) (β i) (γ i)] : SMulCommClass (∀ i, α i) (∀ i, β i) (∀ i, γ i) where smul_comm x y z := funext fun i ↦ smul_comm (x i) (y i) (z i) @[to_additive] instance isCentralScalar [∀ i, SMul M (α i)] [∀ i, SMul Mᵐᵒᵖ (α i)] [∀ i, IsCentralScalar M (α i)] : IsCentralScalar M (∀ i, α i) where op_smul_eq_smul _ _ := funext fun _ ↦ op_smul_eq_smul _ _ /-- If `α i` has a faithful scalar action for a given `i`, then so does `Π i, α i`. This is not an instance as `i` cannot be inferred. -/ @[to_additive "If `α i` has a faithful additive action for a given `i`, then so does `Π i, α i`. This is not an instance as `i` cannot be inferred"] lemma faithfulSMul_at [∀ i, SMul M (α i)] [∀ i, Nonempty (α i)] (i : ι) [FaithfulSMul M (α i)] : FaithfulSMul M (∀ i, α i) where eq_of_smul_eq_smul h := eq_of_smul_eq_smul fun a : α i => by classical simpa using congr_fun (h <| Function.update (fun j => Classical.choice (‹∀ i, Nonempty (α i)› j)) i a) i @[to_additive] instance faithfulSMul [Nonempty ι] [∀ i, SMul M (α i)] [∀ i, Nonempty (α i)] [∀ i, FaithfulSMul M (α i)] : FaithfulSMul M (∀ i, α i) := let ⟨i⟩ := ‹Nonempty ι› faithfulSMul_at i @[to_additive] instance mulAction (M) {m : Monoid M} [∀ i, MulAction M (α i)] : @MulAction M (∀ i, α i) m where smul := (· • ·) mul_smul _ _ _ := funext fun _ ↦ mul_smul _ _ _ one_smul _ := funext fun _ ↦ one_smul _ _ @[to_additive] instance mulAction' {m : ∀ i, Monoid (α i)} [∀ i, MulAction (α i) (β i)] : @MulAction (∀ i, α i) (∀ i, β i) (@Pi.monoid ι α m) where smul := (· • ·) mul_smul _ _ _ := funext fun _ ↦ mul_smul _ _ _ one_smul _ := funext fun _ ↦ one_smul _ _ end Pi namespace Function /-- Non-dependent version of `Pi.smul`. Lean gets confused by the dependent instance if this is not present. -/ @[to_additive "Non-dependent version of `Pi.vadd`. Lean gets confused by the dependent instance if this is not present."] instance hasSMul {α : Type*} [SMul M α] : SMul M (ι → α) := Pi.instSMul /-- Non-dependent version of `Pi.smulCommClass`. Lean gets confused by the dependent instance if this is not present. -/ @[to_additive "Non-dependent version of `Pi.vaddCommClass`. Lean gets confused by the dependent instance if this is not present."] instance smulCommClass {α : Type*} [SMul M α] [SMul N α] [SMulCommClass M N α] : SMulCommClass M N (ι → α) := Pi.smulCommClass @[to_additive] lemma update_smul [∀ i, SMul M (α i)] [DecidableEq ι] (c : M) (f₁ : ∀ i, α i) (i : ι) (x₁ : α i) : update (c • f₁) i (c • x₁) = c • update f₁ i x₁ := funext fun j => (apply_update (β := α) (fun _ ↦ (c • ·)) f₁ i x₁ j).symm @[to_additive] lemma extend_smul {M α β : Type*} [SMul M β] (r : M) (f : ι → α) (g : ι → β) (e : α → β) : extend f (r • g) (r • e) = r • extend f g e := by funext x classical simp only [extend_def, Pi.smul_apply] split_ifs <;> rfl end Function namespace Set @[to_additive] lemma piecewise_smul [∀ i, SMul M (α i)] (s : Set ι) [∀ i, Decidable (i ∈ s)] (c : M) (f₁ g₁ : ∀ i, α i) : s.piecewise (c • f₁) (c • g₁) = c • s.piecewise f₁ g₁ := s.piecewise_op (δ' := α) f₁ _ fun _ ↦ (c • ·) end Set
Algebra\Group\Action\Prod.lean
/- Copyright (c) 2018 Simon Hudon. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Simon Hudon, Patrick Massot, Eric Wieser -/ import Mathlib.Algebra.Group.Action.Defs import Mathlib.Algebra.Group.Prod /-! # Prod instances for additive and multiplicative actions This file defines instances for binary product of additive and multiplicative actions and provides scalar multiplication as a homomorphism from `α × β` to `β`. ## Main declarations * `smulMulHom`/`smulMonoidHom`: Scalar multiplication bundled as a multiplicative/monoid homomorphism. ## See also * `Mathlib.Algebra.Group.Action.Option` * `Mathlib.Algebra.Group.Action.Pi` * `Mathlib.Algebra.Group.Action.Sigma` * `Mathlib.Algebra.Group.Action.Sum` # Porting notes The `to_additive` attribute can be used to generate both the `smul` and `vadd` lemmas from the corresponding `pow` lemmas, as explained on zulip here: https://leanprover.zulipchat.com/#narrow/near/316087838 This was not done as part of the port in order to stay as close as possible to the mathlib3 code. -/ assert_not_exists MonoidWithZero variable {M N P E α β : Type*} namespace Prod section variable [SMul M α] [SMul M β] [SMul N α] [SMul N β] (a : M) (x : α × β) @[to_additive] instance smul : SMul M (α × β) where smul a p := (a • p.1, a • p.2) @[to_additive (attr := simp)] lemma smul_fst : (a • x).1 = a • x.1 := rfl @[to_additive (attr := simp)] lemma smul_snd : (a • x).2 = a • x.2 := rfl @[to_additive (attr := simp)] lemma smul_mk (a : M) (b : α) (c : β) : a • (b, c) = (a • b, a • c) := rfl @[to_additive] lemma smul_def (a : M) (x : α × β) : a • x = (a • x.1, a • x.2) := rfl @[to_additive (attr := simp)] lemma smul_swap : (a • x).swap = a • x.swap := rfl variable [Pow α E] [Pow β E] @[to_additive existing smul] instance pow : Pow (α × β) E where pow p c := (p.1 ^ c, p.2 ^ c) @[to_additive existing (attr := simp) (reorder := 6 7) smul_fst] lemma pow_fst (p : α × β) (c : E) : (p ^ c).fst = p.fst ^ c := rfl @[to_additive existing (attr := simp) (reorder := 6 7) smul_snd] lemma pow_snd (p : α × β) (c : E) : (p ^ c).snd = p.snd ^ c := rfl /- Note that the `c` arguments to this lemmas cannot be in the more natural right-most positions due to limitations in `to_additive` and `to_additive_reorder`, which will silently fail to reorder more than two adjacent arguments -/ @[to_additive existing (attr := simp) (reorder := 6 7) smul_mk] lemma pow_mk (c : E) (a : α) (b : β) : Prod.mk a b ^ c = Prod.mk (a ^ c) (b ^ c) := rfl @[to_additive existing (reorder := 6 7) smul_def] lemma pow_def (p : α × β) (c : E) : p ^ c = (p.1 ^ c, p.2 ^ c) := rfl @[to_additive existing (attr := simp) (reorder := 6 7) smul_swap] lemma pow_swap (p : α × β) (c : E) : (p ^ c).swap = p.swap ^ c := rfl @[to_additive vaddAssocClass] instance isScalarTower [SMul M N] [IsScalarTower M N α] [IsScalarTower M N β] : IsScalarTower M N (α × β) where smul_assoc _ _ _ := mk.inj_iff.mpr ⟨smul_assoc _ _ _, smul_assoc _ _ _⟩ @[to_additive] instance smulCommClass [SMulCommClass M N α] [SMulCommClass M N β] : SMulCommClass M N (α × β) where smul_comm _ _ _ := mk.inj_iff.mpr ⟨smul_comm _ _ _, smul_comm _ _ _⟩ @[to_additive] instance isCentralScalar [SMul Mᵐᵒᵖ α] [SMul Mᵐᵒᵖ β] [IsCentralScalar M α] [IsCentralScalar M β] : IsCentralScalar M (α × β) where op_smul_eq_smul _ _ := Prod.ext (op_smul_eq_smul _ _) (op_smul_eq_smul _ _) @[to_additive] instance faithfulSMulLeft [FaithfulSMul M α] [Nonempty β] : FaithfulSMul M (α × β) where eq_of_smul_eq_smul h := let ⟨b⟩ := ‹Nonempty β› eq_of_smul_eq_smul fun a : α => by injection h (a, b) @[to_additive] instance faithfulSMulRight [Nonempty α] [FaithfulSMul M β] : FaithfulSMul M (α × β) where eq_of_smul_eq_smul h := let ⟨a⟩ := ‹Nonempty α› eq_of_smul_eq_smul fun b : β => by injection h (a, b) end @[to_additive] instance smulCommClassBoth [Mul N] [Mul P] [SMul M N] [SMul M P] [SMulCommClass M N N] [SMulCommClass M P P] : SMulCommClass M (N × P) (N × P) where smul_comm c x y := by simp [smul_def, mul_def, mul_smul_comm] instance isScalarTowerBoth [Mul N] [Mul P] [SMul M N] [SMul M P] [IsScalarTower M N N] [IsScalarTower M P P] : IsScalarTower M (N × P) (N × P) where smul_assoc c x y := by simp [smul_def, mul_def, smul_mul_assoc] @[to_additive] instance mulAction [Monoid M] [MulAction M α] [MulAction M β] : MulAction M (α × β) where mul_smul _ _ _ := mk.inj_iff.mpr ⟨mul_smul _ _ _, mul_smul _ _ _⟩ one_smul _ := mk.inj_iff.mpr ⟨one_smul _ _, one_smul _ _⟩ end Prod /-! ### Scalar multiplication as a homomorphism -/ section BundledSMul /-- Scalar multiplication as a multiplicative homomorphism. -/ @[simps] def smulMulHom [Monoid α] [Mul β] [MulAction α β] [IsScalarTower α β β] [SMulCommClass α β β] : α × β →ₙ* β where toFun a := a.1 • a.2 map_mul' _ _ := (smul_mul_smul _ _ _ _).symm /-- Scalar multiplication as a monoid homomorphism. -/ @[simps] def smulMonoidHom [Monoid α] [MulOneClass β] [MulAction α β] [IsScalarTower α β β] [SMulCommClass α β β] : α × β →* β := { smulMulHom with map_one' := one_smul _ _ } end BundledSMul section Action_by_Prod variable (M N α) [Monoid M] [Monoid N] /-- Construct a `MulAction` by a product monoid from `MulAction`s by the factors. This is not an instance to avoid diamonds for example when `α := M × N`. -/ @[to_additive AddAction.prodOfVAddCommClass "Construct an `AddAction` by a product monoid from `AddAction`s by the factors. This is not an instance to avoid diamonds for example when `α := M × N`."] abbrev MulAction.prodOfSMulCommClass [MulAction M α] [MulAction N α] [SMulCommClass M N α] : MulAction (M × N) α where smul mn a := mn.1 • mn.2 • a one_smul a := (one_smul M _).trans (one_smul N a) mul_smul x y a := by change (x.1 * y.1) • (x.2 * y.2) • a = x.1 • x.2 • y.1 • y.2 • a rw [mul_smul, mul_smul, smul_comm y.1 x.2] /-- A `MulAction` by a product monoid is equivalent to commuting `MulAction`s by the factors. -/ @[to_additive AddAction.prodEquiv "An `AddAction` by a product monoid is equivalent to commuting `AddAction`s by the factors."] def MulAction.prodEquiv : MulAction (M × N) α ≃ Σ' (_ : MulAction M α) (_ : MulAction N α), SMulCommClass M N α where toFun _ := letI instM := MulAction.compHom α (.inl M N) letI instN := MulAction.compHom α (.inr M N) ⟨instM, instN, { smul_comm := fun m n a ↦ by change (m, (1 : N)) • ((1 : M), n) • a = ((1 : M), n) • (m, (1 : N)) • a simp_rw [smul_smul, Prod.mk_mul_mk, mul_one, one_mul] }⟩ invFun _insts := letI := _insts.1; letI := _insts.2.1; have := _insts.2.2 MulAction.prodOfSMulCommClass M N α left_inv := by rintro ⟨-, hsmul⟩; dsimp only; ext ⟨m, n⟩ a change (m, (1 : N)) • ((1 : M), n) • a = _ rw [← hsmul, Prod.mk_mul_mk, mul_one, one_mul]; rfl right_inv := by rintro ⟨hM, hN, -⟩ dsimp only; congr 1 · ext m a; (conv_rhs => rw [← hN.one_smul a]); rfl congr 1 · funext; congr; ext m a; (conv_rhs => rw [← hN.one_smul a]); rfl · ext n a; (conv_rhs => rw [← hM.one_smul (SMul.smul n a)]); rfl · apply heq_prop end Action_by_Prod
Algebra\Group\Action\Sigma.lean
/- Copyright (c) 2022 Yaël Dillies. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Yaël Dillies -/ import Mathlib.Algebra.Group.Action.Defs /-! # Sigma instances for additive and multiplicative actions This file defines instances for arbitrary sum of additive and multiplicative actions. ## See also * `Mathlib.Algebra.Group.Action.Option` * `Mathlib.Algebra.Group.Action.Pi` * `Mathlib.Algebra.Group.Action.Prod` * `Mathlib.Algebra.Group.Action.Sum` -/ assert_not_exists MonoidWithZero variable {ι : Type*} {M N : Type*} {α : ι → Type*} namespace Sigma section SMul variable [∀ i, SMul M (α i)] [∀ i, SMul N (α i)] (a : M) (i : ι) (b : α i) (x : Σi, α i) @[to_additive Sigma.VAdd] instance : SMul M (Σi, α i) := ⟨fun a => (Sigma.map id) fun _ => (a • ·)⟩ @[to_additive] theorem smul_def : a • x = x.map id fun _ => (a • ·) := rfl @[to_additive (attr := simp)] theorem smul_mk : a • mk i b = ⟨i, a • b⟩ := rfl @[to_additive] instance instIsScalarTowerOfSMul [SMul M N] [∀ i, IsScalarTower M N (α i)] : IsScalarTower M N (Σi, α i) := ⟨fun a b x => by cases x rw [smul_mk, smul_mk, smul_mk, smul_assoc]⟩ @[to_additive] instance [∀ i, SMulCommClass M N (α i)] : SMulCommClass M N (Σi, α i) := ⟨fun a b x => by cases x rw [smul_mk, smul_mk, smul_mk, smul_mk, smul_comm]⟩ @[to_additive] instance [∀ i, SMul Mᵐᵒᵖ (α i)] [∀ i, IsCentralScalar M (α i)] : IsCentralScalar M (Σi, α i) := ⟨fun a x => by cases x rw [smul_mk, smul_mk, op_smul_eq_smul]⟩ /-- This is not an instance because `i` becomes a metavariable. -/ @[to_additive "This is not an instance because `i` becomes a metavariable."] protected theorem FaithfulSMul' [FaithfulSMul M (α i)] : FaithfulSMul M (Σi, α i) := ⟨fun h => eq_of_smul_eq_smul fun a : α i => heq_iff_eq.1 (Sigma.ext_iff.1 <| h <| mk i a).2⟩ @[to_additive] instance [Nonempty ι] [∀ i, FaithfulSMul M (α i)] : FaithfulSMul M (Σi, α i) := (Nonempty.elim ‹_›) fun i => Sigma.FaithfulSMul' i end SMul @[to_additive] instance {m : Monoid M} [∀ i, MulAction M (α i)] : MulAction M (Σi, α i) where mul_smul a b x := by cases x rw [smul_mk, smul_mk, smul_mk, mul_smul] one_smul x := by cases x rw [smul_mk, one_smul] end Sigma
Algebra\Group\Action\Sum.lean
/- Copyright (c) 2022 Yaël Dillies. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Yaël Dillies -/ import Mathlib.Algebra.Group.Action.Defs /-! # Sum instances for additive and multiplicative actions This file defines instances for additive and multiplicative actions on the binary `Sum` type. ## See also * `Mathlib.Algebra.Group.Action.Option` * `Mathlib.Algebra.Group.Action.Pi` * `Mathlib.Algebra.Group.Action.Prod` * `Mathlib.Algebra.Group.Action.Sigma` -/ assert_not_exists MonoidWithZero variable {M N P α β γ : Type*} namespace Sum section SMul variable [SMul M α] [SMul M β] [SMul N α] [SMul N β] (a : M) (b : α) (c : β) (x : α ⊕ β) @[to_additive Sum.hasVAdd] instance : SMul M (α ⊕ β) := ⟨fun a => Sum.map (a • ·) (a • ·)⟩ @[to_additive] theorem smul_def : a • x = x.map (a • ·) (a • ·) := rfl @[to_additive (attr := simp)] theorem smul_inl : a • (inl b : α ⊕ β) = inl (a • b) := rfl @[to_additive (attr := simp)] theorem smul_inr : a • (inr c : α ⊕ β) = inr (a • c) := rfl @[to_additive (attr := simp)] theorem smul_swap : (a • x).swap = a • x.swap := by cases x <;> rfl instance [SMul M N] [IsScalarTower M N α] [IsScalarTower M N β] : IsScalarTower M N (α ⊕ β) := ⟨fun a b x => by cases x exacts [congr_arg inl (smul_assoc _ _ _), congr_arg inr (smul_assoc _ _ _)]⟩ @[to_additive] instance [SMulCommClass M N α] [SMulCommClass M N β] : SMulCommClass M N (α ⊕ β) := ⟨fun a b x => by cases x exacts [congr_arg inl (smul_comm _ _ _), congr_arg inr (smul_comm _ _ _)]⟩ @[to_additive] instance [SMul Mᵐᵒᵖ α] [SMul Mᵐᵒᵖ β] [IsCentralScalar M α] [IsCentralScalar M β] : IsCentralScalar M (α ⊕ β) := ⟨fun a x => by cases x exacts [congr_arg inl (op_smul_eq_smul _ _), congr_arg inr (op_smul_eq_smul _ _)]⟩ @[to_additive] instance FaithfulSMulLeft [FaithfulSMul M α] : FaithfulSMul M (α ⊕ β) := ⟨fun h => eq_of_smul_eq_smul fun a : α => by injection h (inl a)⟩ @[to_additive] instance FaithfulSMulRight [FaithfulSMul M β] : FaithfulSMul M (α ⊕ β) := ⟨fun h => eq_of_smul_eq_smul fun b : β => by injection h (inr b)⟩ end SMul @[to_additive] instance {m : Monoid M} [MulAction M α] [MulAction M β] : MulAction M (α ⊕ β) where mul_smul a b x := by cases x exacts [congr_arg inl (mul_smul _ _ _), congr_arg inr (mul_smul _ _ _)] one_smul x := by cases x exacts [congr_arg inl (one_smul _ _), congr_arg inr (one_smul _ _)] end Sum
Algebra\Group\Action\Units.lean
/- Copyright (c) 2021 Eric Wieser. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Eric Wieser -/ import Mathlib.Algebra.Group.Action.Defs import Mathlib.Algebra.Group.Units /-! # Group actions on and by `Mˣ` This file provides the action of a unit on a type `α`, `SMul Mˣ α`, in the presence of `SMul M α`, with the obvious definition stated in `Units.smul_def`. This definition preserves `MulAction` and `DistribMulAction` structures too. Additionally, a `MulAction G M` for some group `G` satisfying some additional properties admits a `MulAction G Mˣ` structure, again with the obvious definition stated in `Units.coe_smul`. These instances use a primed name. The results are repeated for `AddUnits` and `VAdd` where relevant. -/ assert_not_exists MonoidWithZero variable {G H M N α : Type*} namespace Units @[to_additive] instance [Monoid M] [SMul M α] : SMul Mˣ α where smul m a := (m : M) • a @[to_additive] lemma smul_def [Monoid M] [SMul M α] (m : Mˣ) (a : α) : m • a = (m : M) • a := rfl @[to_additive, simp] lemma smul_mk_apply {M α : Type*} [Monoid M] [SMul M α] (m n : M) (h₁) (h₂) (a : α) : (⟨m, n, h₁, h₂⟩ : Mˣ) • a = m • a := rfl @[simp] lemma smul_isUnit [Monoid M] [SMul M α] {m : M} (hm : IsUnit m) (a : α) : hm.unit • a = m • a := rfl @[to_additive] lemma _root_.IsUnit.inv_smul [Monoid α] {a : α} (h : IsUnit a) : h.unit⁻¹ • a = 1 := h.val_inv_mul @[to_additive] instance [Monoid M] [SMul M α] [FaithfulSMul M α] : FaithfulSMul Mˣ α where eq_of_smul_eq_smul h := Units.ext <| eq_of_smul_eq_smul h @[to_additive] instance instMulAction [Monoid M] [MulAction M α] : MulAction Mˣ α where one_smul := (one_smul M : _) mul_smul m n := mul_smul (m : M) n @[to_additive] instance smulCommClass_left [Monoid M] [SMul M α] [SMul N α] [SMulCommClass M N α] : SMulCommClass Mˣ N α where smul_comm m n := (smul_comm (m : M) n : _) @[to_additive] instance smulCommClass_right [Monoid N] [SMul M α] [SMul N α] [SMulCommClass M N α] : SMulCommClass M Nˣ α where smul_comm m n := (smul_comm m (n : N) : _) @[to_additive] instance [Monoid M] [SMul M N] [SMul M α] [SMul N α] [IsScalarTower M N α] : IsScalarTower Mˣ N α where smul_assoc m n := (smul_assoc (m : M) n : _) /-! ### Action of a group `G` on units of `M` -/ /-- If an action `G` associates and commutes with multiplication on `M`, then it lifts to an action on `Mˣ`. Notably, this provides `MulAction Mˣ Nˣ` under suitable conditions. -/ @[to_additive] instance mulAction' [Group G] [Monoid M] [MulAction G M] [SMulCommClass G M M] [IsScalarTower G M M] : MulAction G Mˣ where smul g m := ⟨g • (m : M), (g⁻¹ • ((m⁻¹ : Mˣ) : M)), by rw [smul_mul_smul, Units.mul_inv, mul_right_inv, one_smul], by rw [smul_mul_smul, Units.inv_mul, mul_left_inv, one_smul]⟩ one_smul m := Units.ext <| one_smul _ _ mul_smul g₁ g₂ m := Units.ext <| mul_smul _ _ _ @[to_additive (attr := simp)] lemma val_smul [Group G] [Monoid M] [MulAction G M] [SMulCommClass G M M] [IsScalarTower G M M] (g : G) (m : Mˣ) : ↑(g • m) = g • (m : M) := rfl /-- Note that this lemma exists more generally as the global `smul_inv` -/ @[to_additive (attr := simp)] lemma smul_inv [Group G] [Monoid M] [MulAction G M] [SMulCommClass G M M] [IsScalarTower G M M] (g : G) (m : Mˣ) : (g • m)⁻¹ = g⁻¹ • m⁻¹ := ext rfl /-- Transfer `SMulCommClass G H M` to `SMulCommClass G H Mˣ`. -/ @[to_additive "Transfer `VAddCommClass G H M` to `VAddCommClass G H (AddUnits M)`."] instance smulCommClass' [Group G] [Group H] [Monoid M] [MulAction G M] [SMulCommClass G M M] [MulAction H M] [SMulCommClass H M M] [IsScalarTower G M M] [IsScalarTower H M M] [SMulCommClass G H M] : SMulCommClass G H Mˣ where smul_comm g h m := Units.ext <| smul_comm g h (m : M) /-- Transfer `IsScalarTower G H M` to `IsScalarTower G H Mˣ`. -/ @[to_additive "Transfer `VAddAssocClass G H M` to `VAddAssocClass G H (AddUnits M)`."] instance isScalarTower' [SMul G H] [Group G] [Group H] [Monoid M] [MulAction G M] [SMulCommClass G M M] [MulAction H M] [SMulCommClass H M M] [IsScalarTower G M M] [IsScalarTower H M M] [IsScalarTower G H M] : IsScalarTower G H Mˣ where smul_assoc g h m := Units.ext <| smul_assoc g h (m : M) /-- Transfer `IsScalarTower G M α` to `IsScalarTower G Mˣ α`. -/ @[to_additive "Transfer `VAddAssocClass G M α` to `VAddAssocClass G (AddUnits M) α`."] instance isScalarTower'_left [Group G] [Monoid M] [MulAction G M] [SMul M α] [SMul G α] [SMulCommClass G M M] [IsScalarTower G M M] [IsScalarTower G M α] : IsScalarTower G Mˣ α where smul_assoc g m := (smul_assoc g (m : M) : _) -- Just to prove this transfers a particularly useful instance. example [Monoid M] [Monoid N] [MulAction M N] [SMulCommClass M N N] [IsScalarTower M N N] : MulAction Mˣ Nˣ := Units.mulAction' end Units @[to_additive] lemma IsUnit.smul [Group G] [Monoid M] [MulAction G M] [SMulCommClass G M M] [IsScalarTower G M M] {m : M} (g : G) (h : IsUnit m) : IsUnit (g • m) := let ⟨u, hu⟩ := h hu ▸ ⟨g • u, Units.val_smul _ _⟩
Algebra\Group\Commute\Basic.lean
/- Copyright (c) 2019 Neil Strickland. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Neil Strickland, Yury Kudryashov -/ import Mathlib.Algebra.Group.Commute.Defs import Mathlib.Algebra.Group.Semiconj.Basic /-! # Additional lemmas about commuting pairs of elements in monoids -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered variable {G : Type*} namespace Commute section DivisionMonoid variable [DivisionMonoid G] {a b c d : G} @[to_additive] protected theorem inv_inv : Commute a b → Commute a⁻¹ b⁻¹ := SemiconjBy.inv_inv_symm @[to_additive (attr := simp)] theorem inv_inv_iff : Commute a⁻¹ b⁻¹ ↔ Commute a b := SemiconjBy.inv_inv_symm_iff @[to_additive] protected theorem div_mul_div_comm (hbd : Commute b d) (hbc : Commute b⁻¹ c) : a / b * (c / d) = a * c / (b * d) := by simp_rw [div_eq_mul_inv, mul_inv_rev, hbd.inv_inv.symm.eq, hbc.mul_mul_mul_comm] @[to_additive] protected theorem mul_div_mul_comm (hcd : Commute c d) (hbc : Commute b c⁻¹) : a * b / (c * d) = a / c * (b / d) := (hcd.div_mul_div_comm hbc.symm).symm @[to_additive] protected theorem div_div_div_comm (hbc : Commute b c) (hbd : Commute b⁻¹ d) (hcd : Commute c⁻¹ d) : a / b / (c / d) = a / c / (b / d) := by simp_rw [div_eq_mul_inv, mul_inv_rev, inv_inv, hbd.symm.eq, hcd.symm.eq, hbc.inv_inv.mul_mul_mul_comm] end DivisionMonoid section Group variable [Group G] {a b : G} @[to_additive (attr := simp)] lemma inv_left_iff : Commute a⁻¹ b ↔ Commute a b := SemiconjBy.inv_symm_left_iff @[to_additive] alias ⟨_, inv_left⟩ := inv_left_iff @[to_additive (attr := simp)] lemma inv_right_iff : Commute a b⁻¹ ↔ Commute a b := SemiconjBy.inv_right_iff @[to_additive] alias ⟨_, inv_right⟩ := inv_right_iff @[to_additive] protected lemma inv_mul_cancel (h : Commute a b) : a⁻¹ * b * a = b := by rw [h.inv_left.eq, inv_mul_cancel_right] @[to_additive] lemma inv_mul_cancel_assoc (h : Commute a b) : a⁻¹ * (b * a) = b := by rw [← mul_assoc, h.inv_mul_cancel] @[to_additive (attr := simp)] protected theorem conj_iff (h : G) : Commute (h * a * h⁻¹) (h * b * h⁻¹) ↔ Commute a b := SemiconjBy.conj_iff @[to_additive] protected theorem conj (comm : Commute a b) (h : G) : Commute (h * a * h⁻¹) (h * b * h⁻¹) := (Commute.conj_iff h).mpr comm @[to_additive (attr := simp)] lemma zpow_right (h : Commute a b) (m : ℤ) : Commute a (b ^ m) := SemiconjBy.zpow_right h m @[to_additive (attr := simp)] lemma zpow_left (h : Commute a b) (m : ℤ) : Commute (a ^ m) b := (h.symm.zpow_right m).symm @[to_additive] lemma zpow_zpow (h : Commute a b) (m n : ℤ) : Commute (a ^ m) (b ^ n) := (h.zpow_left m).zpow_right n variable (a) (m n : ℤ) @[to_additive] lemma self_zpow : Commute a (a ^ n) := (Commute.refl a).zpow_right n @[to_additive] lemma zpow_self : Commute (a ^ n) a := (Commute.refl a).zpow_left n @[to_additive] lemma zpow_zpow_self : Commute (a ^ m) (a ^ n) := (Commute.refl a).zpow_zpow m n end Group end Commute section Group variable [Group G] @[to_additive] lemma pow_inv_comm (a : G) (m n : ℕ) : a⁻¹ ^ m * a ^ n = a ^ n * a⁻¹ ^ m := (Commute.refl a).inv_left.pow_pow _ _ end Group
Algebra\Group\Commute\Defs.lean
/- Copyright (c) 2019 Neil Strickland. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Neil Strickland, Yury Kudryashov -/ import Mathlib.Algebra.Group.Semiconj.Defs import Mathlib.Init.Algebra.Classes /-! # Commuting pairs of elements in monoids We define the predicate `Commute a b := a * b = b * a` and provide some operations on terms `(h : Commute a b)`. E.g., if `a`, `b`, and c are elements of a semiring, and that `hb : Commute a b` and `hc : Commute a c`. Then `hb.pow_left 5` proves `Commute (a ^ 5) b` and `(hb.pow_right 2).add_right (hb.mul_right hc)` proves `Commute a (b ^ 2 + b * c)`. Lean does not immediately recognise these terms as equations, so for rewriting we need syntax like `rw [(hb.pow_left 5).eq]` rather than just `rw [hb.pow_left 5]`. This file defines only a few operations (`mul_left`, `inv_right`, etc). Other operations (`pow_right`, field inverse etc) are in the files that define corresponding notions. ## Implementation details Most of the proofs come from the properties of `SemiconjBy`. -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered variable {G M S : Type*} /-- Two elements commute if `a * b = b * a`. -/ @[to_additive "Two elements additively commute if `a + b = b + a`"] def Commute [Mul S] (a b : S) : Prop := SemiconjBy a b b /-- Two elements `a` and `b` commute if `a * b = b * a`. -/ @[to_additive] theorem commute_iff_eq [Mul S] (a b : S) : Commute a b ↔ a * b = b * a := Iff.rfl namespace Commute section Mul variable [Mul S] /-- Equality behind `Commute a b`; useful for rewriting. -/ @[to_additive "Equality behind `AddCommute a b`; useful for rewriting."] protected theorem eq {a b : S} (h : Commute a b) : a * b = b * a := h /-- Any element commutes with itself. -/ @[to_additive (attr := refl, simp) "Any element commutes with itself."] protected theorem refl (a : S) : Commute a a := Eq.refl (a * a) /-- If `a` commutes with `b`, then `b` commutes with `a`. -/ @[to_additive (attr := symm) "If `a` commutes with `b`, then `b` commutes with `a`."] protected theorem symm {a b : S} (h : Commute a b) : Commute b a := Eq.symm h @[to_additive] protected theorem semiconjBy {a b : S} (h : Commute a b) : SemiconjBy a b b := h @[to_additive] protected theorem symm_iff {a b : S} : Commute a b ↔ Commute b a := ⟨Commute.symm, Commute.symm⟩ @[to_additive] instance : IsRefl S Commute := ⟨Commute.refl⟩ -- This instance is useful for `Finset.noncommProd` @[to_additive] instance on_isRefl {f : G → S} : IsRefl G fun a b => Commute (f a) (f b) := ⟨fun _ => Commute.refl _⟩ end Mul section Semigroup variable [Semigroup S] {a b c : S} /-- If `a` commutes with both `b` and `c`, then it commutes with their product. -/ @[to_additive (attr := simp) "If `a` commutes with both `b` and `c`, then it commutes with their sum."] theorem mul_right (hab : Commute a b) (hac : Commute a c) : Commute a (b * c) := SemiconjBy.mul_right hab hac -- I think `ₓ` is necessary because of the `mul` vs `HMul` distinction /-- If both `a` and `b` commute with `c`, then their product commutes with `c`. -/ @[to_additive (attr := simp) "If both `a` and `b` commute with `c`, then their product commutes with `c`."] theorem mul_left (hac : Commute a c) (hbc : Commute b c) : Commute (a * b) c := SemiconjBy.mul_left hac hbc -- I think `ₓ` is necessary because of the `mul` vs `HMul` distinction @[to_additive] protected theorem right_comm (h : Commute b c) (a : S) : a * b * c = a * c * b := by simp only [mul_assoc, h.eq] -- I think `ₓ` is necessary because of the `mul` vs `HMul` distinction @[to_additive] protected theorem left_comm (h : Commute a b) (c) : a * (b * c) = b * (a * c) := by simp only [← mul_assoc, h.eq] -- I think `ₓ` is necessary because of the `mul` vs `HMul` distinction @[to_additive] protected theorem mul_mul_mul_comm (hbc : Commute b c) (a d : S) : a * b * (c * d) = a * c * (b * d) := by simp only [hbc.left_comm, mul_assoc] end Semigroup @[to_additive] protected theorem all [CommMagma S] (a b : S) : Commute a b := mul_comm a b section MulOneClass variable [MulOneClass M] @[to_additive (attr := simp)] theorem one_right (a : M) : Commute a 1 := SemiconjBy.one_right a -- I think `ₓ` is necessary because `One.toOfNat1` appears in the Lean 4 version @[to_additive (attr := simp)] theorem one_left (a : M) : Commute 1 a := SemiconjBy.one_left a -- I think `ₓ` is necessary because `One.toOfNat1` appears in the Lean 4 version end MulOneClass section Monoid variable [Monoid M] {a b : M} @[to_additive (attr := simp)] theorem pow_right (h : Commute a b) (n : ℕ) : Commute a (b ^ n) := SemiconjBy.pow_right h n -- `MulOneClass.toHasMul` vs. `MulOneClass.toMul` @[to_additive (attr := simp)] theorem pow_left (h : Commute a b) (n : ℕ) : Commute (a ^ n) b := (h.symm.pow_right n).symm -- `MulOneClass.toHasMul` vs. `MulOneClass.toMul` -- todo: should nat power be called `nsmul` here? @[to_additive (attr := simp)] theorem pow_pow (h : Commute a b) (m n : ℕ) : Commute (a ^ m) (b ^ n) := (h.pow_left m).pow_right n -- `MulOneClass.toHasMul` vs. `MulOneClass.toMul` -- Porting note: `simpNF` told me to remove the `simp` attribute @[to_additive] theorem self_pow (a : M) (n : ℕ) : Commute a (a ^ n) := (Commute.refl a).pow_right n -- `MulOneClass.toHasMul` vs. `MulOneClass.toMul` -- Porting note: `simpNF` told me to remove the `simp` attribute @[to_additive] theorem pow_self (a : M) (n : ℕ) : Commute (a ^ n) a := (Commute.refl a).pow_left n -- `MulOneClass.toHasMul` vs. `MulOneClass.toMul` -- Porting note: `simpNF` told me to remove the `simp` attribute @[to_additive] theorem pow_pow_self (a : M) (m n : ℕ) : Commute (a ^ m) (a ^ n) := (Commute.refl a).pow_pow m n -- `MulOneClass.toHasMul` vs. `MulOneClass.toMul` @[to_additive] lemma mul_pow (h : Commute a b) : ∀ n, (a * b) ^ n = a ^ n * b ^ n | 0 => by rw [pow_zero, pow_zero, pow_zero, one_mul] | n + 1 => by simp only [pow_succ', h.mul_pow n, ← mul_assoc, (h.pow_left n).right_comm] end Monoid section DivisionMonoid variable [DivisionMonoid G] {a b c d : G} @[to_additive] protected theorem mul_inv (hab : Commute a b) : (a * b)⁻¹ = a⁻¹ * b⁻¹ := by rw [hab.eq, mul_inv_rev] @[to_additive] protected theorem inv (hab : Commute a b) : (a * b)⁻¹ = a⁻¹ * b⁻¹ := by rw [hab.eq, mul_inv_rev] @[to_additive AddCommute.zsmul_add] protected lemma mul_zpow (h : Commute a b) : ∀ n : ℤ, (a * b) ^ n = a ^ n * b ^ n | (n : ℕ) => by simp [zpow_natCast, h.mul_pow n] | .negSucc n => by simp [h.mul_pow, (h.pow_pow _ _).eq, mul_inv_rev] end DivisionMonoid section Group variable [Group G] {a b : G} @[to_additive] protected theorem mul_inv_cancel (h : Commute a b) : a * b * a⁻¹ = b := by rw [h.eq, mul_inv_cancel_right] @[to_additive] theorem mul_inv_cancel_assoc (h : Commute a b) : a * (b * a⁻¹) = b := by rw [← mul_assoc, h.mul_inv_cancel] end Group end Commute
Algebra\Group\Commute\Hom.lean
/- Copyright (c) 2018 Patrick Massot. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Patrick Massot, Kevin Buzzard, Scott Morrison, Johan Commelin, Chris Hughes, Johannes Hölzl, Yury Kudryashov -/ import Mathlib.Algebra.Group.Commute.Defs import Mathlib.Algebra.Group.Hom.Defs /-! # Multiplicative homomorphisms respect semiconjugation and commutation. -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered section Commute variable {F M N : Type*} [Mul M] [Mul N] {a x y : M} [FunLike F M N] @[to_additive (attr := simp)] protected theorem SemiconjBy.map [MulHomClass F M N] (h : SemiconjBy a x y) (f : F) : SemiconjBy (f a) (f x) (f y) := by simpa only [SemiconjBy, map_mul] using congr_arg f h @[to_additive (attr := simp)] protected theorem Commute.map [MulHomClass F M N] (h : Commute x y) (f : F) : Commute (f x) (f y) := SemiconjBy.map h f @[to_additive (attr := simp)] protected theorem SemiconjBy.of_map [MulHomClass F M N] (f : F) (hf : Function.Injective f) (h : SemiconjBy (f a) (f x) (f y)) : SemiconjBy a x y := hf (by simpa only [SemiconjBy, map_mul] using h) @[to_additive (attr := simp)] theorem Commute.of_map [MulHomClass F M N] {f : F} (hf : Function.Injective f) (h : Commute (f x) (f y)) : Commute x y := hf (by simpa only [map_mul] using h.eq) end Commute
Algebra\Group\Commute\Units.lean
/- Copyright (c) 2019 Neil Strickland. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Neil Strickland, Yury Kudryashov -/ import Mathlib.Algebra.Group.Commute.Defs import Mathlib.Algebra.Group.Semiconj.Units /-! # Lemmas about commuting pairs of elements involving units. -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered variable {M : Type*} section Monoid variable [Monoid M] {n : ℕ} {a b : M} {u u₁ u₂ : Mˣ} namespace Commute @[to_additive] theorem units_inv_right : Commute a u → Commute a ↑u⁻¹ := SemiconjBy.units_inv_right @[to_additive (attr := simp)] theorem units_inv_right_iff : Commute a ↑u⁻¹ ↔ Commute a u := SemiconjBy.units_inv_right_iff @[to_additive] theorem units_inv_left : Commute (↑u) a → Commute (↑u⁻¹) a := SemiconjBy.units_inv_symm_left @[to_additive (attr := simp)] theorem units_inv_left_iff : Commute (↑u⁻¹) a ↔ Commute (↑u) a := SemiconjBy.units_inv_symm_left_iff @[to_additive] theorem units_val : Commute u₁ u₂ → Commute (u₁ : M) u₂ := SemiconjBy.units_val @[to_additive] theorem units_of_val : Commute (u₁ : M) u₂ → Commute u₁ u₂ := SemiconjBy.units_of_val @[to_additive (attr := simp)] theorem units_val_iff : Commute (u₁ : M) u₂ ↔ Commute u₁ u₂ := SemiconjBy.units_val_iff end Commute /-- If the product of two commuting elements is a unit, then the left multiplier is a unit. -/ @[to_additive "If the sum of two commuting elements is an additive unit, then the left summand is an additive unit."] def Units.leftOfMul (u : Mˣ) (a b : M) (hu : a * b = u) (hc : Commute a b) : Mˣ where val := a inv := b * ↑u⁻¹ val_inv := by rw [← mul_assoc, hu, u.mul_inv] inv_val := by have : Commute a u := hu ▸ (Commute.refl _).mul_right hc rw [← this.units_inv_right.right_comm, ← hc.eq, hu, u.mul_inv] /-- If the product of two commuting elements is a unit, then the right multiplier is a unit. -/ @[to_additive "If the sum of two commuting elements is an additive unit, then the right summand is an additive unit."] def Units.rightOfMul (u : Mˣ) (a b : M) (hu : a * b = u) (hc : Commute a b) : Mˣ := u.leftOfMul b a (hc.eq ▸ hu) hc.symm @[to_additive] theorem Commute.isUnit_mul_iff (h : Commute a b) : IsUnit (a * b) ↔ IsUnit a ∧ IsUnit b := ⟨fun ⟨u, hu⟩ => ⟨(u.leftOfMul a b hu.symm h).isUnit, (u.rightOfMul a b hu.symm h).isUnit⟩, fun H => H.1.mul H.2⟩ @[to_additive (attr := simp)] theorem isUnit_mul_self_iff : IsUnit (a * a) ↔ IsUnit a := (Commute.refl a).isUnit_mul_iff.trans and_self_iff @[to_additive (attr := simp)] lemma Commute.units_zpow_right (h : Commute a u) (m : ℤ) : Commute a ↑(u ^ m) := SemiconjBy.units_zpow_right h m @[to_additive (attr := simp)] lemma Commute.units_zpow_left (h : Commute ↑u a) (m : ℤ) : Commute ↑(u ^ m) a := (h.symm.units_zpow_right m).symm /-- If a natural power of `x` is a unit, then `x` is a unit. -/ @[to_additive "If a natural multiple of `x` is an additive unit, then `x` is an additive unit."] def Units.ofPow (u : Mˣ) (x : M) {n : ℕ} (hn : n ≠ 0) (hu : x ^ n = u) : Mˣ := u.leftOfMul x (x ^ (n - 1)) (by rwa [← _root_.pow_succ', Nat.sub_add_cancel (Nat.succ_le_of_lt <| Nat.pos_of_ne_zero hn)]) (Commute.self_pow _ _) @[to_additive (attr := simp)] lemma isUnit_pow_iff (hn : n ≠ 0) : IsUnit (a ^ n) ↔ IsUnit a := ⟨fun ⟨u, hu⟩ ↦ (u.ofPow a hn hu.symm).isUnit, IsUnit.pow n⟩ @[to_additive] lemma isUnit_pow_succ_iff : IsUnit (a ^ (n + 1)) ↔ IsUnit a := isUnit_pow_iff n.succ_ne_zero /-- If `a ^ n = 1`, `n ≠ 0`, then `a` is a unit. -/ @[to_additive (attr := simps!) "If `n • x = 0`, `n ≠ 0`, then `x` is an additive unit."] def Units.ofPowEqOne (a : M) (n : ℕ) (ha : a ^ n = 1) (hn : n ≠ 0) : Mˣ := Units.ofPow 1 a hn ha @[to_additive (attr := simp)] lemma Units.pow_ofPowEqOne (ha : a ^ n = 1) (hn : n ≠ 0) : Units.ofPowEqOne _ n ha hn ^ n = 1 := Units.ext <| by simp [ha] @[to_additive] lemma isUnit_ofPowEqOne (ha : a ^ n = 1) (hn : n ≠ 0) : IsUnit a := (Units.ofPowEqOne _ n ha hn).isUnit end Monoid section DivisionMonoid variable [DivisionMonoid M] {a b c d : M} @[to_additive] lemma Commute.div_eq_div_iff_of_isUnit (hbd : Commute b d) (hb : IsUnit b) (hd : IsUnit d) : a / b = c / d ↔ a * d = c * b := by rw [← (hb.mul hd).mul_left_inj, ← mul_assoc, hb.div_mul_cancel, ← mul_assoc, hbd.right_comm, hd.div_mul_cancel] end DivisionMonoid
Algebra\Group\Equiv\Basic.lean
/- Copyright (c) 2018 Johannes Hölzl. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Johannes Hölzl, Callum Sutton, Yury Kudryashov -/ import Mathlib.Algebra.Group.Hom.Basic import Mathlib.Data.FunLike.Equiv import Mathlib.Logic.Equiv.Basic /-! # Multiplicative and additive equivs In this file we define two extensions of `Equiv` called `AddEquiv` and `MulEquiv`, which are datatypes representing isomorphisms of `AddMonoid`s/`AddGroup`s and `Monoid`s/`Group`s. ## Notations * ``infix ` ≃* `:25 := MulEquiv`` * ``infix ` ≃+ `:25 := AddEquiv`` The extended equivs all have coercions to functions, and the coercions are the canonical notation when treating the isomorphisms as maps. ## Tags Equiv, MulEquiv, AddEquiv -/ open Function variable {F α β A B M N P Q G H : Type*} /-- Makes a `OneHom` inverse from the bijective inverse of a `OneHom` -/ @[to_additive (attr := simps) "Make a `ZeroHom` inverse from the bijective inverse of a `ZeroHom`"] def OneHom.inverse [One M] [One N] (f : OneHom M N) (g : N → M) (h₁ : Function.LeftInverse g f) : OneHom N M := { toFun := g, map_one' := by rw [← f.map_one, h₁] } /-- Makes a multiplicative inverse from a bijection which preserves multiplication. -/ @[to_additive (attr := simps) "Makes an additive inverse from a bijection which preserves addition."] def MulHom.inverse [Mul M] [Mul N] (f : M →ₙ* N) (g : N → M) (h₁ : Function.LeftInverse g f) (h₂ : Function.RightInverse g f) : N →ₙ* M where toFun := g map_mul' x y := calc g (x * y) = g (f (g x) * f (g y)) := by rw [h₂ x, h₂ y] _ = g (f (g x * g y)) := by rw [f.map_mul] _ = g x * g y := h₁ _ /-- The inverse of a bijective `MonoidHom` is a `MonoidHom`. -/ @[to_additive (attr := simps) "The inverse of a bijective `AddMonoidHom` is an `AddMonoidHom`."] def MonoidHom.inverse {A B : Type*} [Monoid A] [Monoid B] (f : A →* B) (g : B → A) (h₁ : Function.LeftInverse g f) (h₂ : Function.RightInverse g f) : B →* A := { (f : OneHom A B).inverse g h₁, (f : A →ₙ* B).inverse g h₁ h₂ with toFun := g } /-- `AddEquiv α β` is the type of an equiv `α ≃ β` which preserves addition. -/ structure AddEquiv (A B : Type*) [Add A] [Add B] extends A ≃ B, AddHom A B /-- `AddEquivClass F A B` states that `F` is a type of addition-preserving morphisms. You should extend this class when you extend `AddEquiv`. -/ class AddEquivClass (F : Type*) (A B : outParam Type*) [Add A] [Add B] [EquivLike F A B] : Prop where /-- Preserves addition. -/ map_add : ∀ (f : F) (a b), f (a + b) = f a + f b /-- The `Equiv` underlying an `AddEquiv`. -/ add_decl_doc AddEquiv.toEquiv /-- The `AddHom` underlying an `AddEquiv`. -/ add_decl_doc AddEquiv.toAddHom /-- `MulEquiv α β` is the type of an equiv `α ≃ β` which preserves multiplication. -/ @[to_additive] structure MulEquiv (M N : Type*) [Mul M] [Mul N] extends M ≃ N, M →ₙ* N -- Porting note: remove when `to_additive` can do this -- https://github.com/leanprover-community/mathlib4/issues/660 attribute [to_additive existing] MulEquiv.toMulHom /-- The `Equiv` underlying a `MulEquiv`. -/ add_decl_doc MulEquiv.toEquiv /-- The `MulHom` underlying a `MulEquiv`. -/ add_decl_doc MulEquiv.toMulHom /-- `MulEquivClass F A B` states that `F` is a type of multiplication-preserving morphisms. You should extend this class when you extend `MulEquiv`. -/ -- TODO: make this a synonym for MulHomClass? @[to_additive] class MulEquivClass (F : Type*) (A B : outParam Type*) [Mul A] [Mul B] [EquivLike F A B] : Prop where /-- Preserves multiplication. -/ map_mul : ∀ (f : F) (a b), f (a * b) = f a * f b /-- Notation for a `MulEquiv`. -/ infixl:25 " ≃* " => MulEquiv /-- Notation for an `AddEquiv`. -/ infixl:25 " ≃+ " => AddEquiv namespace MulEquivClass variable (F) variable [EquivLike F M N] -- See note [lower instance priority] @[to_additive] instance (priority := 100) instMulHomClass (F : Type*) [Mul M] [Mul N] [EquivLike F M N] [h : MulEquivClass F M N] : MulHomClass F M N := { h with } -- See note [lower instance priority] @[to_additive] instance (priority := 100) instMonoidHomClass [MulOneClass M] [MulOneClass N] [MulEquivClass F M N] : MonoidHomClass F M N := { MulEquivClass.instMulHomClass F with map_one := fun e => calc e 1 = e 1 * 1 := (mul_one _).symm _ = e 1 * e (EquivLike.inv e (1 : N) : M) := congr_arg _ (EquivLike.right_inv e 1).symm _ = e (EquivLike.inv e (1 : N)) := by rw [← map_mul, one_mul] _ = 1 := EquivLike.right_inv e 1 } variable [EquivLike F α β] variable {F} @[to_additive (attr := simp)] theorem map_eq_one_iff {M N} [MulOneClass M] [MulOneClass N] [EquivLike F M N] [MulEquivClass F M N] (h : F) {x : M} : h x = 1 ↔ x = 1 := _root_.map_eq_one_iff h (EquivLike.injective h) @[to_additive] theorem map_ne_one_iff {M N} [MulOneClass M] [MulOneClass N] [EquivLike F M N] [MulEquivClass F M N] (h : F) {x : M} : h x ≠ 1 ↔ x ≠ 1 := _root_.map_ne_one_iff h (EquivLike.injective h) end MulEquivClass variable [EquivLike F α β] /-- Turn an element of a type `F` satisfying `MulEquivClass F α β` into an actual `MulEquiv`. This is declared as the default coercion from `F` to `α ≃* β`. -/ @[to_additive (attr := coe) "Turn an element of a type `F` satisfying `AddEquivClass F α β` into an actual `AddEquiv`. This is declared as the default coercion from `F` to `α ≃+ β`."] def MulEquivClass.toMulEquiv [Mul α] [Mul β] [MulEquivClass F α β] (f : F) : α ≃* β := { (f : α ≃ β), (f : α →ₙ* β) with } /-- Any type satisfying `MulEquivClass` can be cast into `MulEquiv` via `MulEquivClass.toMulEquiv`. -/ @[to_additive "Any type satisfying `AddEquivClass` can be cast into `AddEquiv` via `AddEquivClass.toAddEquiv`. "] instance [Mul α] [Mul β] [MulEquivClass F α β] : CoeTC F (α ≃* β) := ⟨MulEquivClass.toMulEquiv⟩ @[to_additive] theorem MulEquivClass.toMulEquiv_injective [Mul α] [Mul β] [MulEquivClass F α β] : Function.Injective ((↑) : F → α ≃* β) := fun _ _ e ↦ DFunLike.ext _ _ fun a ↦ congr_arg (fun e : α ≃* β ↦ e.toFun a) e namespace MulEquiv section Mul variable [Mul M] [Mul N] [Mul P] [Mul Q] @[to_additive] instance : EquivLike (M ≃* N) M N where coe f := f.toFun inv f := f.invFun left_inv f := f.left_inv right_inv f := f.right_inv coe_injective' f g h₁ h₂ := by cases f cases g congr apply Equiv.coe_fn_injective h₁ @[to_additive] instance : MulEquivClass (M ≃* N) M N where map_mul f := f.map_mul' @[to_additive] -- shortcut instance that doesn't generate any subgoals instance : CoeFun (M ≃* N) fun _ ↦ M → N where coe f := f @[to_additive (attr := simp)] theorem toEquiv_eq_coe (f : M ≃* N) : f.toEquiv = f := rfl -- Porting note: added, to simplify `f.toMulHom` back to the coercion via `MulHomClass.toMulHom`. @[to_additive (attr := simp)] theorem toMulHom_eq_coe (f : M ≃* N) : f.toMulHom = ↑f := rfl -- Porting note: `to_fun_eq_coe` no longer needed in Lean4 @[to_additive (attr := simp)] theorem coe_toEquiv (f : M ≃* N) : ⇑(f : M ≃ N) = f := rfl -- Porting note (#11215): TODO: `MulHom.coe_mk` simplifies `↑f.toMulHom` to `f.toMulHom.toFun`, -- not `f.toEquiv.toFun`; use higher priority as a workaround @[to_additive (attr := simp 1100)] theorem coe_toMulHom {f : M ≃* N} : (f.toMulHom : M → N) = f := rfl /-- A multiplicative isomorphism preserves multiplication. -/ @[to_additive "An additive isomorphism preserves addition."] protected theorem map_mul (f : M ≃* N) : ∀ x y, f (x * y) = f x * f y := _root_.map_mul f /-- Makes a multiplicative isomorphism from a bijection which preserves multiplication. -/ @[to_additive "Makes an additive isomorphism from a bijection which preserves addition."] def mk' (f : M ≃ N) (h : ∀ x y, f (x * y) = f x * f y) : M ≃* N := ⟨f, h⟩ @[to_additive] protected theorem bijective (e : M ≃* N) : Function.Bijective e := EquivLike.bijective e @[to_additive] protected theorem injective (e : M ≃* N) : Function.Injective e := EquivLike.injective e @[to_additive] protected theorem surjective (e : M ≃* N) : Function.Surjective e := EquivLike.surjective e /-- The identity map is a multiplicative isomorphism. -/ @[to_additive (attr := refl) "The identity map is an additive isomorphism."] def refl (M : Type*) [Mul M] : M ≃* M := { Equiv.refl _ with map_mul' := fun _ _ => rfl } @[to_additive] instance : Inhabited (M ≃* M) := ⟨refl M⟩ /-- An alias for `h.symm.map_mul`. Introduced to fix the issue in https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/!4.234183.20.60simps.60.20maximum.20recursion.20depth -/ @[to_additive] lemma symm_map_mul {M N : Type*} [Mul M] [Mul N] (h : M ≃* N) (x y : N) : h.symm (x * y) = h.symm x * h.symm y := (h.toMulHom.inverse h.toEquiv.symm h.left_inv h.right_inv).map_mul x y /-- The inverse of an isomorphism is an isomorphism. -/ @[to_additive (attr := symm) "The inverse of an isomorphism is an isomorphism."] def symm {M N : Type*} [Mul M] [Mul N] (h : M ≃* N) : N ≃* M := ⟨h.toEquiv.symm, h.symm_map_mul⟩ @[to_additive] -- Porting note: no longer a `simp`, see below theorem invFun_eq_symm {f : M ≃* N} : f.invFun = f.symm := rfl -- Porting note: to_additive translated the name incorrectly in mathlib 3. @[to_additive (attr := simp)] theorem coe_toEquiv_symm (f : M ≃* N) : ((f : M ≃ N).symm : N → M) = f.symm := rfl @[to_additive (attr := simp)] theorem equivLike_inv_eq_symm (f : M ≃* N) : EquivLike.inv f = f.symm := rfl -- we don't hyperlink the note in the additive version, since that breaks syntax highlighting -- in the whole file. /-- See Note [custom simps projection] -/ @[to_additive "See Note [custom simps projection]"] -- this comment fixes the syntax highlighting " def Simps.symm_apply (e : M ≃* N) : N → M := e.symm initialize_simps_projections AddEquiv (toFun → apply, invFun → symm_apply) initialize_simps_projections MulEquiv (toFun → apply, invFun → symm_apply) @[to_additive (attr := simp)] theorem toEquiv_symm (f : M ≃* N) : (f.symm : N ≃ M) = (f : M ≃ N).symm := rfl @[to_additive (attr := simp)] theorem coe_mk (f : M ≃ N) (hf : ∀ x y, f (x * y) = f x * f y) : (mk f hf : M → N) = f := rfl -- Porting note: `toEquiv_mk` no longer needed in Lean4 @[to_additive (attr := simp)] theorem symm_symm (f : M ≃* N) : f.symm.symm = f := rfl @[to_additive] theorem symm_bijective : Function.Bijective (symm : (M ≃* N) → N ≃* M) := Function.bijective_iff_has_inverse.mpr ⟨_, symm_symm, symm_symm⟩ @[to_additive (attr := simp)] theorem symm_mk (f : M ≃ N) (h) : (MulEquiv.mk f h).symm = ⟨f.symm, (MulEquiv.mk f h).symm_map_mul⟩ := rfl @[to_additive (attr := simp)] theorem refl_symm : (refl M).symm = refl M := rfl /-- Transitivity of multiplication-preserving isomorphisms -/ @[to_additive (attr := trans) "Transitivity of addition-preserving isomorphisms"] def trans (h1 : M ≃* N) (h2 : N ≃* P) : M ≃* P := { h1.toEquiv.trans h2.toEquiv with map_mul' := fun x y => show h2 (h1 (x * y)) = h2 (h1 x) * h2 (h1 y) by rw [h1.map_mul, h2.map_mul] } /-- `e.symm` is a right inverse of `e`, written as `e (e.symm y) = y`. -/ @[to_additive (attr := simp) "`e.symm` is a right inverse of `e`, written as `e (e.symm y) = y`."] theorem apply_symm_apply (e : M ≃* N) (y : N) : e (e.symm y) = y := e.toEquiv.apply_symm_apply y /-- `e.symm` is a left inverse of `e`, written as `e.symm (e y) = y`. -/ @[to_additive (attr := simp) "`e.symm` is a left inverse of `e`, written as `e.symm (e y) = y`."] theorem symm_apply_apply (e : M ≃* N) (x : M) : e.symm (e x) = x := e.toEquiv.symm_apply_apply x @[to_additive (attr := simp)] theorem symm_comp_self (e : M ≃* N) : e.symm ∘ e = id := funext e.symm_apply_apply @[to_additive (attr := simp)] theorem self_comp_symm (e : M ≃* N) : e ∘ e.symm = id := funext e.apply_symm_apply @[to_additive (attr := simp)] theorem coe_refl : ↑(refl M) = id := rfl @[to_additive (attr := simp)] theorem refl_apply (m : M) : refl M m = m := rfl @[to_additive (attr := simp)] theorem coe_trans (e₁ : M ≃* N) (e₂ : N ≃* P) : ↑(e₁.trans e₂) = e₂ ∘ e₁ := rfl @[to_additive (attr := simp)] theorem trans_apply (e₁ : M ≃* N) (e₂ : N ≃* P) (m : M) : e₁.trans e₂ m = e₂ (e₁ m) := rfl @[to_additive (attr := simp)] theorem symm_trans_apply (e₁ : M ≃* N) (e₂ : N ≃* P) (p : P) : (e₁.trans e₂).symm p = e₁.symm (e₂.symm p) := rfl -- Porting note (#10618): `simp` can prove this @[to_additive] theorem apply_eq_iff_eq (e : M ≃* N) {x y : M} : e x = e y ↔ x = y := e.injective.eq_iff @[to_additive] theorem apply_eq_iff_symm_apply (e : M ≃* N) {x : M} {y : N} : e x = y ↔ x = e.symm y := e.toEquiv.apply_eq_iff_eq_symm_apply @[to_additive] theorem symm_apply_eq (e : M ≃* N) {x y} : e.symm x = y ↔ x = e y := e.toEquiv.symm_apply_eq @[to_additive] theorem eq_symm_apply (e : M ≃* N) {x y} : y = e.symm x ↔ e y = x := e.toEquiv.eq_symm_apply @[to_additive] theorem eq_comp_symm {α : Type*} (e : M ≃* N) (f : N → α) (g : M → α) : f = g ∘ e.symm ↔ f ∘ e = g := e.toEquiv.eq_comp_symm f g @[to_additive] theorem comp_symm_eq {α : Type*} (e : M ≃* N) (f : N → α) (g : M → α) : g ∘ e.symm = f ↔ g = f ∘ e := e.toEquiv.comp_symm_eq f g @[to_additive] theorem eq_symm_comp {α : Type*} (e : M ≃* N) (f : α → M) (g : α → N) : f = e.symm ∘ g ↔ e ∘ f = g := e.toEquiv.eq_symm_comp f g @[to_additive] theorem symm_comp_eq {α : Type*} (e : M ≃* N) (f : α → M) (g : α → N) : e.symm ∘ g = f ↔ g = e ∘ f := e.toEquiv.symm_comp_eq f g @[to_additive (attr := simp)] theorem symm_trans_self (e : M ≃* N) : e.symm.trans e = refl N := DFunLike.ext _ _ e.apply_symm_apply @[to_additive (attr := simp)] theorem self_trans_symm (e : M ≃* N) : e.trans e.symm = refl M := DFunLike.ext _ _ e.symm_apply_apply /-- Two multiplicative isomorphisms agree if they are defined by the same underlying function. -/ @[to_additive (attr := ext) "Two additive isomorphisms agree if they are defined by the same underlying function."] theorem ext {f g : MulEquiv M N} (h : ∀ x, f x = g x) : f = g := DFunLike.ext f g h @[to_additive (attr := simp)] theorem mk_coe (e : M ≃* N) (e' h₁ h₂ h₃) : (⟨⟨e, e', h₁, h₂⟩, h₃⟩ : M ≃* N) = e := ext fun _ => rfl @[to_additive (attr := simp)] theorem mk_coe' (e : M ≃* N) (f h₁ h₂ h₃) : (MulEquiv.mk ⟨f, e, h₁, h₂⟩ h₃ : N ≃* M) = e.symm := symm_bijective.injective <| ext fun _ => rfl @[to_additive] protected theorem congr_arg {f : MulEquiv M N} {x x' : M} : x = x' → f x = f x' := DFunLike.congr_arg f @[to_additive] protected theorem congr_fun {f g : MulEquiv M N} (h : f = g) (x : M) : f x = g x := DFunLike.congr_fun h x /-- The `MulEquiv` between two monoids with a unique element. -/ @[to_additive "The `AddEquiv` between two `AddMonoid`s with a unique element."] def mulEquivOfUnique {M N} [Unique M] [Unique N] [Mul M] [Mul N] : M ≃* N := { Equiv.equivOfUnique M N with map_mul' := fun _ _ => Subsingleton.elim _ _ } /-- There is a unique monoid homomorphism between two monoids with a unique element. -/ @[to_additive "There is a unique additive monoid homomorphism between two additive monoids with a unique element."] instance {M N} [Unique M] [Unique N] [Mul M] [Mul N] : Unique (M ≃* N) where default := mulEquivOfUnique uniq _ := ext fun _ => Subsingleton.elim _ _ end Mul /-! ## Monoids -/ section MulOneClass variable [MulOneClass M] [MulOneClass N] [MulOneClass P] -- Porting note (#10618): `simp` can prove this @[to_additive] theorem coe_monoidHom_refl : (refl M : M →* M) = MonoidHom.id M := rfl -- Porting note (#10618): `simp` can prove this @[to_additive] lemma coe_monoidHom_trans (e₁ : M ≃* N) (e₂ : N ≃* P) : (e₁.trans e₂ : M →* P) = (e₂ : N →* P).comp ↑e₁ := rfl @[to_additive (attr := simp)] lemma coe_monoidHom_comp_coe_monoidHom_symm (e : M ≃* N) : (e : M →* N).comp e.symm = MonoidHom.id _ := by ext; simp @[to_additive (attr := simp)] lemma coe_monoidHom_symm_comp_coe_monoidHom (e : M ≃* N) : (e.symm : N →* M).comp e = MonoidHom.id _ := by ext; simp @[to_additive] lemma comp_left_injective (e : M ≃* N) : Injective fun f : N →* P ↦ f.comp (e : M →* N) := LeftInverse.injective (g := fun f ↦ f.comp e.symm) fun f ↦ by simp [MonoidHom.comp_assoc] @[to_additive] lemma comp_right_injective (e : M ≃* N) : Injective fun f : P →* M ↦ (e : M →* N).comp f := LeftInverse.injective (g := (e.symm : N →* M).comp) fun f ↦ by simp [← MonoidHom.comp_assoc] /-- A multiplicative isomorphism of monoids sends `1` to `1` (and is hence a monoid isomorphism). -/ @[to_additive "An additive isomorphism of additive monoids sends `0` to `0` (and is hence an additive monoid isomorphism)."] protected theorem map_one (h : M ≃* N) : h 1 = 1 := _root_.map_one h @[to_additive] protected theorem map_eq_one_iff (h : M ≃* N) {x : M} : h x = 1 ↔ x = 1 := MulEquivClass.map_eq_one_iff h @[to_additive] theorem map_ne_one_iff (h : M ≃* N) {x : M} : h x ≠ 1 ↔ x ≠ 1 := MulEquivClass.map_ne_one_iff h /-- A bijective `Semigroup` homomorphism is an isomorphism -/ @[to_additive (attr := simps! apply) "A bijective `AddSemigroup` homomorphism is an isomorphism"] noncomputable def ofBijective {M N F} [Mul M] [Mul N] [FunLike F M N] [MulHomClass F M N] (f : F) (hf : Bijective f) : M ≃* N := { Equiv.ofBijective f hf with map_mul' := map_mul f } -- Porting note (#11215): TODO: simplify `symm_apply` to `surjInv`? @[to_additive (attr := simp)] theorem ofBijective_apply_symm_apply {n : N} (f : M →* N) (hf : Bijective f) : f ((ofBijective f hf).symm n) = n := (ofBijective f hf).apply_symm_apply n /-- Extract the forward direction of a multiplicative equivalence as a multiplication-preserving function. -/ @[to_additive "Extract the forward direction of an additive equivalence as an addition-preserving function."] def toMonoidHom (h : M ≃* N) : M →* N := { h with map_one' := h.map_one } @[to_additive (attr := simp)] theorem coe_toMonoidHom (e : M ≃* N) : ⇑e.toMonoidHom = e := rfl @[to_additive (attr := simp)] theorem toMonoidHom_eq_coe (f : M ≃* N) : f.toMonoidHom = (f : M →* N) := rfl @[to_additive] theorem toMonoidHom_injective : Injective (toMonoidHom : M ≃* N → M →* N) := Injective.of_comp (f := DFunLike.coe) DFunLike.coe_injective end MulOneClass /-- A multiplicative analogue of `Equiv.arrowCongr`, where the equivalence between the targets is multiplicative. -/ @[to_additive (attr := simps apply) "An additive analogue of `Equiv.arrowCongr`, where the equivalence between the targets is additive."] def arrowCongr {M N P Q : Type*} [Mul P] [Mul Q] (f : M ≃ N) (g : P ≃* Q) : (M → P) ≃* (N → Q) where toFun h n := g (h (f.symm n)) invFun k m := g.symm (k (f m)) left_inv h := by ext; simp right_inv k := by ext; simp map_mul' h k := by ext; simp /-- A multiplicative analogue of `Equiv.arrowCongr`, for multiplicative maps from a monoid to a commutative monoid. -/ @[to_additive (attr := simps apply) "An additive analogue of `Equiv.arrowCongr`, for additive maps from an additive monoid to a commutative additive monoid."] -- Porting note: @[simps apply] removed because it was making a lemma which -- wasn't in simp normal form. def monoidHomCongr {M N P Q} [MulOneClass M] [MulOneClass N] [CommMonoid P] [CommMonoid Q] (f : M ≃* N) (g : P ≃* Q) : (M →* P) ≃* (N →* Q) where toFun h := g.toMonoidHom.comp (h.comp f.symm.toMonoidHom) invFun k := g.symm.toMonoidHom.comp (k.comp f.toMonoidHom) left_inv h := by ext; simp right_inv k := by ext; simp map_mul' h k := by ext; simp /-- A family of multiplicative equivalences `Π j, (Ms j ≃* Ns j)` generates a multiplicative equivalence between `Π j, Ms j` and `Π j, Ns j`. This is the `MulEquiv` version of `Equiv.piCongrRight`, and the dependent version of `MulEquiv.arrowCongr`. -/ @[to_additive (attr := simps apply) "A family of additive equivalences `Π j, (Ms j ≃+ Ns j)` generates an additive equivalence between `Π j, Ms j` and `Π j, Ns j`. This is the `AddEquiv` version of `Equiv.piCongrRight`, and the dependent version of `AddEquiv.arrowCongr`."] def piCongrRight {η : Type*} {Ms Ns : η → Type*} [∀ j, Mul (Ms j)] [∀ j, Mul (Ns j)] (es : ∀ j, Ms j ≃* Ns j) : (∀ j, Ms j) ≃* ∀ j, Ns j := { Equiv.piCongrRight fun j => (es j).toEquiv with toFun := fun x j => es j (x j), invFun := fun x j => (es j).symm (x j), map_mul' := fun x y => funext fun j => (es j).map_mul (x j) (y j) } @[to_additive (attr := simp)] theorem piCongrRight_refl {η : Type*} {Ms : η → Type*} [∀ j, Mul (Ms j)] : (piCongrRight fun j => MulEquiv.refl (Ms j)) = MulEquiv.refl _ := rfl @[to_additive (attr := simp)] theorem piCongrRight_symm {η : Type*} {Ms Ns : η → Type*} [∀ j, Mul (Ms j)] [∀ j, Mul (Ns j)] (es : ∀ j, Ms j ≃* Ns j) : (piCongrRight es).symm = piCongrRight fun i => (es i).symm := rfl @[to_additive (attr := simp)] theorem piCongrRight_trans {η : Type*} {Ms Ns Ps : η → Type*} [∀ j, Mul (Ms j)] [∀ j, Mul (Ns j)] [∀ j, Mul (Ps j)] (es : ∀ j, Ms j ≃* Ns j) (fs : ∀ j, Ns j ≃* Ps j) : (piCongrRight es).trans (piCongrRight fs) = piCongrRight fun i => (es i).trans (fs i) := rfl /-- A family indexed by a type with a unique element is `MulEquiv` to the element at the single index. -/ @[to_additive (attr := simps!) "A family indexed by a type with a unique element is `AddEquiv` to the element at the single index."] def piUnique {ι : Type*} (M : ι → Type*) [∀ j, Mul (M j)] [Unique ι] : (∀ j, M j) ≃* M default := { Equiv.piUnique M with map_mul' := fun _ _ => Pi.mul_apply _ _ _ } /-! # Groups -/ /-- A multiplicative equivalence of groups preserves inversion. -/ @[to_additive "An additive equivalence of additive groups preserves negation."] protected theorem map_inv [Group G] [DivisionMonoid H] (h : G ≃* H) (x : G) : h x⁻¹ = (h x)⁻¹ := _root_.map_inv h x /-- A multiplicative equivalence of groups preserves division. -/ @[to_additive "An additive equivalence of additive groups preserves subtractions."] protected theorem map_div [Group G] [DivisionMonoid H] (h : G ≃* H) (x y : G) : h (x / y) = h x / h y := _root_.map_div h x y end MulEquiv -- Porting note: we want to add -- `@[simps (config := .asFn)]` -- here, but it generates simp lemmas which aren't in simp normal form -- (they have `toFun` in) /-- Given a pair of multiplicative homomorphisms `f`, `g` such that `g.comp f = id` and `f.comp g = id`, returns a multiplicative equivalence with `toFun = f` and `invFun = g`. This constructor is useful if the underlying type(s) have specialized `ext` lemmas for multiplicative homomorphisms. -/ @[to_additive "Given a pair of additive homomorphisms `f`, `g` such that `g.comp f = id` and `f.comp g = id`, returns an additive equivalence with `toFun = f` and `invFun = g`. This constructor is useful if the underlying type(s) have specialized `ext` lemmas for additive homomorphisms."] def MulHom.toMulEquiv [Mul M] [Mul N] (f : M →ₙ* N) (g : N →ₙ* M) (h₁ : g.comp f = MulHom.id _) (h₂ : f.comp g = MulHom.id _) : M ≃* N where toFun := f invFun := g left_inv := DFunLike.congr_fun h₁ right_inv := DFunLike.congr_fun h₂ map_mul' := f.map_mul -- Porting note: the next two lemmas were added manually because `@[simps]` is generating -- lemmas with `toFun` in @[to_additive (attr := simp)] theorem MulHom.toMulEquiv_apply [Mul M] [Mul N] (f : M →ₙ* N) (g : N →ₙ* M) (h₁ : g.comp f = MulHom.id _) (h₂ : f.comp g = MulHom.id _) : ((MulHom.toMulEquiv f g h₁ h₂) : M → N) = f := rfl @[to_additive (attr := simp)] theorem MulHom.toMulEquiv_symm_apply [Mul M] [Mul N] (f : M →ₙ* N) (g : N →ₙ* M) (h₁ : g.comp f = MulHom.id _) (h₂ : f.comp g = MulHom.id _) : (MulEquiv.symm (MulHom.toMulEquiv f g h₁ h₂) : N → M) = ↑g := rfl /-- Given a pair of monoid homomorphisms `f`, `g` such that `g.comp f = id` and `f.comp g = id`, returns a multiplicative equivalence with `toFun = f` and `invFun = g`. This constructor is useful if the underlying type(s) have specialized `ext` lemmas for monoid homomorphisms. -/ @[to_additive (attr := simps (config := .asFn)) "Given a pair of additive monoid homomorphisms `f`, `g` such that `g.comp f = id` and `f.comp g = id`, returns an additive equivalence with `toFun = f` and `invFun = g`. This constructor is useful if the underlying type(s) have specialized `ext` lemmas for additive monoid homomorphisms."] def MonoidHom.toMulEquiv [MulOneClass M] [MulOneClass N] (f : M →* N) (g : N →* M) (h₁ : g.comp f = MonoidHom.id _) (h₂ : f.comp g = MonoidHom.id _) : M ≃* N where toFun := f invFun := g left_inv := DFunLike.congr_fun h₁ right_inv := DFunLike.congr_fun h₂ map_mul' := f.map_mul namespace Equiv section InvolutiveInv variable (G) [InvolutiveInv G] /-- Inversion on a `Group` or `GroupWithZero` is a permutation of the underlying type. -/ @[to_additive (attr := simps! (config := .asFn) apply) "Negation on an `AddGroup` is a permutation of the underlying type."] protected def inv : Perm G := inv_involutive.toPerm _ variable {G} @[to_additive (attr := simp)] theorem inv_symm : (Equiv.inv G).symm = Equiv.inv G := rfl end InvolutiveInv end Equiv
Algebra\Group\Equiv\TypeTags.lean
/- Copyright (c) 2018 Johannes Hölzl. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Johannes Hölzl, Callum Sutton, Yury Kudryashov -/ import Mathlib.Algebra.Group.Equiv.Basic import Mathlib.Algebra.Group.TypeTags /-! # Additive and multiplicative equivalences associated to `Multiplicative` and `Additive`. -/ variable {G H : Type*} /-- Reinterpret `G ≃+ H` as `Multiplicative G ≃* Multiplicative H`. -/ @[simps] def AddEquiv.toMultiplicative [AddZeroClass G] [AddZeroClass H] : G ≃+ H ≃ (Multiplicative G ≃* Multiplicative H) where toFun f := { toFun := AddMonoidHom.toMultiplicative f.toAddMonoidHom invFun := AddMonoidHom.toMultiplicative f.symm.toAddMonoidHom left_inv := f.left_inv right_inv := f.right_inv map_mul' := f.map_add } invFun f := { toFun := AddMonoidHom.toMultiplicative.symm f.toMonoidHom invFun := AddMonoidHom.toMultiplicative.symm f.symm.toMonoidHom left_inv := f.left_inv right_inv := f.right_inv map_add' := f.map_mul } left_inv x := by ext; rfl right_inv x := by ext; rfl /-- Reinterpret `G ≃* H` as `Additive G ≃+ Additive H`. -/ @[simps] def MulEquiv.toAdditive [MulOneClass G] [MulOneClass H] : G ≃* H ≃ (Additive G ≃+ Additive H) where toFun f := { toFun := MonoidHom.toAdditive f.toMonoidHom invFun := MonoidHom.toAdditive f.symm.toMonoidHom left_inv := f.left_inv right_inv := f.right_inv map_add' := f.map_mul } invFun f := { toFun := MonoidHom.toAdditive.symm f.toAddMonoidHom invFun := MonoidHom.toAdditive.symm f.symm.toAddMonoidHom left_inv := f.left_inv right_inv := f.right_inv map_mul' := f.map_add } left_inv x := by ext; rfl right_inv x := by ext; rfl /-- Reinterpret `Additive G ≃+ H` as `G ≃* Multiplicative H`. -/ @[simps] def AddEquiv.toMultiplicative' [MulOneClass G] [AddZeroClass H] : Additive G ≃+ H ≃ (G ≃* Multiplicative H) where toFun f := { toFun := AddMonoidHom.toMultiplicative' f.toAddMonoidHom invFun := AddMonoidHom.toMultiplicative'' f.symm.toAddMonoidHom left_inv := f.left_inv right_inv := f.right_inv map_mul' := f.map_add } invFun f := { toFun := AddMonoidHom.toMultiplicative'.symm f.toMonoidHom invFun := AddMonoidHom.toMultiplicative''.symm f.symm.toMonoidHom left_inv := f.left_inv right_inv := f.right_inv map_add' := f.map_mul } left_inv x := by ext; rfl right_inv x := by ext; rfl /-- Reinterpret `G ≃* Multiplicative H` as `Additive G ≃+ H` as. -/ abbrev MulEquiv.toAdditive' [MulOneClass G] [AddZeroClass H] : G ≃* Multiplicative H ≃ (Additive G ≃+ H) := AddEquiv.toMultiplicative'.symm /-- Reinterpret `G ≃+ Additive H` as `Multiplicative G ≃* H`. -/ @[simps] def AddEquiv.toMultiplicative'' [AddZeroClass G] [MulOneClass H] : G ≃+ Additive H ≃ (Multiplicative G ≃* H) where toFun f := { toFun := AddMonoidHom.toMultiplicative'' f.toAddMonoidHom invFun := AddMonoidHom.toMultiplicative' f.symm.toAddMonoidHom left_inv := f.left_inv right_inv := f.right_inv map_mul' := f.map_add } invFun f := { toFun := AddMonoidHom.toMultiplicative''.symm f.toMonoidHom invFun := AddMonoidHom.toMultiplicative'.symm f.symm.toMonoidHom left_inv := f.left_inv right_inv := f.right_inv map_add' := f.map_mul } left_inv x := by ext; rfl right_inv x := by ext; rfl /-- Reinterpret `Multiplicative G ≃* H` as `G ≃+ Additive H` as. -/ abbrev MulEquiv.toAdditive'' [AddZeroClass G] [MulOneClass H] : Multiplicative G ≃* H ≃ (G ≃+ Additive H) := AddEquiv.toMultiplicative''.symm /-- Multiplicative equivalence between multiplicative endomorphisms of a `MulOneClass` `M` and additive endomorphisms of `Additive M`. -/ @[simps!] def monoidEndToAdditive (M : Type*) [MulOneClass M] : Monoid.End M ≃* AddMonoid.End (Additive M) := { MonoidHom.toAdditive with map_mul' := fun _ _ => rfl } /-- Multiplicative equivalence between additive endomorphisms of an `AddZeroClass` `A` and multiplicative endomorphisms of `Multiplicative A`. -/ @[simps!] def addMonoidEndToMultiplicative (A : Type*) [AddZeroClass A] : AddMonoid.End A ≃* Monoid.End (Multiplicative A) := { AddMonoidHom.toMultiplicative with map_mul' := fun _ _ => rfl } section variable (G) (H) /-- `Additive (Multiplicative G)` is just `G`. -/ @[simps!] def AddEquiv.additiveMultiplicative [AddZeroClass G] : Additive (Multiplicative G) ≃+ G := MulEquiv.toAdditive' (MulEquiv.refl (Multiplicative G)) /-- `Multiplicative (Additive H)` is just `H`. -/ @[simps!] def MulEquiv.multiplicativeAdditive [MulOneClass H] : Multiplicative (Additive H) ≃* H := AddEquiv.toMultiplicative'' (AddEquiv.refl (Additive H)) end
Algebra\Group\Fin\Basic.lean
/- Copyright (c) 2021 Yakov Peckersky. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Yakov Peckersky -/ import Mathlib.Algebra.Group.Basic import Mathlib.Algebra.NeZero import Mathlib.Data.Nat.Cast.Defs import Mathlib.Data.Nat.Defs import Mathlib.Data.Fin.Basic /-! # Fin is a group This file contains the additive and multiplicative monoid instances on `Fin n`. See note [foundational algebra order theory]. -/ assert_not_exists OrderedCommMonoid assert_not_exists MonoidWithZero open Nat namespace Fin variable {m n : ℕ} /-! ### Instances -/ instance addCommSemigroup (n : ℕ) : AddCommSemigroup (Fin n) where add_assoc := by simp [Fin.ext_iff, add_def, Nat.add_assoc] add_comm := by simp [Fin.ext_iff, add_def, Nat.add_comm] instance (n) : AddCommSemigroup (Fin n) where add_assoc := by simp [Fin.ext_iff, add_def, Nat.add_assoc] add_comm := by simp [Fin.ext_iff, add_def, add_comm] instance addCommMonoid (n : ℕ) [NeZero n] : AddCommMonoid (Fin n) where zero_add := Fin.zero_add add_zero := Fin.add_zero nsmul := nsmulRec __ := Fin.addCommSemigroup n instance instAddMonoidWithOne (n) [NeZero n] : AddMonoidWithOne (Fin n) where __ := inferInstanceAs (AddCommMonoid (Fin n)) natCast n := Fin.ofNat'' n natCast_zero := rfl natCast_succ _ := Fin.ext (add_mod _ _ _) instance addCommGroup (n : ℕ) [NeZero n] : AddCommGroup (Fin n) where __ := addCommMonoid n __ := neg n add_left_neg := fun ⟨a, ha⟩ ↦ Fin.ext <| (Nat.mod_add_mod _ _ _).trans <| by rw [Fin.val_zero', Nat.sub_add_cancel, Nat.mod_self] exact le_of_lt ha sub := Fin.sub sub_eq_add_neg := fun ⟨a, ha⟩ ⟨b, hb⟩ ↦ Fin.ext <| by simp [Fin.sub_def, Fin.neg_def, Fin.add_def, Nat.add_comm] zsmul := zsmulRec /-- Note this is more general than `Fin.addCommGroup` as it applies (vacuously) to `Fin 0` too. -/ instance instInvolutiveNeg (n : ℕ) : InvolutiveNeg (Fin n) where neg_neg := Nat.casesOn n finZeroElim fun _i ↦ neg_neg /-- Note this is more general than `Fin.addCommGroup` as it applies (vacuously) to `Fin 0` too. -/ instance instIsCancelAdd (n : ℕ) : IsCancelAdd (Fin n) where add_left_cancel := Nat.casesOn n finZeroElim fun _i _ _ _ ↦ add_left_cancel add_right_cancel := Nat.casesOn n finZeroElim fun _i _ _ _ ↦ add_right_cancel /-- Note this is more general than `Fin.addCommGroup` as it applies (vacuously) to `Fin 0` too. -/ instance instAddLeftCancelSemigroup (n : ℕ) : AddLeftCancelSemigroup (Fin n) := { Fin.addCommSemigroup n, Fin.instIsCancelAdd n with } /-- Note this is more general than `Fin.addCommGroup` as it applies (vacuously) to `Fin 0` too. -/ instance instAddRightCancelSemigroup (n : ℕ) : AddRightCancelSemigroup (Fin n) := { Fin.addCommSemigroup n, Fin.instIsCancelAdd n with } /-! ### Miscellaneous lemmas -/ lemma coe_sub_one (a : Fin (n + 1)) : ↑(a - 1) = if a = 0 then n else a - 1 := by cases n · simp split_ifs with h · simp [h] rw [sub_eq_add_neg, val_add_eq_ite, coe_neg_one, if_pos, Nat.add_comm, Nat.add_sub_add_left] conv_rhs => rw [Nat.add_comm] rw [Nat.add_le_add_iff_left, Nat.one_le_iff_ne_zero] rwa [Fin.ext_iff] at h @[simp] lemma lt_sub_one_iff {k : Fin (n + 2)} : k < k - 1 ↔ k = 0 := by rcases k with ⟨_ | k, hk⟩ · simp only [zero_eta, zero_sub, lt_iff_val_lt_val, val_zero, coe_neg_one, zero_lt_succ] have : (n + 1 + (k + 1)) % (n + 2) = k % (n + 2) := by rw [Nat.add_comm, Nat.add_right_comm, Nat.add_assoc, Nat.add_assoc, add_mod_right] simp [lt_iff_val_lt_val, Fin.ext_iff, Fin.coe_sub, this, mod_eq_of_lt ((lt_succ_self _).trans hk)] @[simp] lemma le_sub_one_iff {k : Fin (n + 1)} : k ≤ k - 1 ↔ k = 0 := by cases n · simp [fin_one_eq_zero k] simp [-val_fin_le, le_def] rw [← lt_sub_one_iff, le_iff_lt_or_eq, val_fin_lt, val_inj, lt_sub_one_iff, or_iff_left_iff_imp, eq_comm, sub_eq_iff_eq_add] simp lemma sub_one_lt_iff {k : Fin (n + 1)} : k - 1 < k ↔ 0 < k := not_iff_not.1 <| by simp only [lt_def, not_lt, val_fin_le, le_sub_one_iff, le_zero_iff] @[simp] lemma neg_last (n : ℕ) : -Fin.last n = 1 := by simp [neg_eq_iff_add_eq_zero] lemma neg_natCast_eq_one (n : ℕ) : -(n : Fin (n + 1)) = 1 := by simp only [natCast_eq_last, neg_last] end Fin
Algebra\Group\Fin\Tuple.lean
/- Copyright (c) 2019 Floris van Doorn. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Floris van Doorn, Yury Kudryashov, Sébastien Gouëzel, Chris Hughes -/ import Mathlib.Algebra.Group.Basic import Mathlib.Algebra.Group.Pi.Basic import Mathlib.Data.Fin.VecNotation /-! # Algebraic properties of tuples -/ namespace Fin variable {m n : ℕ} {α : Fin (n + 1) → Type*} @[to_additive (attr := simp)] lemma insertNth_one_right [∀ j, One (α j)] (i : Fin (n + 1)) (x : α i) : i.insertNth x 1 = Pi.mulSingle i x := insertNth_eq_iff.2 <| by unfold removeNth; simp [succAbove_ne, Pi.one_def] @[to_additive (attr := simp)] lemma insertNth_mul [∀ j, Mul (α j)] (i : Fin (n + 1)) (x y : α i) (p q : ∀ j, α (i.succAbove j)) : i.insertNth (x * y) (p * q) = i.insertNth x p * i.insertNth y q := insertNth_binop (fun _ ↦ (· * ·)) i x y p q @[to_additive (attr := simp)] lemma insertNth_div [∀ j, Div (α j)] (i : Fin (n + 1)) (x y : α i)(p q : ∀ j, α (i.succAbove j)) : i.insertNth (x / y) (p / q) = i.insertNth x p / i.insertNth y q := insertNth_binop (fun _ ↦ (· / ·)) i x y p q @[to_additive (attr := simp)] lemma insertNth_div_same [∀ j, Group (α j)] (i : Fin (n + 1)) (x y : α i) (p : ∀ j, α (i.succAbove j)) : i.insertNth x p / i.insertNth y p = Pi.mulSingle i (x / y) := by simp_rw [← insertNth_div, ← insertNth_one_right, Pi.div_def, div_self', Pi.one_def] end Fin namespace Matrix variable {α M : Type*} {n : ℕ} section SMul variable [SMul M α] @[simp] lemma smul_empty (x : M) (v : Fin 0 → α) : x • v = ![] := empty_eq _ @[simp] lemma smul_cons (x : M) (y : α) (v : Fin n → α) : x • vecCons y v = vecCons (x • y) (x • v) := by ext i; refine i.cases ?_ ?_ <;> simp end SMul section Add variable [Add α] @[simp] lemma empty_add_empty (v w : Fin 0 → α) : v + w = ![] := empty_eq _ @[simp] lemma cons_add (x : α) (v : Fin n → α) (w : Fin n.succ → α) : vecCons x v + w = vecCons (x + vecHead w) (v + vecTail w) := by ext i; refine i.cases ?_ ?_ <;> simp [vecHead, vecTail] @[simp] lemma add_cons (v : Fin n.succ → α) (y : α) (w : Fin n → α) : v + vecCons y w = vecCons (vecHead v + y) (vecTail v + w) := by ext i; refine i.cases ?_ ?_ <;> simp [vecHead, vecTail] lemma cons_add_cons (x : α) (v : Fin n → α) (y : α) (w : Fin n → α) : vecCons x v + vecCons y w = vecCons (x + y) (v + w) := by simp @[simp] lemma head_add (a b : Fin n.succ → α) : vecHead (a + b) = vecHead a + vecHead b := rfl @[simp] lemma tail_add (a b : Fin n.succ → α) : vecTail (a + b) = vecTail a + vecTail b := rfl end Add section Sub variable [Sub α] @[simp] lemma empty_sub_empty (v w : Fin 0 → α) : v - w = ![] := empty_eq _ @[simp] lemma cons_sub (x : α) (v : Fin n → α) (w : Fin n.succ → α) : vecCons x v - w = vecCons (x - vecHead w) (v - vecTail w) := by ext i; refine i.cases ?_ ?_ <;> simp [vecHead, vecTail] @[simp] lemma sub_cons (v : Fin n.succ → α) (y : α) (w : Fin n → α) : v - vecCons y w = vecCons (vecHead v - y) (vecTail v - w) := by ext i; refine i.cases ?_ ?_ <;> simp [vecHead, vecTail] lemma cons_sub_cons (x : α) (v : Fin n → α) (y : α) (w : Fin n → α) : vecCons x v - vecCons y w = vecCons (x - y) (v - w) := by simp @[simp] lemma head_sub (a b : Fin n.succ → α) : vecHead (a - b) = vecHead a - vecHead b := rfl @[simp] lemma tail_sub (a b : Fin n.succ → α) : vecTail (a - b) = vecTail a - vecTail b := rfl end Sub section Zero variable [Zero α] @[simp] lemma zero_empty : (0 : Fin 0 → α) = ![] := empty_eq _ @[simp] lemma cons_zero_zero : vecCons (0 : α) (0 : Fin n → α) = 0 := by ext i; exact i.cases rfl (by simp) @[simp] lemma head_zero : vecHead (0 : Fin n.succ → α) = 0 := rfl @[simp] lemma tail_zero : vecTail (0 : Fin n.succ → α) = 0 := rfl @[simp] lemma cons_eq_zero_iff {v : Fin n → α} {x : α} : vecCons x v = 0 ↔ x = 0 ∧ v = 0 where mp h := ⟨congr_fun h 0, by convert congr_arg vecTail h⟩ mpr := fun ⟨hx, hv⟩ ↦ by simp [hx, hv] lemma cons_nonzero_iff {v : Fin n → α} {x : α} : vecCons x v ≠ 0 ↔ x ≠ 0 ∨ v ≠ 0 where mp h := not_and_or.mp (h ∘ cons_eq_zero_iff.mpr) mpr h := mt cons_eq_zero_iff.mp (not_and_or.mpr h) end Zero section Neg variable [Neg α] @[simp] lemma neg_empty (v : Fin 0 → α) : -v = ![] := empty_eq _ @[simp] lemma neg_cons (x : α) (v : Fin n → α) : -vecCons x v = vecCons (-x) (-v) := by ext i; refine i.cases ?_ ?_ <;> simp @[simp] lemma head_neg (a : Fin n.succ → α) : vecHead (-a) = -vecHead a := rfl @[simp] lemma tail_neg (a : Fin n.succ → α) : vecTail (-a) = -vecTail a := rfl end Neg end Matrix
Algebra\Group\Hom\Basic.lean
/- Copyright (c) 2018 Patrick Massot. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Patrick Massot, Kevin Buzzard, Scott Morrison, Johan Commelin, Chris Hughes, Johannes Hölzl, Yury Kudryashov -/ import Mathlib.Algebra.Group.Basic import Mathlib.Algebra.Group.Hom.Defs /-! # Additional lemmas about monoid and group homomorphisms -/ -- `NeZero` cannot be additivised, hence its theory should be developed outside of the -- `Algebra.Group` folder. assert_not_exists NeZero variable {α β M N P : Type*} -- monoids variable {G : Type*} {H : Type*} -- groups variable {F : Type*} section CommMonoid variable [CommMonoid α] /-- The `n`th power map on a commutative monoid for a natural `n`, considered as a morphism of monoids. -/ @[to_additive (attr := simps) "Multiplication by a natural `n` on a commutative additive monoid, considered as a morphism of additive monoids."] def powMonoidHom (n : ℕ) : α →* α where toFun := (· ^ n) map_one' := one_pow _ map_mul' a b := mul_pow a b n end CommMonoid section DivisionCommMonoid variable [DivisionCommMonoid α] /-- The `n`-th power map (for an integer `n`) on a commutative group, considered as a group homomorphism. -/ @[to_additive (attr := simps) "Multiplication by an integer `n` on a commutative additive group, considered as an additive group homomorphism."] def zpowGroupHom (n : ℤ) : α →* α where toFun := (· ^ n) map_one' := one_zpow n map_mul' a b := mul_zpow a b n /-- Inversion on a commutative group, considered as a monoid homomorphism. -/ @[to_additive "Negation on a commutative additive group, considered as an additive monoid homomorphism."] def invMonoidHom : α →* α where toFun := Inv.inv map_one' := inv_one map_mul' := mul_inv @[simp] theorem coe_invMonoidHom : (invMonoidHom : α → α) = Inv.inv := rfl @[simp] theorem invMonoidHom_apply (a : α) : invMonoidHom a = a⁻¹ := rfl end DivisionCommMonoid namespace MulHom /-- Given two mul morphisms `f`, `g` to a commutative semigroup, `f * g` is the mul morphism sending `x` to `f x * g x`. -/ @[to_additive "Given two additive morphisms `f`, `g` to an additive commutative semigroup, `f + g` is the additive morphism sending `x` to `f x + g x`."] instance [Mul M] [CommSemigroup N] : Mul (M →ₙ* N) := ⟨fun f g => { toFun := fun m => f m * g m, map_mul' := fun x y => by show f (x * y) * g (x * y) = f x * g x * (f y * g y) rw [f.map_mul, g.map_mul, ← mul_assoc, ← mul_assoc, mul_right_comm (f x)] }⟩ @[to_additive (attr := simp)] theorem mul_apply {M N} [Mul M] [CommSemigroup N] (f g : M →ₙ* N) (x : M) : (f * g) x = f x * g x := rfl @[to_additive] theorem mul_comp [Mul M] [Mul N] [CommSemigroup P] (g₁ g₂ : N →ₙ* P) (f : M →ₙ* N) : (g₁ * g₂).comp f = g₁.comp f * g₂.comp f := rfl @[to_additive] theorem comp_mul [Mul M] [CommSemigroup N] [CommSemigroup P] (g : N →ₙ* P) (f₁ f₂ : M →ₙ* N) : g.comp (f₁ * f₂) = g.comp f₁ * g.comp f₂ := by ext simp only [mul_apply, Function.comp_apply, map_mul, coe_comp] end MulHom namespace MonoidHom section Group variable [Group G] [CommGroup H] /-- A homomorphism from a group to a monoid is injective iff its kernel is trivial. For the iff statement on the triviality of the kernel, see `injective_iff_map_eq_one'`. -/ @[to_additive "A homomorphism from an additive group to an additive monoid is injective iff its kernel is trivial. For the iff statement on the triviality of the kernel, see `injective_iff_map_eq_zero'`."] theorem _root_.injective_iff_map_eq_one {G H} [Group G] [MulOneClass H] [FunLike F G H] [MonoidHomClass F G H] (f : F) : Function.Injective f ↔ ∀ a, f a = 1 → a = 1 := ⟨fun h x => (map_eq_one_iff f h).mp, fun h x y hxy => mul_inv_eq_one.1 <| h _ <| by rw [map_mul, hxy, ← map_mul, mul_inv_self, map_one]⟩ /-- A homomorphism from a group to a monoid is injective iff its kernel is trivial, stated as an iff on the triviality of the kernel. For the implication, see `injective_iff_map_eq_one`. -/ @[to_additive "A homomorphism from an additive group to an additive monoid is injective iff its kernel is trivial, stated as an iff on the triviality of the kernel. For the implication, see `injective_iff_map_eq_zero`."] theorem _root_.injective_iff_map_eq_one' {G H} [Group G] [MulOneClass H] [FunLike F G H] [MonoidHomClass F G H] (f : F) : Function.Injective f ↔ ∀ a, f a = 1 ↔ a = 1 := (injective_iff_map_eq_one f).trans <| forall_congr' fun _ => ⟨fun h => ⟨h, fun H => H.symm ▸ map_one f⟩, Iff.mp⟩ variable [MulOneClass M] /-- Makes a group homomorphism from a proof that the map preserves right division `fun x y => x * y⁻¹`. See also `MonoidHom.of_map_div` for a version using `fun x y => x / y`. -/ @[to_additive "Makes an additive group homomorphism from a proof that the map preserves the operation `fun a b => a + -b`. See also `AddMonoidHom.ofMapSub` for a version using `fun a b => a - b`."] def ofMapMulInv {H : Type*} [Group H] (f : G → H) (map_div : ∀ a b : G, f (a * b⁻¹) = f a * (f b)⁻¹) : G →* H := (mk' f) fun x y => calc f (x * y) = f x * (f <| 1 * 1⁻¹ * y⁻¹)⁻¹ := by { simp only [one_mul, inv_one, ← map_div, inv_inv] } _ = f x * f y := by { simp only [map_div] simp only [mul_right_inv, one_mul, inv_inv] } @[to_additive (attr := simp)] theorem coe_of_map_mul_inv {H : Type*} [Group H] (f : G → H) (map_div : ∀ a b : G, f (a * b⁻¹) = f a * (f b)⁻¹) : ↑(ofMapMulInv f map_div) = f := rfl /-- Define a morphism of additive groups given a map which respects ratios. -/ @[to_additive "Define a morphism of additive groups given a map which respects difference."] def ofMapDiv {H : Type*} [Group H] (f : G → H) (hf : ∀ x y, f (x / y) = f x / f y) : G →* H := ofMapMulInv f (by simpa only [div_eq_mul_inv] using hf) @[to_additive (attr := simp)] theorem coe_of_map_div {H : Type*} [Group H] (f : G → H) (hf : ∀ x y, f (x / y) = f x / f y) : ↑(ofMapDiv f hf) = f := rfl end Group section Mul variable [MulOneClass M] [CommMonoid N] /-- Given two monoid morphisms `f`, `g` to a commutative monoid, `f * g` is the monoid morphism sending `x` to `f x * g x`. -/ @[to_additive] instance mul : Mul (M →* N) := ⟨fun f g => { toFun := fun m => f m * g m, map_one' := show f 1 * g 1 = 1 by simp, map_mul' := fun x y => by show f (x * y) * g (x * y) = f x * g x * (f y * g y) rw [f.map_mul, g.map_mul, ← mul_assoc, ← mul_assoc, mul_right_comm (f x)] }⟩ /-- Given two additive monoid morphisms `f`, `g` to an additive commutative monoid, `f + g` is the additive monoid morphism sending `x` to `f x + g x`. -/ add_decl_doc AddMonoidHom.add @[to_additive (attr := simp)] lemma mul_apply (f g : M →* N) (x : M) : (f * g) x = f x * g x := rfl @[to_additive] lemma mul_comp [MulOneClass P] (g₁ g₂ : M →* N) (f : P →* M) : (g₁ * g₂).comp f = g₁.comp f * g₂.comp f := rfl @[to_additive] lemma comp_mul [CommMonoid P] (g : N →* P) (f₁ f₂ : M →* N) : g.comp (f₁ * f₂) = g.comp f₁ * g.comp f₂ := by ext; simp only [mul_apply, Function.comp_apply, map_mul, coe_comp] end Mul section InvDiv variable [MulOneClass M] [MulOneClass N] [CommGroup G] [CommGroup H] /-- If `f` is a monoid homomorphism to a commutative group, then `f⁻¹` is the homomorphism sending `x` to `(f x)⁻¹`. -/ @[to_additive "If `f` is an additive monoid homomorphism to an additive commutative group, then `-f` is the homomorphism sending `x` to `-(f x)`."] instance : Inv (M →* G) where inv f := mk' (fun g ↦ (f g)⁻¹) fun a b ↦ by simp_rw [← mul_inv, f.map_mul] @[to_additive (attr := simp)] lemma inv_apply (f : M →* G) (x : M) : f⁻¹ x = (f x)⁻¹ := rfl @[to_additive (attr := simp)] theorem inv_comp (φ : N →* G) (ψ : M →* N) : φ⁻¹.comp ψ = (φ.comp ψ)⁻¹ := rfl @[to_additive (attr := simp)] theorem comp_inv (φ : G →* H) (ψ : M →* G) : φ.comp ψ⁻¹ = (φ.comp ψ)⁻¹ := by ext simp only [Function.comp_apply, inv_apply, map_inv, coe_comp] /-- If `f` and `g` are monoid homomorphisms to a commutative group, then `f / g` is the homomorphism sending `x` to `(f x) / (g x)`. -/ @[to_additive "If `f` and `g` are monoid homomorphisms to an additive commutative group, then `f - g` is the homomorphism sending `x` to `(f x) - (g x)`."] instance : Div (M →* G) where div f g := mk' (fun x ↦ f x / g x) fun a b ↦ by simp [div_eq_mul_inv, mul_assoc, mul_left_comm, mul_comm] @[to_additive (attr := simp)] lemma div_apply (f g : M →* G) (x : M) : (f / g) x = f x / g x := rfl @[to_additive (attr := simp)] lemma div_comp (f g : N →* G) (h : M →* N) : (f / g).comp h = f.comp h / g.comp h := rfl @[to_additive (attr := simp)] lemma comp_div (f : G →* H) (g h : M →* G) : f.comp (g / h) = f.comp g / f.comp h := by ext; simp only [Function.comp_apply, div_apply, map_div, coe_comp] end InvDiv end MonoidHom
Algebra\Group\Hom\CompTypeclasses.lean
/- Copyright (c) 2024 Antoine Chambert-Loir. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Antoine Chambert-Loir -/ import Mathlib.Logic.Function.CompTypeclasses import Mathlib.Algebra.Group.Hom.Defs /-! # Propositional typeclasses on several monoid homs This file contains typeclasses used in the definition of equivariant maps, in the spirit what was initially developed by Frédéric Dupuis and Heather Macbeth for linear maps. However, we do not expect that all maps should be guessed automatically, as it happens for linear maps. If `φ`, `ψ`… are monoid homs and `M`, `N`… are monoids, we add two instances: * `MonoidHom.CompTriple φ ψ χ`, which expresses that `ψ.comp φ = χ` * `MonoidHom.IsId φ`, which expresses that `φ = id` Some basic lemmas are proved: * `MonoidHom.CompTriple.comp` asserts `MonoidHom.CompTriple φ ψ (ψ.comp φ)` * `MonoidHom.CompTriple.id_comp` asserts `MonoidHom.CompTriple φ ψ ψ` in the presence of `MonoidHom.IsId φ` * its variant `MonoidHom.CompTriple.comp_id` TODO : * align with RingHomCompTriple * probably rename MonoidHom.CompTriple as MonoidHomCompTriple (or, on the opposite, rename RingHomCompTriple as RingHom.CompTriple) * does one need AddHom.CompTriple ? -/ section MonoidHomCompTriple namespace MonoidHom /-- Class of composing triples -/ class CompTriple {M N P : Type*} [Monoid M] [Monoid N] [Monoid P] (φ : M →* N) (ψ : N →* P) (χ : outParam (M →* P)) : Prop where /-- The maps form a commuting triangle -/ comp_eq : ψ.comp φ = χ attribute [simp] CompTriple.comp_eq namespace CompTriple variable {M' : Type*} [Monoid M'] variable {M N P : Type*} [Monoid M] [Monoid N] [Monoid P] /-- Class of Id maps -/ class IsId (σ : M →* M) : Prop where eq_id : σ = MonoidHom.id M instance instIsId {M : Type*} [Monoid M] : IsId (MonoidHom.id M) where eq_id := rfl instance {σ : M →* M} [h : _root_.CompTriple.IsId σ] : IsId σ where eq_id := by ext; exact _root_.congr_fun h.eq_id _ instance instComp_id {N P : Type*} [Monoid N] [Monoid P] {φ : N →* N} [IsId φ] {ψ : N →* P} : CompTriple φ ψ ψ where comp_eq := by simp only [IsId.eq_id, MonoidHom.comp_id] instance instId_comp {M N : Type*} [Monoid M] [Monoid N] {φ : M →* N} {ψ : N →* N} [IsId ψ] : CompTriple φ ψ φ where comp_eq := by simp only [IsId.eq_id, MonoidHom.id_comp] lemma comp_inv {φ : M →* N} {ψ : N →* M} (h : Function.RightInverse φ ψ) {χ : M →* M} [IsId χ] : CompTriple φ ψ χ where comp_eq := by simp only [IsId.eq_id, ← DFunLike.coe_fn_eq, coe_comp, h.id] rfl instance instRootCompTriple {φ : M →* N} {ψ : N →* P} {χ : M →* P} [κ : CompTriple φ ψ χ] : _root_.CompTriple φ ψ χ where comp_eq := by rw [← MonoidHom.coe_comp, κ.comp_eq] /-- `φ`, `ψ` and `ψ.comp φ` form a `MonoidHom.CompTriple` (to be used with care, because no simplification is done)-/ theorem comp {φ : M →* N} {ψ : N →* P} : CompTriple φ ψ (ψ.comp φ) where comp_eq := rfl lemma comp_apply {φ : M →* N} {ψ : N →* P} {χ : M →* P} (h : CompTriple φ ψ χ) (x : M) : ψ (φ x) = χ x := by rw [← h.comp_eq, MonoidHom.comp_apply] @[simp] theorem comp_assoc {Q : Type*} [Monoid Q] {φ₁ : M →* N} {φ₂ : N →* P} {φ₁₂ : M →* P} (κ : CompTriple φ₁ φ₂ φ₁₂) {φ₃ : P →* Q} {φ₂₃ : N →* Q} (κ' : CompTriple φ₂ φ₃ φ₂₃) {φ₁₂₃ : M →* Q} : CompTriple φ₁ φ₂₃ φ₁₂₃ ↔ CompTriple φ₁₂ φ₃ φ₁₂₃ := by constructor <;> · rintro ⟨h⟩ exact ⟨by simp only [← κ.comp_eq, ← h, ← κ'.comp_eq, MonoidHom.comp_assoc]⟩ end MonoidHom.CompTriple
Algebra\Group\Hom\Defs.lean
/- Copyright (c) 2018 Patrick Massot. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Patrick Massot, Kevin Buzzard, Scott Morrison, Johan Commelin, Chris Hughes, Johannes Hölzl, Yury Kudryashov -/ import Mathlib.Algebra.Group.Pi.Basic import Mathlib.Data.FunLike.Basic import Mathlib.Logic.Function.Iterate /-! # Monoid and group homomorphisms This file defines the bundled structures for monoid and group homomorphisms. Namely, we define `MonoidHom` (resp., `AddMonoidHom`) to be bundled homomorphisms between multiplicative (resp., additive) monoids or groups. We also define coercion to a function, and usual operations: composition, identity homomorphism, pointwise multiplication and pointwise inversion. This file also defines the lesser-used (and notation-less) homomorphism types which are used as building blocks for other homomorphisms: * `ZeroHom` * `OneHom` * `AddHom` * `MulHom` ## Notations * `→+`: Bundled `AddMonoid` homs. Also use for `AddGroup` homs. * `→*`: Bundled `Monoid` homs. Also use for `Group` homs. * `→ₙ*`: Bundled `Semigroup` homs. ## Implementation notes There's a coercion from bundled homs to fun, and the canonical notation is to use the bundled hom as a function via this coercion. There is no `GroupHom` -- the idea is that `MonoidHom` is used. The constructor for `MonoidHom` needs a proof of `map_one` as well as `map_mul`; a separate constructor `MonoidHom.mk'` will construct group homs (i.e. monoid homs between groups) given only a proof that multiplication is preserved, Implicit `{}` brackets are often used instead of type class `[]` brackets. This is done when the instances can be inferred because they are implicit arguments to the type `MonoidHom`. When they can be inferred from the type it is faster to use this method than to use type class inference. Historically this file also included definitions of unbundled homomorphism classes; they were deprecated and moved to `Deprecated/Group`. ## Tags MonoidHom, AddMonoidHom -/ variable {ι α β M N P : Type*} -- monoids variable {G : Type*} {H : Type*} -- groups variable {F : Type*} -- homs section Zero /-- `ZeroHom M N` is the type of functions `M → N` that preserve zero. When possible, instead of parametrizing results over `(f : ZeroHom M N)`, you should parametrize over `(F : Type*) [ZeroHomClass F M N] (f : F)`. When you extend this structure, make sure to also extend `ZeroHomClass`. -/ structure ZeroHom (M : Type*) (N : Type*) [Zero M] [Zero N] where /-- The underlying function -/ protected toFun : M → N /-- The proposition that the function preserves 0 -/ protected map_zero' : toFun 0 = 0 /-- `ZeroHomClass F M N` states that `F` is a type of zero-preserving homomorphisms. You should extend this typeclass when you extend `ZeroHom`. -/ class ZeroHomClass (F : Type*) (M N : outParam Type*) [Zero M] [Zero N] [FunLike F M N] : Prop where /-- The proposition that the function preserves 0 -/ map_zero : ∀ f : F, f 0 = 0 -- Instances and lemmas are defined below through `@[to_additive]`. end Zero section Add /-- `AddHom M N` is the type of functions `M → N` that preserve addition. When possible, instead of parametrizing results over `(f : AddHom M N)`, you should parametrize over `(F : Type*) [AddHomClass F M N] (f : F)`. When you extend this structure, make sure to extend `AddHomClass`. -/ structure AddHom (M : Type*) (N : Type*) [Add M] [Add N] where /-- The underlying function -/ protected toFun : M → N /-- The proposition that the function preserves addition -/ protected map_add' : ∀ x y, toFun (x + y) = toFun x + toFun y /-- `AddHomClass F M N` states that `F` is a type of addition-preserving homomorphisms. You should declare an instance of this typeclass when you extend `AddHom`. -/ class AddHomClass (F : Type*) (M N : outParam Type*) [Add M] [Add N] [FunLike F M N] : Prop where /-- The proposition that the function preserves addition -/ map_add : ∀ (f : F) (x y : M), f (x + y) = f x + f y -- Instances and lemmas are defined below through `@[to_additive]`. end Add section add_zero /-- `M →+ N` is the type of functions `M → N` that preserve the `AddZeroClass` structure. `AddMonoidHom` is also used for group homomorphisms. When possible, instead of parametrizing results over `(f : M →+ N)`, you should parametrize over `(F : Type*) [AddMonoidHomClass F M N] (f : F)`. When you extend this structure, make sure to extend `AddMonoidHomClass`. -/ structure AddMonoidHom (M : Type*) (N : Type*) [AddZeroClass M] [AddZeroClass N] extends ZeroHom M N, AddHom M N attribute [nolint docBlame] AddMonoidHom.toAddHom attribute [nolint docBlame] AddMonoidHom.toZeroHom /-- `M →+ N` denotes the type of additive monoid homomorphisms from `M` to `N`. -/ infixr:25 " →+ " => AddMonoidHom /-- `AddMonoidHomClass F M N` states that `F` is a type of `AddZeroClass`-preserving homomorphisms. You should also extend this typeclass when you extend `AddMonoidHom`. -/ class AddMonoidHomClass (F M N : Type*) [AddZeroClass M] [AddZeroClass N] [FunLike F M N] extends AddHomClass F M N, ZeroHomClass F M N : Prop -- Instances and lemmas are defined below through `@[to_additive]`. end add_zero section One variable [One M] [One N] /-- `OneHom M N` is the type of functions `M → N` that preserve one. When possible, instead of parametrizing results over `(f : OneHom M N)`, you should parametrize over `(F : Type*) [OneHomClass F M N] (f : F)`. When you extend this structure, make sure to also extend `OneHomClass`. -/ @[to_additive] structure OneHom (M : Type*) (N : Type*) [One M] [One N] where /-- The underlying function -/ protected toFun : M → N /-- The proposition that the function preserves 1 -/ protected map_one' : toFun 1 = 1 /-- `OneHomClass F M N` states that `F` is a type of one-preserving homomorphisms. You should extend this typeclass when you extend `OneHom`. -/ @[to_additive] class OneHomClass (F : Type*) (M N : outParam Type*) [One M] [One N] [FunLike F M N] : Prop where /-- The proposition that the function preserves 1 -/ map_one : ∀ f : F, f 1 = 1 @[to_additive] instance OneHom.funLike : FunLike (OneHom M N) M N where coe := OneHom.toFun coe_injective' f g h := by cases f; cases g; congr @[to_additive] instance OneHom.oneHomClass : OneHomClass (OneHom M N) M N where map_one := OneHom.map_one' variable [FunLike F M N] @[to_additive (attr := simp)] theorem map_one [OneHomClass F M N] (f : F) : f 1 = 1 := OneHomClass.map_one f @[to_additive] lemma map_comp_one [OneHomClass F M N] (f : F) : f ∘ (1 : ι → M) = 1 := by simp /-- In principle this could be an instance, but in practice it causes performance issues. -/ @[to_additive] theorem Subsingleton.of_oneHomClass [Subsingleton M] [OneHomClass F M N] : Subsingleton F where allEq f g := DFunLike.ext _ _ fun x ↦ by simp [Subsingleton.elim x 1] @[to_additive] instance [Subsingleton M] : Subsingleton (OneHom M N) := .of_oneHomClass @[to_additive] theorem map_eq_one_iff [OneHomClass F M N] (f : F) (hf : Function.Injective f) {x : M} : f x = 1 ↔ x = 1 := hf.eq_iff' (map_one f) @[to_additive] theorem map_ne_one_iff {R S F : Type*} [One R] [One S] [FunLike F R S] [OneHomClass F R S] (f : F) (hf : Function.Injective f) {x : R} : f x ≠ 1 ↔ x ≠ 1 := (map_eq_one_iff f hf).not @[to_additive] theorem ne_one_of_map {R S F : Type*} [One R] [One S] [FunLike F R S] [OneHomClass F R S] {f : F} {x : R} (hx : f x ≠ 1) : x ≠ 1 := ne_of_apply_ne f <| (by rwa [(map_one f)]) /-- Turn an element of a type `F` satisfying `OneHomClass F M N` into an actual `OneHom`. This is declared as the default coercion from `F` to `OneHom M N`. -/ @[to_additive (attr := coe) "Turn an element of a type `F` satisfying `ZeroHomClass F M N` into an actual `ZeroHom`. This is declared as the default coercion from `F` to `ZeroHom M N`."] def OneHomClass.toOneHom [OneHomClass F M N] (f : F) : OneHom M N where toFun := f map_one' := map_one f /-- Any type satisfying `OneHomClass` can be cast into `OneHom` via `OneHomClass.toOneHom`. -/ @[to_additive "Any type satisfying `ZeroHomClass` can be cast into `ZeroHom` via `ZeroHomClass.toZeroHom`. "] instance [OneHomClass F M N] : CoeTC F (OneHom M N) := ⟨OneHomClass.toOneHom⟩ @[to_additive (attr := simp)] theorem OneHom.coe_coe [OneHomClass F M N] (f : F) : ((f : OneHom M N) : M → N) = f := rfl end One section Mul variable [Mul M] [Mul N] /-- `M →ₙ* N` is the type of functions `M → N` that preserve multiplication. The `ₙ` in the notation stands for "non-unital" because it is intended to match the notation for `NonUnitalAlgHom` and `NonUnitalRingHom`, so a `MulHom` is a non-unital monoid hom. When possible, instead of parametrizing results over `(f : M →ₙ* N)`, you should parametrize over `(F : Type*) [MulHomClass F M N] (f : F)`. When you extend this structure, make sure to extend `MulHomClass`. -/ @[to_additive] structure MulHom (M : Type*) (N : Type*) [Mul M] [Mul N] where /-- The underlying function -/ protected toFun : M → N /-- The proposition that the function preserves multiplication -/ protected map_mul' : ∀ x y, toFun (x * y) = toFun x * toFun y /-- `M →ₙ* N` denotes the type of multiplication-preserving maps from `M` to `N`. -/ infixr:25 " →ₙ* " => MulHom /-- `MulHomClass F M N` states that `F` is a type of multiplication-preserving homomorphisms. You should declare an instance of this typeclass when you extend `MulHom`. -/ @[to_additive] class MulHomClass (F : Type*) (M N : outParam Type*) [Mul M] [Mul N] [FunLike F M N] : Prop where /-- The proposition that the function preserves multiplication -/ map_mul : ∀ (f : F) (x y : M), f (x * y) = f x * f y @[to_additive] instance MulHom.funLike : FunLike (M →ₙ* N) M N where coe := MulHom.toFun coe_injective' f g h := by cases f; cases g; congr /-- `MulHom` is a type of multiplication-preserving homomorphisms -/ @[to_additive "`AddHom` is a type of addition-preserving homomorphisms"] instance MulHom.mulHomClass : MulHomClass (M →ₙ* N) M N where map_mul := MulHom.map_mul' variable [FunLike F M N] @[to_additive (attr := simp)] theorem map_mul [MulHomClass F M N] (f : F) (x y : M) : f (x * y) = f x * f y := MulHomClass.map_mul f x y @[to_additive (attr := simp)] lemma map_comp_mul [MulHomClass F M N] (f : F) (g h : ι → M) : f ∘ (g * h) = f ∘ g * f ∘ h := by ext; simp /-- Turn an element of a type `F` satisfying `MulHomClass F M N` into an actual `MulHom`. This is declared as the default coercion from `F` to `M →ₙ* N`. -/ @[to_additive (attr := coe) "Turn an element of a type `F` satisfying `AddHomClass F M N` into an actual `AddHom`. This is declared as the default coercion from `F` to `M →ₙ+ N`."] def MulHomClass.toMulHom [MulHomClass F M N] (f : F) : M →ₙ* N where toFun := f map_mul' := map_mul f /-- Any type satisfying `MulHomClass` can be cast into `MulHom` via `MulHomClass.toMulHom`. -/ @[to_additive "Any type satisfying `AddHomClass` can be cast into `AddHom` via `AddHomClass.toAddHom`."] instance [MulHomClass F M N] : CoeTC F (M →ₙ* N) := ⟨MulHomClass.toMulHom⟩ @[to_additive (attr := simp)] theorem MulHom.coe_coe [MulHomClass F M N] (f : F) : ((f : MulHom M N) : M → N) = f := rfl end Mul section mul_one variable [MulOneClass M] [MulOneClass N] /-- `M →* N` is the type of functions `M → N` that preserve the `Monoid` structure. `MonoidHom` is also used for group homomorphisms. When possible, instead of parametrizing results over `(f : M →+ N)`, you should parametrize over `(F : Type*) [MonoidHomClass F M N] (f : F)`. When you extend this structure, make sure to extend `MonoidHomClass`. -/ @[to_additive] structure MonoidHom (M : Type*) (N : Type*) [MulOneClass M] [MulOneClass N] extends OneHom M N, M →ₙ* N -- Porting note: remove once `to_additive` is updated -- This is waiting on https://github.com/leanprover-community/mathlib4/issues/660 attribute [to_additive existing] MonoidHom.toMulHom attribute [nolint docBlame] MonoidHom.toMulHom attribute [nolint docBlame] MonoidHom.toOneHom /-- `M →* N` denotes the type of monoid homomorphisms from `M` to `N`. -/ infixr:25 " →* " => MonoidHom /-- `MonoidHomClass F M N` states that `F` is a type of `Monoid`-preserving homomorphisms. You should also extend this typeclass when you extend `MonoidHom`. -/ @[to_additive] class MonoidHomClass (F : Type*) (M N : outParam Type*) [MulOneClass M] [MulOneClass N] [FunLike F M N] extends MulHomClass F M N, OneHomClass F M N : Prop @[to_additive] instance MonoidHom.instFunLike : FunLike (M →* N) M N where coe f := f.toFun coe_injective' f g h := by cases f cases g congr apply DFunLike.coe_injective' exact h @[to_additive] instance MonoidHom.instMonoidHomClass : MonoidHomClass (M →* N) M N where map_mul := MonoidHom.map_mul' map_one f := f.toOneHom.map_one' @[to_additive] instance [Subsingleton M] : Subsingleton (M →* N) := .of_oneHomClass variable [FunLike F M N] /-- Turn an element of a type `F` satisfying `MonoidHomClass F M N` into an actual `MonoidHom`. This is declared as the default coercion from `F` to `M →* N`. -/ @[to_additive (attr := coe) "Turn an element of a type `F` satisfying `AddMonoidHomClass F M N` into an actual `MonoidHom`. This is declared as the default coercion from `F` to `M →+ N`."] def MonoidHomClass.toMonoidHom [MonoidHomClass F M N] (f : F) : M →* N := { (f : M →ₙ* N), (f : OneHom M N) with } /-- Any type satisfying `MonoidHomClass` can be cast into `MonoidHom` via `MonoidHomClass.toMonoidHom`. -/ @[to_additive "Any type satisfying `AddMonoidHomClass` can be cast into `AddMonoidHom` via `AddMonoidHomClass.toAddMonoidHom`."] instance [MonoidHomClass F M N] : CoeTC F (M →* N) := ⟨MonoidHomClass.toMonoidHom⟩ @[to_additive (attr := simp)] theorem MonoidHom.coe_coe [MonoidHomClass F M N] (f : F) : ((f : M →* N) : M → N) = f := rfl @[to_additive] theorem map_mul_eq_one [MonoidHomClass F M N] (f : F) {a b : M} (h : a * b = 1) : f a * f b = 1 := by rw [← map_mul, h, map_one] variable [FunLike F G H] @[to_additive] theorem map_div' [DivInvMonoid G] [DivInvMonoid H] [MonoidHomClass F G H] (f : F) (hf : ∀ a, f a⁻¹ = (f a)⁻¹) (a b : G) : f (a / b) = f a / f b := by rw [div_eq_mul_inv, div_eq_mul_inv, map_mul, hf] @[to_additive] lemma map_comp_div' [DivInvMonoid G] [DivInvMonoid H] [MonoidHomClass F G H] (f : F) (hf : ∀ a, f a⁻¹ = (f a)⁻¹) (g h : ι → G) : f ∘ (g / h) = f ∘ g / f ∘ h := by ext; simp [map_div' f hf] /-- Group homomorphisms preserve inverse. -/ @[to_additive (attr := simp) "Additive group homomorphisms preserve negation."] theorem map_inv [Group G] [DivisionMonoid H] [MonoidHomClass F G H] (f : F) (a : G) : f a⁻¹ = (f a)⁻¹ := eq_inv_of_mul_eq_one_left <| map_mul_eq_one f <| inv_mul_self _ @[to_additive (attr := simp)] lemma map_comp_inv [Group G] [DivisionMonoid H] [MonoidHomClass F G H] (f : F) (g : ι → G) : f ∘ g⁻¹ = (f ∘ g)⁻¹ := by ext; simp /-- Group homomorphisms preserve division. -/ @[to_additive "Additive group homomorphisms preserve subtraction."] theorem map_mul_inv [Group G] [DivisionMonoid H] [MonoidHomClass F G H] (f : F) (a b : G) : f (a * b⁻¹) = f a * (f b)⁻¹ := by rw [map_mul, map_inv] @[to_additive] lemma map_comp_mul_inv [Group G] [DivisionMonoid H] [MonoidHomClass F G H] (f : F) (g h : ι → G) : f ∘ (g * h⁻¹) = f ∘ g * (f ∘ h)⁻¹ := by simp /-- Group homomorphisms preserve division. -/ @[to_additive (attr := simp) "Additive group homomorphisms preserve subtraction."] theorem map_div [Group G] [DivisionMonoid H] [MonoidHomClass F G H] (f : F) : ∀ a b, f (a / b) = f a / f b := map_div' _ <| map_inv f @[to_additive (attr := simp)] lemma map_comp_div [Group G] [DivisionMonoid H] [MonoidHomClass F G H] (f : F) (g h : ι → G) : f ∘ (g / h) = f ∘ g / f ∘ h := by ext; simp @[to_additive (attr := simp) (reorder := 9 10)] theorem map_pow [Monoid G] [Monoid H] [MonoidHomClass F G H] (f : F) (a : G) : ∀ n : ℕ, f (a ^ n) = f a ^ n | 0 => by rw [pow_zero, pow_zero, map_one] | n + 1 => by rw [pow_succ, pow_succ, map_mul, map_pow f a n] @[to_additive (attr := simp)] lemma map_comp_pow [Group G] [DivisionMonoid H] [MonoidHomClass F G H] (f : F) (g : ι → G) (n : ℕ) : f ∘ (g ^ n) = f ∘ g ^ n := by ext; simp @[to_additive] theorem map_zpow' [DivInvMonoid G] [DivInvMonoid H] [MonoidHomClass F G H] (f : F) (hf : ∀ x : G, f x⁻¹ = (f x)⁻¹) (a : G) : ∀ n : ℤ, f (a ^ n) = f a ^ n | (n : ℕ) => by rw [zpow_natCast, map_pow, zpow_natCast] | Int.negSucc n => by rw [zpow_negSucc, hf, map_pow, ← zpow_negSucc] @[to_additive (attr := simp)] lemma map_comp_zpow' [DivInvMonoid G] [DivInvMonoid H] [MonoidHomClass F G H] (f : F) (hf : ∀ x : G, f x⁻¹ = (f x)⁻¹) (g : ι → G) (n : ℤ) : f ∘ (g ^ n) = f ∘ g ^ n := by ext; simp [map_zpow' f hf] /-- Group homomorphisms preserve integer power. -/ @[to_additive (attr := simp) (reorder := 9 10) "Additive group homomorphisms preserve integer scaling."] theorem map_zpow [Group G] [DivisionMonoid H] [MonoidHomClass F G H] (f : F) (g : G) (n : ℤ) : f (g ^ n) = f g ^ n := map_zpow' f (map_inv f) g n @[to_additive] lemma map_comp_zpow [Group G] [DivisionMonoid H] [MonoidHomClass F G H] (f : F) (g : ι → G) (n : ℤ) : f ∘ (g ^ n) = f ∘ g ^ n := by simp end mul_one -- completely uninteresting lemmas about coercion to function, that all homs need section Coes /-! Bundled morphisms can be down-cast to weaker bundlings -/ attribute [coe] MonoidHom.toOneHom attribute [coe] AddMonoidHom.toZeroHom /-- `MonoidHom` down-cast to a `OneHom`, forgetting the multiplicative property. -/ @[to_additive "`AddMonoidHom` down-cast to a `ZeroHom`, forgetting the additive property"] instance MonoidHom.coeToOneHom [MulOneClass M] [MulOneClass N] : Coe (M →* N) (OneHom M N) := ⟨MonoidHom.toOneHom⟩ attribute [coe] MonoidHom.toMulHom attribute [coe] AddMonoidHom.toAddHom /-- `MonoidHom` down-cast to a `MulHom`, forgetting the 1-preserving property. -/ @[to_additive "`AddMonoidHom` down-cast to an `AddHom`, forgetting the 0-preserving property."] instance MonoidHom.coeToMulHom [MulOneClass M] [MulOneClass N] : Coe (M →* N) (M →ₙ* N) := ⟨MonoidHom.toMulHom⟩ -- these must come after the coe_toFun definitions initialize_simps_projections ZeroHom (toFun → apply) initialize_simps_projections AddHom (toFun → apply) initialize_simps_projections AddMonoidHom (toFun → apply) initialize_simps_projections OneHom (toFun → apply) initialize_simps_projections MulHom (toFun → apply) initialize_simps_projections MonoidHom (toFun → apply) @[to_additive (attr := simp)] theorem OneHom.coe_mk [One M] [One N] (f : M → N) (h1) : (OneHom.mk f h1 : M → N) = f := rfl @[to_additive (attr := simp)] theorem OneHom.toFun_eq_coe [One M] [One N] (f : OneHom M N) : f.toFun = f := rfl @[to_additive (attr := simp)] theorem MulHom.coe_mk [Mul M] [Mul N] (f : M → N) (hmul) : (MulHom.mk f hmul : M → N) = f := rfl @[to_additive (attr := simp)] theorem MulHom.toFun_eq_coe [Mul M] [Mul N] (f : M →ₙ* N) : f.toFun = f := rfl @[to_additive (attr := simp)] theorem MonoidHom.coe_mk [MulOneClass M] [MulOneClass N] (f hmul) : (MonoidHom.mk f hmul : M → N) = f := rfl @[to_additive (attr := simp)] theorem MonoidHom.toOneHom_coe [MulOneClass M] [MulOneClass N] (f : M →* N) : (f.toOneHom : M → N) = f := rfl @[to_additive (attr := simp)] theorem MonoidHom.toMulHom_coe [MulOneClass M] [MulOneClass N] (f : M →* N) : f.toMulHom.toFun = f := rfl @[to_additive] theorem MonoidHom.toFun_eq_coe [MulOneClass M] [MulOneClass N] (f : M →* N) : f.toFun = f := rfl @[to_additive (attr := ext)] theorem OneHom.ext [One M] [One N] ⦃f g : OneHom M N⦄ (h : ∀ x, f x = g x) : f = g := DFunLike.ext _ _ h @[to_additive (attr := ext)] theorem MulHom.ext [Mul M] [Mul N] ⦃f g : M →ₙ* N⦄ (h : ∀ x, f x = g x) : f = g := DFunLike.ext _ _ h @[to_additive (attr := ext)] theorem MonoidHom.ext [MulOneClass M] [MulOneClass N] ⦃f g : M →* N⦄ (h : ∀ x, f x = g x) : f = g := DFunLike.ext _ _ h namespace MonoidHom variable [Group G] variable [MulOneClass M] /-- Makes a group homomorphism from a proof that the map preserves multiplication. -/ @[to_additive (attr := simps (config := .asFn)) "Makes an additive group homomorphism from a proof that the map preserves addition."] def mk' (f : M → G) (map_mul : ∀ a b : M, f (a * b) = f a * f b) : M →* G where toFun := f map_mul' := map_mul map_one' := by rw [← mul_right_cancel_iff, ← map_mul _ 1, one_mul, one_mul] end MonoidHom section Deprecated end Deprecated @[to_additive (attr := simp)] theorem OneHom.mk_coe [One M] [One N] (f : OneHom M N) (h1) : OneHom.mk f h1 = f := OneHom.ext fun _ => rfl @[to_additive (attr := simp)] theorem MulHom.mk_coe [Mul M] [Mul N] (f : M →ₙ* N) (hmul) : MulHom.mk f hmul = f := MulHom.ext fun _ => rfl @[to_additive (attr := simp)] theorem MonoidHom.mk_coe [MulOneClass M] [MulOneClass N] (f : M →* N) (hmul) : MonoidHom.mk f hmul = f := MonoidHom.ext fun _ => rfl end Coes /-- Copy of a `OneHom` with a new `toFun` equal to the old one. Useful to fix definitional equalities. -/ @[to_additive "Copy of a `ZeroHom` with a new `toFun` equal to the old one. Useful to fix definitional equalities."] protected def OneHom.copy [One M] [One N] (f : OneHom M N) (f' : M → N) (h : f' = f) : OneHom M N where toFun := f' map_one' := h.symm ▸ f.map_one' @[to_additive (attr := simp)] theorem OneHom.coe_copy {_ : One M} {_ : One N} (f : OneHom M N) (f' : M → N) (h : f' = f) : (f.copy f' h) = f' := rfl @[to_additive] theorem OneHom.coe_copy_eq {_ : One M} {_ : One N} (f : OneHom M N) (f' : M → N) (h : f' = f) : f.copy f' h = f := DFunLike.ext' h /-- Copy of a `MulHom` with a new `toFun` equal to the old one. Useful to fix definitional equalities. -/ @[to_additive "Copy of an `AddHom` with a new `toFun` equal to the old one. Useful to fix definitional equalities."] protected def MulHom.copy [Mul M] [Mul N] (f : M →ₙ* N) (f' : M → N) (h : f' = f) : M →ₙ* N where toFun := f' map_mul' := h.symm ▸ f.map_mul' @[to_additive (attr := simp)] theorem MulHom.coe_copy {_ : Mul M} {_ : Mul N} (f : M →ₙ* N) (f' : M → N) (h : f' = f) : (f.copy f' h) = f' := rfl @[to_additive] theorem MulHom.coe_copy_eq {_ : Mul M} {_ : Mul N} (f : M →ₙ* N) (f' : M → N) (h : f' = f) : f.copy f' h = f := DFunLike.ext' h /-- Copy of a `MonoidHom` with a new `toFun` equal to the old one. Useful to fix definitional equalities. -/ @[to_additive "Copy of an `AddMonoidHom` with a new `toFun` equal to the old one. Useful to fix definitional equalities."] protected def MonoidHom.copy [MulOneClass M] [MulOneClass N] (f : M →* N) (f' : M → N) (h : f' = f) : M →* N := { f.toOneHom.copy f' h, f.toMulHom.copy f' h with } @[to_additive (attr := simp)] theorem MonoidHom.coe_copy {_ : MulOneClass M} {_ : MulOneClass N} (f : M →* N) (f' : M → N) (h : f' = f) : (f.copy f' h) = f' := rfl @[to_additive] theorem MonoidHom.copy_eq {_ : MulOneClass M} {_ : MulOneClass N} (f : M →* N) (f' : M → N) (h : f' = f) : f.copy f' h = f := DFunLike.ext' h @[to_additive] protected theorem OneHom.map_one [One M] [One N] (f : OneHom M N) : f 1 = 1 := f.map_one' /-- If `f` is a monoid homomorphism then `f 1 = 1`. -/ @[to_additive "If `f` is an additive monoid homomorphism then `f 0 = 0`."] protected theorem MonoidHom.map_one [MulOneClass M] [MulOneClass N] (f : M →* N) : f 1 = 1 := f.map_one' @[to_additive] protected theorem MulHom.map_mul [Mul M] [Mul N] (f : M →ₙ* N) (a b : M) : f (a * b) = f a * f b := f.map_mul' a b /-- If `f` is a monoid homomorphism then `f (a * b) = f a * f b`. -/ @[to_additive "If `f` is an additive monoid homomorphism then `f (a + b) = f a + f b`."] protected theorem MonoidHom.map_mul [MulOneClass M] [MulOneClass N] (f : M →* N) (a b : M) : f (a * b) = f a * f b := f.map_mul' a b namespace MonoidHom variable [MulOneClass M] [MulOneClass N] [FunLike F M N] [MonoidHomClass F M N] /-- Given a monoid homomorphism `f : M →* N` and an element `x : M`, if `x` has a right inverse, then `f x` has a right inverse too. For elements invertible on both sides see `IsUnit.map`. -/ @[to_additive "Given an AddMonoid homomorphism `f : M →+ N` and an element `x : M`, if `x` has a right inverse, then `f x` has a right inverse too."] theorem map_exists_right_inv (f : F) {x : M} (hx : ∃ y, x * y = 1) : ∃ y, f x * y = 1 := let ⟨y, hy⟩ := hx ⟨f y, map_mul_eq_one f hy⟩ /-- Given a monoid homomorphism `f : M →* N` and an element `x : M`, if `x` has a left inverse, then `f x` has a left inverse too. For elements invertible on both sides see `IsUnit.map`. -/ @[to_additive "Given an AddMonoid homomorphism `f : M →+ N` and an element `x : M`, if `x` has a left inverse, then `f x` has a left inverse too. For elements invertible on both sides see `IsAddUnit.map`."] theorem map_exists_left_inv (f : F) {x : M} (hx : ∃ y, y * x = 1) : ∃ y, y * f x = 1 := let ⟨y, hy⟩ := hx ⟨f y, map_mul_eq_one f hy⟩ end MonoidHom /-- The identity map from a type with 1 to itself. -/ @[to_additive (attr := simps) "The identity map from a type with zero to itself."] def OneHom.id (M : Type*) [One M] : OneHom M M where toFun x := x map_one' := rfl /-- The identity map from a type with multiplication to itself. -/ @[to_additive (attr := simps) "The identity map from a type with addition to itself."] def MulHom.id (M : Type*) [Mul M] : M →ₙ* M where toFun x := x map_mul' _ _ := rfl /-- The identity map from a monoid to itself. -/ @[to_additive (attr := simps) "The identity map from an additive monoid to itself."] def MonoidHom.id (M : Type*) [MulOneClass M] : M →* M where toFun x := x map_one' := rfl map_mul' _ _ := rfl /-- Composition of `OneHom`s as a `OneHom`. -/ @[to_additive "Composition of `ZeroHom`s as a `ZeroHom`."] def OneHom.comp [One M] [One N] [One P] (hnp : OneHom N P) (hmn : OneHom M N) : OneHom M P where toFun := hnp ∘ hmn map_one' := by simp /-- Composition of `MulHom`s as a `MulHom`. -/ @[to_additive "Composition of `AddHom`s as an `AddHom`."] def MulHom.comp [Mul M] [Mul N] [Mul P] (hnp : N →ₙ* P) (hmn : M →ₙ* N) : M →ₙ* P where toFun := hnp ∘ hmn map_mul' x y := by simp /-- Composition of monoid morphisms as a monoid morphism. -/ @[to_additive "Composition of additive monoid morphisms as an additive monoid morphism."] def MonoidHom.comp [MulOneClass M] [MulOneClass N] [MulOneClass P] (hnp : N →* P) (hmn : M →* N) : M →* P where toFun := hnp ∘ hmn map_one' := by simp map_mul' := by simp @[to_additive (attr := simp)] theorem OneHom.coe_comp [One M] [One N] [One P] (g : OneHom N P) (f : OneHom M N) : ↑(g.comp f) = g ∘ f := rfl @[to_additive (attr := simp)] theorem MulHom.coe_comp [Mul M] [Mul N] [Mul P] (g : N →ₙ* P) (f : M →ₙ* N) : ↑(g.comp f) = g ∘ f := rfl @[to_additive (attr := simp)] theorem MonoidHom.coe_comp [MulOneClass M] [MulOneClass N] [MulOneClass P] (g : N →* P) (f : M →* N) : ↑(g.comp f) = g ∘ f := rfl @[to_additive] theorem OneHom.comp_apply [One M] [One N] [One P] (g : OneHom N P) (f : OneHom M N) (x : M) : g.comp f x = g (f x) := rfl @[to_additive] theorem MulHom.comp_apply [Mul M] [Mul N] [Mul P] (g : N →ₙ* P) (f : M →ₙ* N) (x : M) : g.comp f x = g (f x) := rfl @[to_additive] theorem MonoidHom.comp_apply [MulOneClass M] [MulOneClass N] [MulOneClass P] (g : N →* P) (f : M →* N) (x : M) : g.comp f x = g (f x) := rfl /-- Composition of monoid homomorphisms is associative. -/ @[to_additive "Composition of additive monoid homomorphisms is associative."] theorem OneHom.comp_assoc {Q : Type*} [One M] [One N] [One P] [One Q] (f : OneHom M N) (g : OneHom N P) (h : OneHom P Q) : (h.comp g).comp f = h.comp (g.comp f) := rfl @[to_additive] theorem MulHom.comp_assoc {Q : Type*} [Mul M] [Mul N] [Mul P] [Mul Q] (f : M →ₙ* N) (g : N →ₙ* P) (h : P →ₙ* Q) : (h.comp g).comp f = h.comp (g.comp f) := rfl @[to_additive] theorem MonoidHom.comp_assoc {Q : Type*} [MulOneClass M] [MulOneClass N] [MulOneClass P] [MulOneClass Q] (f : M →* N) (g : N →* P) (h : P →* Q) : (h.comp g).comp f = h.comp (g.comp f) := rfl @[to_additive] theorem OneHom.cancel_right [One M] [One N] [One P] {g₁ g₂ : OneHom N P} {f : OneHom M N} (hf : Function.Surjective f) : g₁.comp f = g₂.comp f ↔ g₁ = g₂ := ⟨fun h => OneHom.ext <| hf.forall.2 (DFunLike.ext_iff.1 h), fun h => h ▸ rfl⟩ @[to_additive] theorem MulHom.cancel_right [Mul M] [Mul N] [Mul P] {g₁ g₂ : N →ₙ* P} {f : M →ₙ* N} (hf : Function.Surjective f) : g₁.comp f = g₂.comp f ↔ g₁ = g₂ := ⟨fun h => MulHom.ext <| hf.forall.2 (DFunLike.ext_iff.1 h), fun h => h ▸ rfl⟩ @[to_additive] theorem MonoidHom.cancel_right [MulOneClass M] [MulOneClass N] [MulOneClass P] {g₁ g₂ : N →* P} {f : M →* N} (hf : Function.Surjective f) : g₁.comp f = g₂.comp f ↔ g₁ = g₂ := ⟨fun h => MonoidHom.ext <| hf.forall.2 (DFunLike.ext_iff.1 h), fun h => h ▸ rfl⟩ @[to_additive] theorem OneHom.cancel_left [One M] [One N] [One P] {g : OneHom N P} {f₁ f₂ : OneHom M N} (hg : Function.Injective g) : g.comp f₁ = g.comp f₂ ↔ f₁ = f₂ := ⟨fun h => OneHom.ext fun x => hg <| by rw [← OneHom.comp_apply, h, OneHom.comp_apply], fun h => h ▸ rfl⟩ @[to_additive] theorem MulHom.cancel_left [Mul M] [Mul N] [Mul P] {g : N →ₙ* P} {f₁ f₂ : M →ₙ* N} (hg : Function.Injective g) : g.comp f₁ = g.comp f₂ ↔ f₁ = f₂ := ⟨fun h => MulHom.ext fun x => hg <| by rw [← MulHom.comp_apply, h, MulHom.comp_apply], fun h => h ▸ rfl⟩ @[to_additive] theorem MonoidHom.cancel_left [MulOneClass M] [MulOneClass N] [MulOneClass P] {g : N →* P} {f₁ f₂ : M →* N} (hg : Function.Injective g) : g.comp f₁ = g.comp f₂ ↔ f₁ = f₂ := ⟨fun h => MonoidHom.ext fun x => hg <| by rw [← MonoidHom.comp_apply, h, MonoidHom.comp_apply], fun h => h ▸ rfl⟩ section @[to_additive] theorem MonoidHom.toOneHom_injective [MulOneClass M] [MulOneClass N] : Function.Injective (MonoidHom.toOneHom : (M →* N) → OneHom M N) := Function.Injective.of_comp (f := DFunLike.coe) DFunLike.coe_injective @[to_additive] theorem MonoidHom.toMulHom_injective [MulOneClass M] [MulOneClass N] : Function.Injective (MonoidHom.toMulHom : (M →* N) → M →ₙ* N) := Function.Injective.of_comp (f := DFunLike.coe) DFunLike.coe_injective end @[to_additive (attr := simp)] theorem OneHom.comp_id [One M] [One N] (f : OneHom M N) : f.comp (OneHom.id M) = f := OneHom.ext fun _ => rfl @[to_additive (attr := simp)] theorem MulHom.comp_id [Mul M] [Mul N] (f : M →ₙ* N) : f.comp (MulHom.id M) = f := MulHom.ext fun _ => rfl @[to_additive (attr := simp)] theorem MonoidHom.comp_id [MulOneClass M] [MulOneClass N] (f : M →* N) : f.comp (MonoidHom.id M) = f := MonoidHom.ext fun _ => rfl @[to_additive (attr := simp)] theorem OneHom.id_comp [One M] [One N] (f : OneHom M N) : (OneHom.id N).comp f = f := OneHom.ext fun _ => rfl @[to_additive (attr := simp)] theorem MulHom.id_comp [Mul M] [Mul N] (f : M →ₙ* N) : (MulHom.id N).comp f = f := MulHom.ext fun _ => rfl @[to_additive (attr := simp)] theorem MonoidHom.id_comp [MulOneClass M] [MulOneClass N] (f : M →* N) : (MonoidHom.id N).comp f = f := MonoidHom.ext fun _ => rfl @[to_additive] protected theorem MonoidHom.map_pow [Monoid M] [Monoid N] (f : M →* N) (a : M) (n : ℕ) : f (a ^ n) = f a ^ n := map_pow f a n @[to_additive] protected theorem MonoidHom.map_zpow' [DivInvMonoid M] [DivInvMonoid N] (f : M →* N) (hf : ∀ x, f x⁻¹ = (f x)⁻¹) (a : M) (n : ℤ) : f (a ^ n) = f a ^ n := map_zpow' f hf a n section End namespace Monoid variable (M) [MulOneClass M] /-- The monoid of endomorphisms. -/ protected def End := M →* M namespace End instance instFunLike : FunLike (Monoid.End M) M M := MonoidHom.instFunLike instance instMonoidHomClass : MonoidHomClass (Monoid.End M) M M := MonoidHom.instMonoidHomClass instance instOne : One (Monoid.End M) where one := .id _ instance instMul : Mul (Monoid.End M) where mul := .comp instance : Monoid (Monoid.End M) where mul := MonoidHom.comp one := MonoidHom.id M mul_assoc _ _ _ := MonoidHom.comp_assoc _ _ _ mul_one := MonoidHom.comp_id one_mul := MonoidHom.id_comp npow n f := (npowRec n f).copy f^[n] $ by induction n <;> simp [npowRec, *] <;> rfl npow_succ n f := DFunLike.coe_injective $ Function.iterate_succ _ _ instance : Inhabited (Monoid.End M) := ⟨1⟩ @[simp, norm_cast] lemma coe_pow (f : Monoid.End M) (n : ℕ) : (↑(f ^ n) : M → M) = f^[n] := rfl end End @[simp] theorem coe_one : ((1 : Monoid.End M) : M → M) = id := rfl @[simp] theorem coe_mul (f g) : ((f * g : Monoid.End M) : M → M) = f ∘ g := rfl end Monoid namespace AddMonoid variable (A : Type*) [AddZeroClass A] /-- The monoid of endomorphisms. -/ protected def End := A →+ A namespace End instance instFunLike : FunLike (AddMonoid.End A) A A := AddMonoidHom.instFunLike instance instAddMonoidHomClass : AddMonoidHomClass (AddMonoid.End A) A A := AddMonoidHom.instAddMonoidHomClass instance instOne : One (AddMonoid.End A) where one := .id _ instance instMul : Mul (AddMonoid.End A) where mul := .comp @[simp, norm_cast] lemma coe_one : ((1 : AddMonoid.End A) : A → A) = id := rfl @[simp, norm_cast] lemma coe_mul (f g : AddMonoid.End A) : (f * g : A → A) = f ∘ g := rfl instance monoid : Monoid (AddMonoid.End A) where mul_assoc _ _ _ := AddMonoidHom.comp_assoc _ _ _ mul_one := AddMonoidHom.comp_id one_mul := AddMonoidHom.id_comp npow n f := (npowRec n f).copy (Nat.iterate f n) $ by induction n <;> simp [npowRec, *] <;> rfl npow_succ n f := DFunLike.coe_injective $ Function.iterate_succ _ _ @[simp, norm_cast] lemma coe_pow (f : AddMonoid.End A) (n : ℕ) : (↑(f ^ n) : A → A) = f^[n] := rfl instance : Inhabited (AddMonoid.End A) := ⟨1⟩ end End end AddMonoid end End /-- `1` is the homomorphism sending all elements to `1`. -/ @[to_additive "`0` is the homomorphism sending all elements to `0`."] instance [One M] [One N] : One (OneHom M N) := ⟨⟨fun _ => 1, rfl⟩⟩ /-- `1` is the multiplicative homomorphism sending all elements to `1`. -/ @[to_additive "`0` is the additive homomorphism sending all elements to `0`"] instance [Mul M] [MulOneClass N] : One (M →ₙ* N) := ⟨⟨fun _ => 1, fun _ _ => (one_mul 1).symm⟩⟩ /-- `1` is the monoid homomorphism sending all elements to `1`. -/ @[to_additive "`0` is the additive monoid homomorphism sending all elements to `0`."] instance [MulOneClass M] [MulOneClass N] : One (M →* N) := ⟨⟨⟨fun _ => 1, rfl⟩, fun _ _ => (one_mul 1).symm⟩⟩ @[to_additive (attr := simp)] theorem OneHom.one_apply [One M] [One N] (x : M) : (1 : OneHom M N) x = 1 := rfl @[to_additive (attr := simp)] theorem MonoidHom.one_apply [MulOneClass M] [MulOneClass N] (x : M) : (1 : M →* N) x = 1 := rfl @[to_additive (attr := simp)] theorem OneHom.one_comp [One M] [One N] [One P] (f : OneHom M N) : (1 : OneHom N P).comp f = 1 := rfl @[to_additive (attr := simp)] theorem OneHom.comp_one [One M] [One N] [One P] (f : OneHom N P) : f.comp (1 : OneHom M N) = 1 := by ext simp only [OneHom.map_one, OneHom.coe_comp, Function.comp_apply, OneHom.one_apply] @[to_additive] instance [One M] [One N] : Inhabited (OneHom M N) := ⟨1⟩ @[to_additive] instance [Mul M] [MulOneClass N] : Inhabited (M →ₙ* N) := ⟨1⟩ @[to_additive] instance [MulOneClass M] [MulOneClass N] : Inhabited (M →* N) := ⟨1⟩ namespace MonoidHom variable [Group G] [CommGroup H] @[to_additive (attr := simp)] theorem one_comp [MulOneClass M] [MulOneClass N] [MulOneClass P] (f : M →* N) : (1 : N →* P).comp f = 1 := rfl @[to_additive (attr := simp)] theorem comp_one [MulOneClass M] [MulOneClass N] [MulOneClass P] (f : N →* P) : f.comp (1 : M →* N) = 1 := by ext simp only [map_one, coe_comp, Function.comp_apply, one_apply] /-- Group homomorphisms preserve inverse. -/ @[to_additive "Additive group homomorphisms preserve negation."] protected theorem map_inv [Group α] [DivisionMonoid β] (f : α →* β) (a : α) : f a⁻¹ = (f a)⁻¹ := map_inv f _ /-- Group homomorphisms preserve integer power. -/ @[to_additive "Additive group homomorphisms preserve integer scaling."] protected theorem map_zpow [Group α] [DivisionMonoid β] (f : α →* β) (g : α) (n : ℤ) : f (g ^ n) = f g ^ n := map_zpow f g n /-- Group homomorphisms preserve division. -/ @[to_additive "Additive group homomorphisms preserve subtraction."] protected theorem map_div [Group α] [DivisionMonoid β] (f : α →* β) (g h : α) : f (g / h) = f g / f h := map_div f g h /-- Group homomorphisms preserve division. -/ @[to_additive "Additive group homomorphisms preserve subtraction."] protected theorem map_mul_inv [Group α] [DivisionMonoid β] (f : α →* β) (g h : α) : f (g * h⁻¹) = f g * (f h)⁻¹ := by simp end MonoidHom
Algebra\Group\Hom\End.lean
/- Copyright (c) 2018 Patrick Massot. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Patrick Massot, Kevin Buzzard, Scott Morrison, Johan Commelin, Chris Hughes, Johannes Hölzl, Yury Kudryashov -/ import Mathlib.Algebra.Group.Commute.Defs import Mathlib.Algebra.Group.Hom.Instances import Mathlib.Algebra.Ring.Basic /-! # Instances on spaces of monoid and group morphisms This file does two things involving `AddMonoid.End` and `Ring`. They are separate, and if someone would like to split this file in two that may be helpful. * We provide the `Ring` structure on `AddMonoid.End`. * Results about `AddMonoid.End R` when `R` is a ring. -/ universe uM uN uP uQ variable {M : Type uM} {N : Type uN} {P : Type uP} {Q : Type uQ} namespace AddMonoid.End instance instAddMonoidWithOne (M) [AddCommMonoid M] : AddMonoidWithOne (AddMonoid.End M) where natCast n := n • (1 : AddMonoid.End M) natCast_zero := AddMonoid.nsmul_zero _ natCast_succ n := AddMonoid.nsmul_succ n 1 /-- See also `AddMonoid.End.natCast_def`. -/ @[simp] lemma natCast_apply [AddCommMonoid M] (n : ℕ) (m : M) : (↑n : AddMonoid.End M) m = n • m := rfl -- See note [no_index around OfNat.ofNat] @[simp] lemma ofNat_apply [AddCommMonoid M] (n : ℕ) [n.AtLeastTwo] (m : M) : (no_index (OfNat.ofNat n : AddMonoid.End M)) m = n • m := rfl instance instSemiring [AddCommMonoid M] : Semiring (AddMonoid.End M) := { AddMonoid.End.monoid M, AddMonoidHom.addCommMonoid, AddMonoid.End.instAddMonoidWithOne M with zero_mul := fun _ => AddMonoidHom.ext fun _ => rfl, mul_zero := fun _ => AddMonoidHom.ext fun _ => AddMonoidHom.map_zero _, left_distrib := fun _ _ _ => AddMonoidHom.ext fun _ => AddMonoidHom.map_add _ _ _, right_distrib := fun _ _ _ => AddMonoidHom.ext fun _ => rfl } instance instRing [AddCommGroup M] : Ring (AddMonoid.End M) := { AddMonoid.End.instSemiring, AddMonoid.End.instAddCommGroup with intCast := fun z => z • (1 : AddMonoid.End M), intCast_ofNat := natCast_zsmul _, intCast_negSucc := negSucc_zsmul _ } end AddMonoid.End /-! ### Miscellaneous definitions This file used to import `Algebra.GroupPower.Basic`, hence it was not possible to import it in some of the lower-level files like `Algebra.Ring.Basic`. The following lemmas should be rehomed now that `Algebra.GroupPower.Basic` was deleted. -/ section Semiring variable {R S : Type*} [NonUnitalNonAssocSemiring R] [NonUnitalNonAssocSemiring S] /-- Multiplication of an element of a (semi)ring is an `AddMonoidHom` in both arguments. This is a more-strongly bundled version of `AddMonoidHom.mulLeft` and `AddMonoidHom.mulRight`. Stronger versions of this exists for algebras as `LinearMap.mul`, `NonUnitalAlgHom.mul` and `Algebra.lmul`. -/ def AddMonoidHom.mul : R →+ R →+ R where toFun := AddMonoidHom.mulLeft map_zero' := AddMonoidHom.ext <| zero_mul map_add' a b := AddMonoidHom.ext <| add_mul a b theorem AddMonoidHom.mul_apply (x y : R) : AddMonoidHom.mul x y = x * y := rfl @[simp] theorem AddMonoidHom.coe_mul : ⇑(AddMonoidHom.mul : R →+ R →+ R) = AddMonoidHom.mulLeft := rfl @[simp] theorem AddMonoidHom.coe_flip_mul : ⇑(AddMonoidHom.mul : R →+ R →+ R).flip = AddMonoidHom.mulRight := rfl /-- An `AddMonoidHom` preserves multiplication if pre- and post- composition with `AddMonoidHom.mul` are equivalent. By converting the statement into an equality of `AddMonoidHom`s, this lemma allows various specialized `ext` lemmas about `→+` to then be applied. -/ theorem AddMonoidHom.map_mul_iff (f : R →+ S) : (∀ x y, f (x * y) = f x * f y) ↔ (AddMonoidHom.mul : R →+ R →+ R).compr₂ f = (AddMonoidHom.mul.comp f).compl₂ f := Iff.symm AddMonoidHom.ext_iff₂ lemma AddMonoidHom.mulLeft_eq_mulRight_iff_forall_commute {a : R} : mulLeft a = mulRight a ↔ ∀ b, Commute a b := DFunLike.ext_iff lemma AddMonoidHom.mulRight_eq_mulLeft_iff_forall_commute {b : R} : mulRight b = mulLeft b ↔ ∀ a, Commute a b := DFunLike.ext_iff /-- The left multiplication map: `(a, b) ↦ a * b`. See also `AddMonoidHom.mulLeft`. -/ @[simps!] def AddMonoid.End.mulLeft : R →+ AddMonoid.End R := AddMonoidHom.mul /-- The right multiplication map: `(a, b) ↦ b * a`. See also `AddMonoidHom.mulRight`. -/ @[simps!] def AddMonoid.End.mulRight : R →+ AddMonoid.End R := (AddMonoidHom.mul : R →+ AddMonoid.End R).flip end Semiring section CommSemiring variable {R S : Type*} [NonUnitalNonAssocCommSemiring R] namespace AddMonoid.End lemma mulRight_eq_mulLeft : mulRight = (mulLeft : R →+ AddMonoid.End R) := AddMonoidHom.ext fun _ => Eq.symm <| AddMonoidHom.mulLeft_eq_mulRight_iff_forall_commute.2 (.all _) end AddMonoid.End end CommSemiring
Algebra\Group\Hom\Instances.lean
/- Copyright (c) 2018 Patrick Massot. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Patrick Massot, Kevin Buzzard, Scott Morrison, Johan Commelin, Chris Hughes, Johannes Hölzl, Yury Kudryashov -/ import Mathlib.Algebra.Group.Hom.Basic /-! # Instances on spaces of monoid and group morphisms We endow the space of monoid morphisms `M →* N` with a `CommMonoid` structure when the target is commutative, through pointwise multiplication, and with a `CommGroup` structure when the target is a commutative group. We also prove the same instances for additive situations. Since these structures permit morphisms of morphisms, we also provide some composition-like operations. Finally, we provide the `Ring` structure on `AddMonoid.End`. -/ assert_not_exists AddMonoidWithOne universe uM uN uP uQ variable {M : Type uM} {N : Type uN} {P : Type uP} {Q : Type uQ} /-- `(M →* N)` is a `CommMonoid` if `N` is commutative. -/ @[to_additive "`(M →+ N)` is an `AddCommMonoid` if `N` is commutative."] instance MonoidHom.commMonoid [MulOneClass M] [CommMonoid N] : CommMonoid (M →* N) where mul := (· * ·) mul_assoc := by intros; ext; apply mul_assoc one := 1 one_mul := by intros; ext; apply one_mul mul_one := by intros; ext; apply mul_one mul_comm := by intros; ext; apply mul_comm npow n f := { toFun := fun x => f x ^ n, map_one' := by simp, map_mul' := fun x y => by simp [mul_pow] } npow_zero f := by ext x simp npow_succ n f := by ext x simp [pow_succ] /-- If `G` is a commutative group, then `M →* G` is a commutative group too. -/ @[to_additive "If `G` is an additive commutative group, then `M →+ G` is an additive commutative group too."] instance MonoidHom.commGroup {M G} [MulOneClass M] [CommGroup G] : CommGroup (M →* G) := { MonoidHom.commMonoid with inv := Inv.inv, div := Div.div, div_eq_mul_inv := by intros ext apply div_eq_mul_inv, mul_left_inv := by intros; ext; apply mul_left_inv, zpow := fun n f => { toFun := fun x => f x ^ n, map_one' := by simp, map_mul' := fun x y => by simp [mul_zpow] }, zpow_zero' := fun f => by ext x simp, zpow_succ' := fun n f => by ext x simp [zpow_add_one], zpow_neg' := fun n f => by ext x simp [zpow_natCast, -Int.natCast_add] } instance AddMonoid.End.instAddCommMonoid [AddCommMonoid M] : AddCommMonoid (AddMonoid.End M) := AddMonoidHom.addCommMonoid @[simp] theorem AddMonoid.End.zero_apply [AddCommMonoid M] (m : M) : (0 : AddMonoid.End M) m = 0 := rfl -- Note: `@[simp]` omitted because `(1 : AddMonoid.End M) = id` by `AddMonoid.coe_one` theorem AddMonoid.End.one_apply [AddCommMonoid M] (m : M) : (1 : AddMonoid.End M) m = m := rfl instance AddMonoid.End.instAddCommGroup [AddCommGroup M] : AddCommGroup (AddMonoid.End M) := AddMonoidHom.addCommGroup instance AddMonoid.End.instIntCast [AddCommGroup M] : IntCast (AddMonoid.End M) := { intCast := fun z => z • (1 : AddMonoid.End M) } /-- See also `AddMonoid.End.intCast_def`. -/ @[simp] theorem AddMonoid.End.intCast_apply [AddCommGroup M] (z : ℤ) (m : M) : (↑z : AddMonoid.End M) m = z • m := rfl @[deprecated (since := "2024-04-17")] alias AddMonoid.End.int_cast_apply := AddMonoid.End.intCast_apply @[to_additive (attr := simp)] lemma MonoidHom.pow_apply {M N : Type*} [MulOneClass M] [CommMonoid N] (f : M →* N) (n : ℕ) (x : M) : (f ^ n) x = (f x) ^ n := rfl /-! ### Morphisms of morphisms The structures above permit morphisms that themselves produce morphisms, provided the codomain is commutative. -/ namespace MonoidHom @[to_additive] theorem ext_iff₂ {_ : MulOneClass M} {_ : MulOneClass N} {_ : CommMonoid P} {f g : M →* N →* P} : f = g ↔ ∀ x y, f x y = g x y := DFunLike.ext_iff.trans <| forall_congr' fun _ => DFunLike.ext_iff /-- `flip` arguments of `f : M →* N →* P` -/ @[to_additive "`flip` arguments of `f : M →+ N →+ P`"] def flip {mM : MulOneClass M} {mN : MulOneClass N} {mP : CommMonoid P} (f : M →* N →* P) : N →* M →* P where toFun y := { toFun := fun x => f x y, map_one' := by simp [f.map_one, one_apply], map_mul' := fun x₁ x₂ => by simp [f.map_mul, mul_apply] } map_one' := ext fun x => (f x).map_one map_mul' y₁ y₂ := ext fun x => (f x).map_mul y₁ y₂ @[to_additive (attr := simp)] theorem flip_apply {_ : MulOneClass M} {_ : MulOneClass N} {_ : CommMonoid P} (f : M →* N →* P) (x : M) (y : N) : f.flip y x = f x y := rfl @[to_additive] theorem map_one₂ {_ : MulOneClass M} {_ : MulOneClass N} {_ : CommMonoid P} (f : M →* N →* P) (n : N) : f 1 n = 1 := (flip f n).map_one @[to_additive] theorem map_mul₂ {_ : MulOneClass M} {_ : MulOneClass N} {_ : CommMonoid P} (f : M →* N →* P) (m₁ m₂ : M) (n : N) : f (m₁ * m₂) n = f m₁ n * f m₂ n := (flip f n).map_mul _ _ @[to_additive] theorem map_inv₂ {_ : Group M} {_ : MulOneClass N} {_ : CommGroup P} (f : M →* N →* P) (m : M) (n : N) : f m⁻¹ n = (f m n)⁻¹ := (flip f n).map_inv _ @[to_additive] theorem map_div₂ {_ : Group M} {_ : MulOneClass N} {_ : CommGroup P} (f : M →* N →* P) (m₁ m₂ : M) (n : N) : f (m₁ / m₂) n = f m₁ n / f m₂ n := (flip f n).map_div _ _ /-- Evaluation of a `MonoidHom` at a point as a monoid homomorphism. See also `MonoidHom.apply` for the evaluation of any function at a point. -/ @[to_additive (attr := simps!) "Evaluation of an `AddMonoidHom` at a point as an additive monoid homomorphism. See also `AddMonoidHom.apply` for the evaluation of any function at a point."] def eval [MulOneClass M] [CommMonoid N] : M →* (M →* N) →* N := (MonoidHom.id (M →* N)).flip /-- The expression `fun g m ↦ g (f m)` as a `MonoidHom`. Equivalently, `(fun g ↦ MonoidHom.comp g f)` as a `MonoidHom`. -/ @[to_additive (attr := simps!) "The expression `fun g m ↦ g (f m)` as an `AddMonoidHom`. Equivalently, `(fun g ↦ AddMonoidHom.comp g f)` as an `AddMonoidHom`. This also exists in a `LinearMap` version, `LinearMap.lcomp`."] def compHom' [MulOneClass M] [MulOneClass N] [CommMonoid P] (f : M →* N) : (N →* P) →* M →* P := flip <| eval.comp f /-- Composition of monoid morphisms (`MonoidHom.comp`) as a monoid morphism. Note that unlike `MonoidHom.comp_hom'` this requires commutativity of `N`. -/ @[to_additive (attr := simps) "Composition of additive monoid morphisms (`AddMonoidHom.comp`) as an additive monoid morphism. Note that unlike `AddMonoidHom.comp_hom'` this requires commutativity of `N`. This also exists in a `LinearMap` version, `LinearMap.llcomp`."] def compHom [MulOneClass M] [CommMonoid N] [CommMonoid P] : (N →* P) →* (M →* N) →* M →* P where toFun g := { toFun := g.comp, map_one' := comp_one g, map_mul' := comp_mul g } map_one' := by ext1 f exact one_comp f map_mul' g₁ g₂ := by ext1 f exact mul_comp g₁ g₂ f /-- Flipping arguments of monoid morphisms (`MonoidHom.flip`) as a monoid morphism. -/ @[to_additive (attr := simps) "Flipping arguments of additive monoid morphisms (`AddMonoidHom.flip`) as an additive monoid morphism."] def flipHom {_ : MulOneClass M} {_ : MulOneClass N} {_ : CommMonoid P} : (M →* N →* P) →* N →* M →* P where toFun := MonoidHom.flip map_one' := rfl map_mul' _ _ := rfl /-- The expression `fun m q ↦ f m (g q)` as a `MonoidHom`. Note that the expression `fun q n ↦ f (g q) n` is simply `MonoidHom.comp`. -/ @[to_additive "The expression `fun m q ↦ f m (g q)` as an `AddMonoidHom`. Note that the expression `fun q n ↦ f (g q) n` is simply `AddMonoidHom.comp`. This also exists as a `LinearMap` version, `LinearMap.compl₂`"] def compl₂ [MulOneClass M] [MulOneClass N] [CommMonoid P] [MulOneClass Q] (f : M →* N →* P) (g : Q →* N) : M →* Q →* P := (compHom' g).comp f @[to_additive (attr := simp)] theorem compl₂_apply [MulOneClass M] [MulOneClass N] [CommMonoid P] [MulOneClass Q] (f : M →* N →* P) (g : Q →* N) (m : M) (q : Q) : (compl₂ f g) m q = f m (g q) := rfl /-- The expression `fun m n ↦ g (f m n)` as a `MonoidHom`. -/ @[to_additive "The expression `fun m n ↦ g (f m n)` as an `AddMonoidHom`. This also exists as a `LinearMap` version, `LinearMap.compr₂`"] def compr₂ [MulOneClass M] [MulOneClass N] [CommMonoid P] [CommMonoid Q] (f : M →* N →* P) (g : P →* Q) : M →* N →* Q := (compHom g).comp f @[to_additive (attr := simp)] theorem compr₂_apply [MulOneClass M] [MulOneClass N] [CommMonoid P] [CommMonoid Q] (f : M →* N →* P) (g : P →* Q) (m : M) (n : N) : (compr₂ f g) m n = g (f m n) := rfl end MonoidHom assert_not_exists Ring
Algebra\Group\Invertible\Basic.lean
/- Copyright (c) 2020 Anne Baanen. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Anne Baanen -/ import Mathlib.Algebra.Group.Commute.Units import Mathlib.Algebra.Group.Invertible.Defs import Mathlib.Algebra.Group.Hom.Defs import Mathlib.Logic.Equiv.Defs /-! # Theorems about invertible elements -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered universe u variable {α : Type u} /-- An `Invertible` element is a unit. -/ @[simps] def unitOfInvertible [Monoid α] (a : α) [Invertible a] : αˣ where val := a inv := ⅟ a val_inv := by simp inv_val := by simp theorem isUnit_of_invertible [Monoid α] (a : α) [Invertible a] : IsUnit a := ⟨unitOfInvertible a, rfl⟩ /-- Units are invertible in their associated monoid. -/ def Units.invertible [Monoid α] (u : αˣ) : Invertible (u : α) where invOf := ↑u⁻¹ invOf_mul_self := u.inv_mul mul_invOf_self := u.mul_inv @[simp] theorem invOf_units [Monoid α] (u : αˣ) [Invertible (u : α)] : ⅟ (u : α) = ↑u⁻¹ := invOf_eq_right_inv u.mul_inv theorem IsUnit.nonempty_invertible [Monoid α] {a : α} (h : IsUnit a) : Nonempty (Invertible a) := let ⟨x, hx⟩ := h ⟨x.invertible.copy _ hx.symm⟩ /-- Convert `IsUnit` to `Invertible` using `Classical.choice`. Prefer `casesI h.nonempty_invertible` over `letI := h.invertible` if you want to avoid choice. -/ noncomputable def IsUnit.invertible [Monoid α] {a : α} (h : IsUnit a) : Invertible a := Classical.choice h.nonempty_invertible @[simp] theorem nonempty_invertible_iff_isUnit [Monoid α] (a : α) : Nonempty (Invertible a) ↔ IsUnit a := ⟨Nonempty.rec <| @isUnit_of_invertible _ _ _, IsUnit.nonempty_invertible⟩ theorem Commute.invOf_right [Monoid α] {a b : α} [Invertible b] (h : Commute a b) : Commute a (⅟ b) := calc a * ⅟ b = ⅟ b * (b * a * ⅟ b) := by simp [mul_assoc] _ = ⅟ b * (a * b * ⅟ b) := by rw [h.eq] _ = ⅟ b * a := by simp [mul_assoc] theorem Commute.invOf_left [Monoid α] {a b : α} [Invertible b] (h : Commute b a) : Commute (⅟ b) a := calc ⅟ b * a = ⅟ b * (a * b * ⅟ b) := by simp [mul_assoc] _ = ⅟ b * (b * a * ⅟ b) := by rw [h.eq] _ = a * ⅟ b := by simp [mul_assoc] theorem commute_invOf {M : Type*} [One M] [Mul M] (m : M) [Invertible m] : Commute m (⅟ m) := calc m * ⅟ m = 1 := mul_invOf_self m _ = ⅟ m * m := (invOf_mul_self m).symm section Monoid variable [Monoid α] /-- This is the `Invertible` version of `Units.isUnit_units_mul` -/ abbrev invertibleOfInvertibleMul (a b : α) [Invertible a] [Invertible (a * b)] : Invertible b where invOf := ⅟ (a * b) * a invOf_mul_self := by rw [mul_assoc, invOf_mul_self] mul_invOf_self := by rw [← (isUnit_of_invertible a).mul_right_inj, ← mul_assoc, ← mul_assoc, mul_invOf_self, mul_one, one_mul] /-- This is the `Invertible` version of `Units.isUnit_mul_units` -/ abbrev invertibleOfMulInvertible (a b : α) [Invertible (a * b)] [Invertible b] : Invertible a where invOf := b * ⅟ (a * b) invOf_mul_self := by rw [← (isUnit_of_invertible b).mul_left_inj, mul_assoc, mul_assoc, invOf_mul_self, mul_one, one_mul] mul_invOf_self := by rw [← mul_assoc, mul_invOf_self] /-- `invertibleOfInvertibleMul` and `invertibleMul` as an equivalence. -/ @[simps apply symm_apply] def Invertible.mulLeft {a : α} (_ : Invertible a) (b : α) : Invertible b ≃ Invertible (a * b) where toFun _ := invertibleMul a b invFun _ := invertibleOfInvertibleMul a _ left_inv _ := Subsingleton.elim _ _ right_inv _ := Subsingleton.elim _ _ /-- `invertibleOfMulInvertible` and `invertibleMul` as an equivalence. -/ @[simps apply symm_apply] def Invertible.mulRight (a : α) {b : α} (_ : Invertible b) : Invertible a ≃ Invertible (a * b) where toFun _ := invertibleMul a b invFun _ := invertibleOfMulInvertible _ b left_inv _ := Subsingleton.elim _ _ right_inv _ := Subsingleton.elim _ _ instance invertiblePow (m : α) [Invertible m] (n : ℕ) : Invertible (m ^ n) where invOf := ⅟ m ^ n invOf_mul_self := by rw [← (commute_invOf m).symm.mul_pow, invOf_mul_self, one_pow] mul_invOf_self := by rw [← (commute_invOf m).mul_pow, mul_invOf_self, one_pow] lemma invOf_pow (m : α) [Invertible m] (n : ℕ) [Invertible (m ^ n)] : ⅟ (m ^ n) = ⅟ m ^ n := @invertible_unique _ _ _ _ _ (invertiblePow m n) rfl /-- If `x ^ n = 1` then `x` has an inverse, `x^(n - 1)`. -/ def invertibleOfPowEqOne (x : α) (n : ℕ) (hx : x ^ n = 1) (hn : n ≠ 0) : Invertible x := (Units.ofPowEqOne x n hx hn).invertible end Monoid /-- Monoid homs preserve invertibility. -/ def Invertible.map {R : Type*} {S : Type*} {F : Type*} [MulOneClass R] [MulOneClass S] [FunLike F R S] [MonoidHomClass F R S] (f : F) (r : R) [Invertible r] : Invertible (f r) where invOf := f (⅟ r) invOf_mul_self := by rw [← map_mul, invOf_mul_self, map_one] mul_invOf_self := by rw [← map_mul, mul_invOf_self, map_one] /-- Note that the `Invertible (f r)` argument can be satisfied by using `letI := Invertible.map f r` before applying this lemma. -/ theorem map_invOf {R : Type*} {S : Type*} {F : Type*} [MulOneClass R] [Monoid S] [FunLike F R S] [MonoidHomClass F R S] (f : F) (r : R) [Invertible r] [ifr : Invertible (f r)] : f (⅟ r) = ⅟ (f r) := have h : ifr = Invertible.map f r := Subsingleton.elim _ _ by subst h; rfl /-- If a function `f : R → S` has a left-inverse that is a monoid hom, then `r : R` is invertible if `f r` is. The inverse is computed as `g (⅟(f r))` -/ @[simps! (config := .lemmasOnly)] def Invertible.ofLeftInverse {R : Type*} {S : Type*} {G : Type*} [MulOneClass R] [MulOneClass S] [FunLike G S R] [MonoidHomClass G S R] (f : R → S) (g : G) (r : R) (h : Function.LeftInverse g f) [Invertible (f r)] : Invertible r := (Invertible.map g (f r)).copy _ (h r).symm /-- Invertibility on either side of a monoid hom with a left-inverse is equivalent. -/ @[simps] def invertibleEquivOfLeftInverse {R : Type*} {S : Type*} {F G : Type*} [Monoid R] [Monoid S] [FunLike F R S] [MonoidHomClass F R S] [FunLike G S R] [MonoidHomClass G S R] (f : F) (g : G) (r : R) (h : Function.LeftInverse g f) : Invertible (f r) ≃ Invertible r where toFun _ := Invertible.ofLeftInverse f _ _ h invFun _ := Invertible.map f _ left_inv _ := Subsingleton.elim _ _ right_inv _ := Subsingleton.elim _ _
Algebra\Group\Invertible\Defs.lean
/- Copyright (c) 2020 Anne Baanen. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Anne Baanen -/ import Mathlib.Algebra.Group.Defs /-! # Invertible elements This file defines a typeclass `Invertible a` for elements `a` with a two-sided multiplicative inverse. The intent of the typeclass is to provide a way to write e.g. `⅟2` in a ring like `ℤ[1/2]` where some inverses exist but there is no general `⁻¹` operator; or to specify that a field has characteristic `≠ 2`. It is the `Type`-valued analogue to the `Prop`-valued `IsUnit`. For constructions of the invertible element given a characteristic, see `Algebra/CharP/Invertible` and other lemmas in that file. ## Notation * `⅟a` is `Invertible.invOf a`, the inverse of `a` ## Implementation notes The `Invertible` class lives in `Type`, not `Prop`, to make computation easier. If multiplication is associative, `Invertible` is a subsingleton anyway. The `simp` normal form tries to normalize `⅟a` to `a ⁻¹`. Otherwise, it pushes `⅟` inside the expression as much as possible. Since `Invertible a` is not a `Prop` (but it is a `Subsingleton`), we have to be careful about coherence issues: we should avoid having multiple non-defeq instances for `Invertible a` in the same context. This file plays it safe and uses `def` rather than `instance` for most definitions, users can choose which instances to use at the point of use. For example, here's how you can use an `Invertible 1` instance: ```lean variable {α : Type*} [Monoid α] def something_that_needs_inverses (x : α) [Invertible x] := sorry section attribute [local instance] invertibleOne def something_one := something_that_needs_inverses 1 end ``` ### Typeclass search vs. unification for `simp` lemmas Note that since typeclass search searches the local context first, an instance argument like `[Invertible a]` might sometimes be filled by a different term than the one we'd find by unification (i.e., the one that's used as an implicit argument to `⅟`). This can cause issues with `simp`. Therefore, some lemmas are duplicated, with the `@[simp]` versions using unification and the user-facing ones using typeclass search. Since unification can make backwards rewriting (e.g. `rw [← mylemma]`) impractical, we still want the instance-argument versions; therefore the user-facing versions retain the instance arguments and the original lemma name, whereas the `@[simp]`/unification ones acquire a `'` at the end of their name. We modify this file according to the above pattern only as needed; therefore, most `@[simp]` lemmas here are not part of such a duplicate pair. This is not (yet) intended as a permanent solution. See Zulip: [https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Invertible.201.20simps/near/320558233] ## Tags invertible, inverse element, invOf, a half, one half, a third, one third, ½, ⅓ -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered universe u variable {α : Type u} /-- `Invertible a` gives a two-sided multiplicative inverse of `a`. -/ class Invertible [Mul α] [One α] (a : α) : Type u where /-- The inverse of an `Invertible` element -/ invOf : α /-- `invOf a` is a left inverse of `a` -/ invOf_mul_self : invOf * a = 1 /-- `invOf a` is a right inverse of `a` -/ mul_invOf_self : a * invOf = 1 /-- The inverse of an `Invertible` element -/ prefix:max "⅟" =>-- This notation has the same precedence as `Inv.inv`. Invertible.invOf @[simp] theorem invOf_mul_self' [Mul α] [One α] (a : α) {_ : Invertible a} : ⅟ a * a = 1 := Invertible.invOf_mul_self theorem invOf_mul_self [Mul α] [One α] (a : α) [Invertible a] : ⅟ a * a = 1 := Invertible.invOf_mul_self @[simp] theorem mul_invOf_self' [Mul α] [One α] (a : α) {_ : Invertible a} : a * ⅟ a = 1 := Invertible.mul_invOf_self theorem mul_invOf_self [Mul α] [One α] (a : α) [Invertible a] : a * ⅟ a = 1 := Invertible.mul_invOf_self @[simp] theorem invOf_mul_self_assoc' [Monoid α] (a b : α) {_ : Invertible a} : ⅟ a * (a * b) = b := by rw [← mul_assoc, invOf_mul_self, one_mul] theorem invOf_mul_self_assoc [Monoid α] (a b : α) [Invertible a] : ⅟ a * (a * b) = b := by rw [← mul_assoc, invOf_mul_self, one_mul] @[simp] theorem mul_invOf_self_assoc' [Monoid α] (a b : α) {_ : Invertible a} : a * (⅟ a * b) = b := by rw [← mul_assoc, mul_invOf_self, one_mul] theorem mul_invOf_self_assoc [Monoid α] (a b : α) [Invertible a] : a * (⅟ a * b) = b := by rw [← mul_assoc, mul_invOf_self, one_mul] @[simp] theorem mul_invOf_mul_self_cancel' [Monoid α] (a b : α) {_ : Invertible b} : a * ⅟ b * b = a := by simp [mul_assoc] theorem mul_invOf_mul_self_cancel [Monoid α] (a b : α) [Invertible b] : a * ⅟ b * b = a := by simp [mul_assoc] @[simp] theorem mul_mul_invOf_self_cancel' [Monoid α] (a b : α) {_ : Invertible b} : a * b * ⅟ b = a := by simp [mul_assoc] theorem mul_mul_invOf_self_cancel [Monoid α] (a b : α) [Invertible b] : a * b * ⅟ b = a := by simp [mul_assoc] theorem invOf_eq_right_inv [Monoid α] {a b : α} [Invertible a] (hac : a * b = 1) : ⅟ a = b := left_inv_eq_right_inv (invOf_mul_self _) hac theorem invOf_eq_left_inv [Monoid α] {a b : α} [Invertible a] (hac : b * a = 1) : ⅟ a = b := (left_inv_eq_right_inv hac (mul_invOf_self _)).symm theorem invertible_unique {α : Type u} [Monoid α] (a b : α) [Invertible a] [Invertible b] (h : a = b) : ⅟ a = ⅟ b := by apply invOf_eq_right_inv rw [h, mul_invOf_self] instance Invertible.subsingleton [Monoid α] (a : α) : Subsingleton (Invertible a) := ⟨fun ⟨b, hba, hab⟩ ⟨c, _, hac⟩ => by congr exact left_inv_eq_right_inv hba hac⟩ /-- If `a` is invertible and `a = b`, then `⅟a = ⅟b`. -/ @[congr] theorem Invertible.congr [Monoid α] (a b : α) [Invertible a] [Invertible b] (h : a = b) : ⅟a = ⅟b := by subst h; congr; apply Subsingleton.allEq /-- If `r` is invertible and `s = r` and `si = ⅟r`, then `s` is invertible with `⅟s = si`. -/ def Invertible.copy' [MulOneClass α] {r : α} (hr : Invertible r) (s : α) (si : α) (hs : s = r) (hsi : si = ⅟ r) : Invertible s where invOf := si invOf_mul_self := by rw [hs, hsi, invOf_mul_self] mul_invOf_self := by rw [hs, hsi, mul_invOf_self] /-- If `r` is invertible and `s = r`, then `s` is invertible. -/ abbrev Invertible.copy [MulOneClass α] {r : α} (hr : Invertible r) (s : α) (hs : s = r) : Invertible s := hr.copy' _ _ hs rfl /-- Each element of a group is invertible. -/ def invertibleOfGroup [Group α] (a : α) : Invertible a := ⟨a⁻¹, inv_mul_self a, mul_inv_self a⟩ @[simp] theorem invOf_eq_group_inv [Group α] (a : α) [Invertible a] : ⅟ a = a⁻¹ := invOf_eq_right_inv (mul_inv_self a) /-- `1` is the inverse of itself -/ def invertibleOne [Monoid α] : Invertible (1 : α) := ⟨1, mul_one _, one_mul _⟩ @[simp] theorem invOf_one' [Monoid α] {_ : Invertible (1 : α)} : ⅟ (1 : α) = 1 := invOf_eq_right_inv (mul_one _) theorem invOf_one [Monoid α] [Invertible (1 : α)] : ⅟ (1 : α) = 1 := invOf_eq_right_inv (mul_one _) /-- `a` is the inverse of `⅟a`. -/ instance invertibleInvOf [One α] [Mul α] {a : α} [Invertible a] : Invertible (⅟ a) := ⟨a, mul_invOf_self a, invOf_mul_self a⟩ @[simp] theorem invOf_invOf [Monoid α] (a : α) [Invertible a] [Invertible (⅟ a)] : ⅟ (⅟ a) = a := invOf_eq_right_inv (invOf_mul_self _) @[simp] theorem invOf_inj [Monoid α] {a b : α} [Invertible a] [Invertible b] : ⅟ a = ⅟ b ↔ a = b := ⟨invertible_unique _ _, invertible_unique _ _⟩ /-- `⅟b * ⅟a` is the inverse of `a * b` -/ def invertibleMul [Monoid α] (a b : α) [Invertible a] [Invertible b] : Invertible (a * b) := ⟨⅟ b * ⅟ a, by simp [← mul_assoc], by simp [← mul_assoc]⟩ @[simp] theorem invOf_mul [Monoid α] (a b : α) [Invertible a] [Invertible b] [Invertible (a * b)] : ⅟ (a * b) = ⅟ b * ⅟ a := invOf_eq_right_inv (by simp [← mul_assoc]) /-- A copy of `invertibleMul` for dot notation. -/ abbrev Invertible.mul [Monoid α] {a b : α} (_ : Invertible a) (_ : Invertible b) : Invertible (a * b) := invertibleMul _ _ section variable [Monoid α] {a b c : α} [Invertible c] variable (c) in theorem mul_right_inj_of_invertible : a * c = b * c ↔ a = b := ⟨fun h => by simpa using congr_arg (· * ⅟c) h, congr_arg (· * _)⟩ variable (c) in theorem mul_left_inj_of_invertible : c * a = c * b ↔ a = b := ⟨fun h => by simpa using congr_arg (⅟c * ·) h, congr_arg (_ * ·)⟩ theorem invOf_mul_eq_iff_eq_mul_left : ⅟c * a = b ↔ a = c * b := by rw [← mul_left_inj_of_invertible (c := c), mul_invOf_self_assoc] theorem mul_left_eq_iff_eq_invOf_mul : c * a = b ↔ a = ⅟c * b := by rw [← mul_left_inj_of_invertible (c := ⅟c), invOf_mul_self_assoc] theorem mul_invOf_eq_iff_eq_mul_right : a * ⅟c = b ↔ a = b * c := by rw [← mul_right_inj_of_invertible (c := c), mul_invOf_mul_self_cancel] theorem mul_right_eq_iff_eq_mul_invOf : a * c = b ↔ a = b * ⅟c := by rw [← mul_right_inj_of_invertible (c := ⅟c), mul_mul_invOf_self_cancel] end
Algebra\Group\Pi\Basic.lean
/- Copyright (c) 2020 Eric Wieser. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Simon Hudon, Patrick Massot, Eric Wieser -/ import Mathlib.Algebra.Group.Defs import Mathlib.Data.Prod.Basic import Mathlib.Data.Sum.Basic import Mathlib.Logic.Unique import Mathlib.Tactic.Spread import Batteries.Tactic.Classical /-! # Instances and theorems on pi types This file provides instances for the typeclass defined in `Algebra.Group.Defs`. More sophisticated instances are defined in `Algebra.Group.Pi.Lemmas` files elsewhere. ## Porting note This file relied on the `pi_instance` tactic, which was not available at the time of porting. The comment `--pi_instance` is inserted before all fields which were previously derived by `pi_instance`. See this Zulip discussion: [https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/not.20porting.20pi_instance] -/ -- We enforce to only import `Algebra.Group.Defs` and basic logic assert_not_exists Set.range assert_not_exists MonoidHom assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered open Function universe u v₁ v₂ v₃ variable {I : Type u} -- The indexing type variable {α β γ : Type*} -- The families of types already equipped with instances variable {f : I → Type v₁} {g : I → Type v₂} {h : I → Type v₃} variable (x y : ∀ i, f i) (i : I) namespace Pi /-! `1`, `0`, `+`, `*`, `+ᵥ`, `•`, `^`, `-`, `⁻¹`, and `/` are defined pointwise. -/ @[to_additive] instance instOne [∀ i, One <| f i] : One (∀ i : I, f i) := ⟨fun _ => 1⟩ #adaptation_note /-- After https://github.com/leanprover/lean4/pull/4481 the `simpNF` linter incorrectly claims this lemma can't be applied by `simp`. -/ @[to_additive (attr := simp, nolint simpNF)] theorem one_apply [∀ i, One <| f i] : (1 : ∀ i, f i) i = 1 := rfl @[to_additive] theorem one_def [∀ i, One <| f i] : (1 : ∀ i, f i) = fun _ => 1 := rfl @[to_additive (attr := simp)] lemma _root_.Function.const_one [One β] : const α (1 : β) = 1 := rfl @[to_additive (attr := simp)] theorem one_comp [One γ] (x : α → β) : (1 : β → γ) ∘ x = 1 := rfl @[to_additive (attr := simp)] theorem comp_one [One β] (x : β → γ) : x ∘ (1 : α → β) = const α (x 1) := rfl @[to_additive] instance instMul [∀ i, Mul <| f i] : Mul (∀ i : I, f i) := ⟨fun f g i => f i * g i⟩ @[to_additive (attr := simp)] theorem mul_apply [∀ i, Mul <| f i] : (x * y) i = x i * y i := rfl @[to_additive] theorem mul_def [∀ i, Mul <| f i] : x * y = fun i => x i * y i := rfl @[to_additive (attr := simp)] lemma _root_.Function.const_mul [Mul β] (a b : β) : const α a * const α b = const α (a * b) := rfl @[to_additive] theorem mul_comp [Mul γ] (x y : β → γ) (z : α → β) : (x * y) ∘ z = x ∘ z * y ∘ z := rfl @[to_additive] instance instSMul [∀ i, SMul α <| f i] : SMul α (∀ i : I, f i) := ⟨fun s x => fun i => s • x i⟩ @[to_additive existing instSMul] instance instPow [∀ i, Pow (f i) β] : Pow (∀ i, f i) β := ⟨fun x b i => x i ^ b⟩ @[to_additive (attr := simp, to_additive) (reorder := 5 6) smul_apply] theorem pow_apply [∀ i, Pow (f i) β] (x : ∀ i, f i) (b : β) (i : I) : (x ^ b) i = x i ^ b := rfl @[to_additive (attr := to_additive) (reorder := 5 6) smul_def] theorem pow_def [∀ i, Pow (f i) β] (x : ∀ i, f i) (b : β) : x ^ b = fun i => x i ^ b := rfl @[to_additive (attr := simp, to_additive) (reorder := 2 3, 5 6) smul_const] lemma _root_.Function.const_pow [Pow α β] (a : α) (b : β) : const I a ^ b = const I (a ^ b) := rfl @[to_additive (attr := to_additive) (reorder := 6 7) smul_comp] theorem pow_comp [Pow γ α] (x : β → γ) (a : α) (y : I → β) : (x ^ a) ∘ y = x ∘ y ^ a := rfl -- Use `Pi.ofNat_apply` instead @[to_additive] instance instInv [∀ i, Inv <| f i] : Inv (∀ i : I, f i) := ⟨fun f i => (f i)⁻¹⟩ @[to_additive (attr := simp)] theorem inv_apply [∀ i, Inv <| f i] : x⁻¹ i = (x i)⁻¹ := rfl @[to_additive] theorem inv_def [∀ i, Inv <| f i] : x⁻¹ = fun i => (x i)⁻¹ := rfl @[to_additive] lemma _root_.Function.const_inv [Inv β] (a : β) : (const α a)⁻¹ = const α a⁻¹ := rfl @[to_additive] theorem inv_comp [Inv γ] (x : β → γ) (y : α → β) : x⁻¹ ∘ y = (x ∘ y)⁻¹ := rfl @[to_additive] instance instDiv [∀ i, Div <| f i] : Div (∀ i : I, f i) := ⟨fun f g i => f i / g i⟩ @[to_additive (attr := simp)] theorem div_apply [∀ i, Div <| f i] : (x / y) i = x i / y i := rfl @[to_additive] theorem div_def [∀ i, Div <| f i] : x / y = fun i => x i / y i := rfl @[to_additive] theorem div_comp [Div γ] (x y : β → γ) (z : α → β) : (x / y) ∘ z = x ∘ z / y ∘ z := rfl @[to_additive (attr := simp)] lemma _root_.Function.const_div [Div β] (a b : β) : const α a / const α b = const α (a / b) := rfl @[to_additive] instance semigroup [∀ i, Semigroup (f i)] : Semigroup (∀ i, f i) where mul_assoc := by intros; ext; exact mul_assoc _ _ _ @[to_additive] instance commSemigroup [∀ i, CommSemigroup (f i)] : CommSemigroup (∀ i, f i) where mul_comm := by intros; ext; exact mul_comm _ _ @[to_additive] instance mulOneClass [∀ i, MulOneClass (f i)] : MulOneClass (∀ i, f i) where one_mul := by intros; ext; exact one_mul _ mul_one := by intros; ext; exact mul_one _ @[to_additive] instance invOneClass [∀ i, InvOneClass (f i)] : InvOneClass (∀ i, f i) where inv_one := by ext; exact inv_one @[to_additive] instance monoid [∀ i, Monoid (f i)] : Monoid (∀ i, f i) where __ := semigroup __ := mulOneClass npow := fun n x i => x i ^ n npow_zero := by intros; ext; exact Monoid.npow_zero _ npow_succ := by intros; ext; exact Monoid.npow_succ _ _ @[to_additive] instance commMonoid [∀ i, CommMonoid (f i)] : CommMonoid (∀ i, f i) := { monoid, commSemigroup with } @[to_additive Pi.subNegMonoid] instance divInvMonoid [∀ i, DivInvMonoid (f i)] : DivInvMonoid (∀ i, f i) where zpow := fun z x i => x i ^ z div_eq_mul_inv := by intros; ext; exact div_eq_mul_inv _ _ zpow_zero' := by intros; ext; exact DivInvMonoid.zpow_zero' _ zpow_succ' := by intros; ext; exact DivInvMonoid.zpow_succ' _ _ zpow_neg' := by intros; ext; exact DivInvMonoid.zpow_neg' _ _ @[to_additive Pi.subNegZeroMonoid] instance divInvOneMonoid [∀ i, DivInvOneMonoid (f i)] : DivInvOneMonoid (∀ i, f i) where inv_one := by ext; exact inv_one @[to_additive] instance involutiveInv [∀ i, InvolutiveInv (f i)] : InvolutiveInv (∀ i, f i) where inv_inv := by intros; ext; exact inv_inv _ @[to_additive Pi.subtractionMonoid] instance divisionMonoid [∀ i, DivisionMonoid (f i)] : DivisionMonoid (∀ i, f i) where __ := divInvMonoid __ := involutiveInv mul_inv_rev := by intros; ext; exact mul_inv_rev _ _ inv_eq_of_mul := by intros _ _ h; ext; exact DivisionMonoid.inv_eq_of_mul _ _ (congrFun h _) @[to_additive instSubtractionCommMonoid] instance divisionCommMonoid [∀ i, DivisionCommMonoid (f i)] : DivisionCommMonoid (∀ i, f i) := { divisionMonoid, commSemigroup with } @[to_additive] instance group [∀ i, Group (f i)] : Group (∀ i, f i) where mul_left_inv := by intros; ext; exact mul_left_inv _ @[to_additive] instance commGroup [∀ i, CommGroup (f i)] : CommGroup (∀ i, f i) := { group, commMonoid with } @[to_additive] instance instIsLeftCancelMul [∀ i, Mul (f i)] [∀ i, IsLeftCancelMul (f i)] : IsLeftCancelMul (∀ i, f i) where mul_left_cancel _ _ _ h := funext fun _ ↦ mul_left_cancel (congr_fun h _) @[to_additive] instance instIsRightCancelMul [∀ i, Mul (f i)] [∀ i, IsRightCancelMul (f i)] : IsRightCancelMul (∀ i, f i) where mul_right_cancel _ _ _ h := funext fun _ ↦ mul_right_cancel (congr_fun h _) @[to_additive] instance instIsCancelMul [∀ i, Mul (f i)] [∀ i, IsCancelMul (f i)] : IsCancelMul (∀ i, f i) where @[to_additive] instance leftCancelSemigroup [∀ i, LeftCancelSemigroup (f i)] : LeftCancelSemigroup (∀ i, f i) := { semigroup with mul_left_cancel := fun _ _ _ => mul_left_cancel } @[to_additive] instance rightCancelSemigroup [∀ i, RightCancelSemigroup (f i)] : RightCancelSemigroup (∀ i, f i) := { semigroup with mul_right_cancel := fun _ _ _ => mul_right_cancel } @[to_additive] instance leftCancelMonoid [∀ i, LeftCancelMonoid (f i)] : LeftCancelMonoid (∀ i, f i) := { leftCancelSemigroup, monoid with } @[to_additive] instance rightCancelMonoid [∀ i, RightCancelMonoid (f i)] : RightCancelMonoid (∀ i, f i) := { rightCancelSemigroup, monoid with } @[to_additive] instance cancelMonoid [∀ i, CancelMonoid (f i)] : CancelMonoid (∀ i, f i) := { leftCancelMonoid, rightCancelMonoid with } @[to_additive] instance cancelCommMonoid [∀ i, CancelCommMonoid (f i)] : CancelCommMonoid (∀ i, f i) := { leftCancelMonoid, commMonoid with } section variable [DecidableEq I] variable [∀ i, One (f i)] [∀ i, One (g i)] [∀ i, One (h i)] /-- The function supported at `i`, with value `x` there, and `1` elsewhere. -/ @[to_additive "The function supported at `i`, with value `x` there, and `0` elsewhere."] def mulSingle (i : I) (x : f i) : ∀ (j : I), f j := Function.update 1 i x @[to_additive (attr := simp)] theorem mulSingle_eq_same (i : I) (x : f i) : mulSingle i x i = x := Function.update_same i x _ @[to_additive (attr := simp)] theorem mulSingle_eq_of_ne {i i' : I} (h : i' ≠ i) (x : f i) : mulSingle i x i' = 1 := Function.update_noteq h x _ /-- Abbreviation for `mulSingle_eq_of_ne h.symm`, for ease of use by `simp`. -/ @[to_additive (attr := simp) "Abbreviation for `single_eq_of_ne h.symm`, for ease of use by `simp`."] theorem mulSingle_eq_of_ne' {i i' : I} (h : i ≠ i') (x : f i) : mulSingle i x i' = 1 := mulSingle_eq_of_ne h.symm x @[to_additive (attr := simp)] theorem mulSingle_one (i : I) : mulSingle i (1 : f i) = 1 := Function.update_eq_self _ _ -- Porting note: -- 1) Why do I have to specify the type of `mulSingle i x` explicitly? -- 2) Why do I have to specify the type of `(1 : I → β)`? -- 3) Removed `{β : Sort*}` as `[One β]` converts it to a type anyways. /-- On non-dependent functions, `Pi.mulSingle` can be expressed as an `ite` -/ @[to_additive "On non-dependent functions, `Pi.single` can be expressed as an `ite`"] theorem mulSingle_apply [One β] (i : I) (x : β) (i' : I) : (mulSingle i x : I → β) i' = if i' = i then x else 1 := Function.update_apply (1 : I → β) i x i' -- Porting note: Same as above. /-- On non-dependent functions, `Pi.mulSingle` is symmetric in the two indices. -/ @[to_additive "On non-dependent functions, `Pi.single` is symmetric in the two indices."] theorem mulSingle_comm [One β] (i : I) (x : β) (i' : I) : (mulSingle i x : I → β) i' = (mulSingle i' x : I → β) i := by simp [mulSingle_apply, eq_comm] @[to_additive] theorem apply_mulSingle (f' : ∀ i, f i → g i) (hf' : ∀ i, f' i 1 = 1) (i : I) (x : f i) (j : I) : f' j (mulSingle i x j) = mulSingle i (f' i x) j := by simpa only [Pi.one_apply, hf', mulSingle] using Function.apply_update f' 1 i x j @[to_additive apply_single₂] theorem apply_mulSingle₂ (f' : ∀ i, f i → g i → h i) (hf' : ∀ i, f' i 1 1 = 1) (i : I) (x : f i) (y : g i) (j : I) : f' j (mulSingle i x j) (mulSingle i y j) = mulSingle i (f' i x y) j := by by_cases h : j = i · subst h simp only [mulSingle_eq_same] · simp only [mulSingle_eq_of_ne h, hf'] @[to_additive] theorem mulSingle_op {g : I → Type*} [∀ i, One (g i)] (op : ∀ i, f i → g i) (h : ∀ i, op i 1 = 1) (i : I) (x : f i) : mulSingle i (op i x) = fun j => op j (mulSingle i x j) := Eq.symm <| funext <| apply_mulSingle op h i x @[to_additive] theorem mulSingle_op₂ {g₁ g₂ : I → Type*} [∀ i, One (g₁ i)] [∀ i, One (g₂ i)] (op : ∀ i, g₁ i → g₂ i → f i) (h : ∀ i, op i 1 1 = 1) (i : I) (x₁ : g₁ i) (x₂ : g₂ i) : mulSingle i (op i x₁ x₂) = fun j => op j (mulSingle i x₁ j) (mulSingle i x₂ j) := Eq.symm <| funext <| apply_mulSingle₂ op h i x₁ x₂ variable (f) @[to_additive] theorem mulSingle_injective (i : I) : Function.Injective (mulSingle i : f i → ∀ i, f i) := Function.update_injective _ i @[to_additive (attr := simp)] theorem mulSingle_inj (i : I) {x y : f i} : mulSingle i x = mulSingle i y ↔ x = y := (Pi.mulSingle_injective _ _).eq_iff end /-- The mapping into a product type built from maps into each component. -/ @[simp] protected def prod (f' : ∀ i, f i) (g' : ∀ i, g i) (i : I) : f i × g i := (f' i, g' i) -- Porting note: simp now unfolds the lhs, so we are not marking these as simp. -- @[simp] theorem prod_fst_snd : Pi.prod (Prod.fst : α × β → α) (Prod.snd : α × β → β) = id := rfl -- Porting note: simp now unfolds the lhs, so we are not marking these as simp. -- @[simp] theorem prod_snd_fst : Pi.prod (Prod.snd : α × β → β) (Prod.fst : α × β → α) = Prod.swap := rfl end Pi namespace Function section Extend @[to_additive] theorem extend_one [One γ] (f : α → β) : Function.extend f (1 : α → γ) (1 : β → γ) = 1 := funext fun _ => by apply ite_self @[to_additive] theorem extend_mul [Mul γ] (f : α → β) (g₁ g₂ : α → γ) (e₁ e₂ : β → γ) : Function.extend f (g₁ * g₂) (e₁ * e₂) = Function.extend f g₁ e₁ * Function.extend f g₂ e₂ := by classical funext x simp only [not_exists, extend_def, Pi.mul_apply, apply_dite₂, dite_eq_ite, ite_self] -- Porting note: The Lean3 statement was -- `funext <| λ _, by convert (apply_dite2 (*) _ _ _ _ _).symm` -- which converts to -- `funext fun _ => by convert (apply_dite₂ (· * ·) _ _ _ _ _).symm` -- However this does not work, and we're not sure why. @[to_additive] theorem extend_inv [Inv γ] (f : α → β) (g : α → γ) (e : β → γ) : Function.extend f g⁻¹ e⁻¹ = (Function.extend f g e)⁻¹ := by classical funext x simp only [not_exists, extend_def, Pi.inv_apply, apply_dite Inv.inv] -- Porting note: The Lean3 statement was -- `funext <| λ _, by convert (apply_dite has_inv.inv _ _ _).symm` -- which converts to -- `funext fun _ => by convert (apply_dite Inv.inv _ _ _).symm` -- However this does not work, and we're not sure why. @[to_additive] theorem extend_div [Div γ] (f : α → β) (g₁ g₂ : α → γ) (e₁ e₂ : β → γ) : Function.extend f (g₁ / g₂) (e₁ / e₂) = Function.extend f g₁ e₁ / Function.extend f g₂ e₂ := by classical funext x simp [Function.extend_def, apply_dite₂] -- Porting note: The Lean3 statement was -- `funext <| λ _, by convert (apply_dite2 (/) _ _ _ _ _).symm` -- which converts to -- `funext fun _ => by convert (apply_dite₂ (· / ·) _ _ _ _ _).symm` -- However this does not work, and we're not sure why. end Extend theorem surjective_pi_map {F : ∀ i, f i → g i} (hF : ∀ i, Surjective (F i)) : Surjective fun x : ∀ i, f i => fun i => F i (x i) := fun y => ⟨fun i => (hF i (y i)).choose, funext fun i => (hF i (y i)).choose_spec⟩ theorem injective_pi_map {F : ∀ i, f i → g i} (hF : ∀ i, Injective (F i)) : Injective fun x : ∀ i, f i => fun i => F i (x i) := fun _ _ h => funext fun i => hF i <| (congr_fun h i : _) theorem bijective_pi_map {F : ∀ i, f i → g i} (hF : ∀ i, Bijective (F i)) : Bijective fun x : ∀ i, f i => fun i => F i (x i) := ⟨injective_pi_map fun i => (hF i).injective, surjective_pi_map fun i => (hF i).surjective⟩ lemma comp_eq_const_iff (b : β) (f : α → β) {g : β → γ} (hg : Injective g) : g ∘ f = Function.const _ (g b) ↔ f = Function.const _ b := hg.comp_left.eq_iff' rfl @[to_additive] lemma comp_eq_one_iff [One β] [One γ] (f : α → β) {g : β → γ} (hg : Injective g) (hg0 : g 1 = 1) : g ∘ f = 1 ↔ f = 1 := by simpa [hg0, const_one] using comp_eq_const_iff 1 f hg @[to_additive] lemma comp_ne_one_iff [One β] [One γ] (f : α → β) {g : β → γ} (hg : Injective g) (hg0 : g 1 = 1) : g ∘ f ≠ 1 ↔ f ≠ 1 := (comp_eq_one_iff f hg hg0).ne end Function /-- If the one function is surjective, the codomain is trivial. -/ @[to_additive "If the zero function is surjective, the codomain is trivial."] def uniqueOfSurjectiveOne (α : Type*) {β : Type*} [One β] (h : Function.Surjective (1 : α → β)) : Unique β := h.uniqueOfSurjectiveConst α (1 : β) @[to_additive] theorem Subsingleton.pi_mulSingle_eq {α : Type*} [DecidableEq I] [Subsingleton I] [One α] (i : I) (x : α) : Pi.mulSingle i x = fun _ => x := funext fun j => by rw [Subsingleton.elim j i, Pi.mulSingle_eq_same] namespace Sum variable (a a' : α → γ) (b b' : β → γ) @[to_additive (attr := simp)] theorem elim_one_one [One γ] : Sum.elim (1 : α → γ) (1 : β → γ) = 1 := Sum.elim_const_const 1 @[to_additive (attr := simp)] theorem elim_mulSingle_one [DecidableEq α] [DecidableEq β] [One γ] (i : α) (c : γ) : Sum.elim (Pi.mulSingle i c) (1 : β → γ) = Pi.mulSingle (Sum.inl i) c := by simp only [Pi.mulSingle, Sum.elim_update_left, elim_one_one] @[to_additive (attr := simp)] theorem elim_one_mulSingle [DecidableEq α] [DecidableEq β] [One γ] (i : β) (c : γ) : Sum.elim (1 : α → γ) (Pi.mulSingle i c) = Pi.mulSingle (Sum.inr i) c := by simp only [Pi.mulSingle, Sum.elim_update_right, elim_one_one] @[to_additive] theorem elim_inv_inv [Inv γ] : Sum.elim a⁻¹ b⁻¹ = (Sum.elim a b)⁻¹ := (Sum.comp_elim Inv.inv a b).symm @[to_additive] theorem elim_mul_mul [Mul γ] : Sum.elim (a * a') (b * b') = Sum.elim a b * Sum.elim a' b' := by ext x cases x <;> rfl @[to_additive] theorem elim_div_div [Div γ] : Sum.elim (a / a') (b / b') = Sum.elim a b / Sum.elim a' b' := by ext x cases x <;> rfl end Sum
Algebra\Group\Pi\Lemmas.lean
/- Copyright (c) 2018 Simon Hudon. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Simon Hudon, Patrick Massot -/ import Mathlib.Algebra.Group.Commute.Defs import Mathlib.Algebra.Group.Hom.Instances import Mathlib.Data.Set.Function import Mathlib.Logic.Pairwise /-! # Extra lemmas about products of monoids and groups This file proves lemmas about the instances defined in `Algebra.Group.Pi.Basic` that require more imports. -/ assert_not_exists AddMonoidWithOne assert_not_exists MonoidWithZero universe u v w variable {ι α : Type*} variable {I : Type u} -- The indexing type variable {f : I → Type v} -- The family of types already equipped with instances variable (x y : ∀ i, f i) (i j : I) @[to_additive (attr := simp)] theorem Set.range_one {α β : Type*} [One β] [Nonempty α] : Set.range (1 : α → β) = {1} := range_const @[to_additive] theorem Set.preimage_one {α β : Type*} [One β] (s : Set β) [Decidable ((1 : β) ∈ s)] : (1 : α → β) ⁻¹' s = if (1 : β) ∈ s then Set.univ else ∅ := Set.preimage_const 1 s namespace MulHom @[to_additive] theorem coe_mul {M N} {_ : Mul M} {_ : CommSemigroup N} (f g : M →ₙ* N) : (f * g : M → N) = fun x => f x * g x := rfl end MulHom section MulHom /-- A family of MulHom's `f a : γ →ₙ* β a` defines a MulHom `Pi.mulHom f : γ →ₙ* Π a, β a` given by `Pi.mulHom f x b = f b x`. -/ @[to_additive (attr := simps) "A family of AddHom's `f a : γ → β a` defines an AddHom `Pi.addHom f : γ → Π a, β a` given by `Pi.addHom f x b = f b x`."] def Pi.mulHom {γ : Type w} [∀ i, Mul (f i)] [Mul γ] (g : ∀ i, γ →ₙ* f i) : γ →ₙ* ∀ i, f i where toFun x i := g i x map_mul' x y := funext fun i => (g i).map_mul x y @[to_additive] theorem Pi.mulHom_injective {γ : Type w} [Nonempty I] [∀ i, Mul (f i)] [Mul γ] (g : ∀ i, γ →ₙ* f i) (hg : ∀ i, Function.Injective (g i)) : Function.Injective (Pi.mulHom g) := fun x y h => let ⟨i⟩ := ‹Nonempty I› hg i ((Function.funext_iff.mp h : _) i) /-- A family of monoid homomorphisms `f a : γ →* β a` defines a monoid homomorphism `Pi.monoidHom f : γ →* Π a, β a` given by `Pi.monoidHom f x b = f b x`. -/ @[to_additive (attr := simps) "A family of additive monoid homomorphisms `f a : γ →+ β a` defines a monoid homomorphism `Pi.addMonoidHom f : γ →+ Π a, β a` given by `Pi.addMonoidHom f x b = f b x`."] def Pi.monoidHom {γ : Type w} [∀ i, MulOneClass (f i)] [MulOneClass γ] (g : ∀ i, γ →* f i) : γ →* ∀ i, f i := { Pi.mulHom fun i => (g i).toMulHom with toFun := fun x i => g i x map_one' := funext fun i => (g i).map_one } @[to_additive] theorem Pi.monoidHom_injective {γ : Type w} [Nonempty I] [∀ i, MulOneClass (f i)] [MulOneClass γ] (g : ∀ i, γ →* f i) (hg : ∀ i, Function.Injective (g i)) : Function.Injective (Pi.monoidHom g) := Pi.mulHom_injective (fun i => (g i).toMulHom) hg variable (f) variable [(i : I) → Mul (f i)] /-- Evaluation of functions into an indexed collection of semigroups at a point is a semigroup homomorphism. This is `Function.eval i` as a `MulHom`. -/ @[to_additive (attr := simps) "Evaluation of functions into an indexed collection of additive semigroups at a point is an additive semigroup homomorphism. This is `Function.eval i` as an `AddHom`."] def Pi.evalMulHom (i : I) : (∀ i, f i) →ₙ* f i where toFun g := g i map_mul' _ _ := Pi.mul_apply _ _ i /-- `Function.const` as a `MulHom`. -/ @[to_additive (attr := simps) "`Function.const` as an `AddHom`."] def Pi.constMulHom (α β : Type*) [Mul β] : β →ₙ* α → β where toFun := Function.const α map_mul' _ _ := rfl /-- Coercion of a `MulHom` into a function is itself a `MulHom`. See also `MulHom.eval`. -/ @[to_additive (attr := simps) "Coercion of an `AddHom` into a function is itself an `AddHom`. See also `AddHom.eval`."] def MulHom.coeFn (α β : Type*) [Mul α] [CommSemigroup β] : (α →ₙ* β) →ₙ* α → β where toFun g := g map_mul' _ _ := rfl /-- Semigroup homomorphism between the function spaces `I → α` and `I → β`, induced by a semigroup homomorphism `f` between `α` and `β`. -/ @[to_additive (attr := simps) "Additive semigroup homomorphism between the function spaces `I → α` and `I → β`, induced by an additive semigroup homomorphism `f` between `α` and `β`"] protected def MulHom.compLeft {α β : Type*} [Mul α] [Mul β] (f : α →ₙ* β) (I : Type*) : (I → α) →ₙ* I → β where toFun h := f ∘ h map_mul' _ _ := by ext; simp end MulHom section MonoidHom variable (f) variable [(i : I) → MulOneClass (f i)] /-- Evaluation of functions into an indexed collection of monoids at a point is a monoid homomorphism. This is `Function.eval i` as a `MonoidHom`. -/ @[to_additive (attr := simps) "Evaluation of functions into an indexed collection of additive monoids at a point is an additive monoid homomorphism. This is `Function.eval i` as an `AddMonoidHom`."] def Pi.evalMonoidHom (i : I) : (∀ i, f i) →* f i where toFun g := g i map_one' := Pi.one_apply i map_mul' _ _ := Pi.mul_apply _ _ i /-- `Function.const` as a `MonoidHom`. -/ @[to_additive (attr := simps) "`Function.const` as an `AddMonoidHom`."] def Pi.constMonoidHom (α β : Type*) [MulOneClass β] : β →* α → β where toFun := Function.const α map_one' := rfl map_mul' _ _ := rfl /-- Coercion of a `MonoidHom` into a function is itself a `MonoidHom`. See also `MonoidHom.eval`. -/ @[to_additive (attr := simps) "Coercion of an `AddMonoidHom` into a function is itself an `AddMonoidHom`. See also `AddMonoidHom.eval`."] def MonoidHom.coeFn (α β : Type*) [MulOneClass α] [CommMonoid β] : (α →* β) →* α → β where toFun g := g map_one' := rfl map_mul' _ _ := rfl /-- Monoid homomorphism between the function spaces `I → α` and `I → β`, induced by a monoid homomorphism `f` between `α` and `β`. -/ @[to_additive (attr := simps) "Additive monoid homomorphism between the function spaces `I → α` and `I → β`, induced by an additive monoid homomorphism `f` between `α` and `β`"] protected def MonoidHom.compLeft {α β : Type*} [MulOneClass α] [MulOneClass β] (f : α →* β) (I : Type*) : (I → α) →* I → β where toFun h := f ∘ h map_one' := by ext; dsimp; simp map_mul' _ _ := by ext; simp end MonoidHom section Single variable [DecidableEq I] open Pi variable (f) /-- The one-preserving homomorphism including a single value into a dependent family of values, as functions supported at a point. This is the `OneHom` version of `Pi.mulSingle`. -/ @[to_additive "The zero-preserving homomorphism including a single value into a dependent family of values, as functions supported at a point. This is the `ZeroHom` version of `Pi.single`."] nonrec def OneHom.mulSingle [∀ i, One <| f i] (i : I) : OneHom (f i) (∀ i, f i) where toFun := mulSingle i map_one' := mulSingle_one i @[to_additive (attr := simp)] theorem OneHom.mulSingle_apply [∀ i, One <| f i] (i : I) (x : f i) : mulSingle f i x = Pi.mulSingle i x := rfl /-- The monoid homomorphism including a single monoid into a dependent family of additive monoids, as functions supported at a point. This is the `MonoidHom` version of `Pi.mulSingle`. -/ @[to_additive "The additive monoid homomorphism including a single additive monoid into a dependent family of additive monoids, as functions supported at a point. This is the `AddMonoidHom` version of `Pi.single`."] def MonoidHom.mulSingle [∀ i, MulOneClass <| f i] (i : I) : f i →* ∀ i, f i := { OneHom.mulSingle f i with map_mul' := mulSingle_op₂ (fun _ => (· * ·)) (fun _ => one_mul _) _ } @[to_additive (attr := simp)] theorem MonoidHom.mulSingle_apply [∀ i, MulOneClass <| f i] (i : I) (x : f i) : mulSingle f i x = Pi.mulSingle i x := rfl variable {f} @[to_additive] theorem Pi.mulSingle_sup [∀ i, SemilatticeSup (f i)] [∀ i, One (f i)] (i : I) (x y : f i) : Pi.mulSingle i (x ⊔ y) = Pi.mulSingle i x ⊔ Pi.mulSingle i y := Function.update_sup _ _ _ _ @[to_additive] theorem Pi.mulSingle_inf [∀ i, SemilatticeInf (f i)] [∀ i, One (f i)] (i : I) (x y : f i) : Pi.mulSingle i (x ⊓ y) = Pi.mulSingle i x ⊓ Pi.mulSingle i y := Function.update_inf _ _ _ _ @[to_additive] theorem Pi.mulSingle_mul [∀ i, MulOneClass <| f i] (i : I) (x y : f i) : mulSingle i (x * y) = mulSingle i x * mulSingle i y := (MonoidHom.mulSingle f i).map_mul x y @[to_additive] theorem Pi.mulSingle_inv [∀ i, Group <| f i] (i : I) (x : f i) : mulSingle i x⁻¹ = (mulSingle i x)⁻¹ := (MonoidHom.mulSingle f i).map_inv x @[to_additive] theorem Pi.mulSingle_div [∀ i, Group <| f i] (i : I) (x y : f i) : mulSingle i (x / y) = mulSingle i x / mulSingle i y := (MonoidHom.mulSingle f i).map_div x y /-- The injection into a pi group at different indices commutes. For injections of commuting elements at the same index, see `Commute.map` -/ @[to_additive "The injection into an additive pi group at different indices commutes. For injections of commuting elements at the same index, see `AddCommute.map`"] theorem Pi.mulSingle_commute [∀ i, MulOneClass <| f i] : Pairwise fun i j => ∀ (x : f i) (y : f j), Commute (mulSingle i x) (mulSingle j y) := by intro i j hij x y; ext k by_cases h1 : i = k · subst h1 simp [hij] by_cases h2 : j = k · subst h2 simp [hij] simp [h1, h2] /-- The injection into a pi group with the same values commutes. -/ @[to_additive "The injection into an additive pi group with the same values commutes."] theorem Pi.mulSingle_apply_commute [∀ i, MulOneClass <| f i] (x : ∀ i, f i) (i j : I) : Commute (mulSingle i (x i)) (mulSingle j (x j)) := by obtain rfl | hij := Decidable.eq_or_ne i j · rfl · exact Pi.mulSingle_commute hij _ _ @[to_additive] theorem Pi.update_eq_div_mul_mulSingle [∀ i, Group <| f i] (g : ∀ i : I, f i) (x : f i) : Function.update g i x = g / mulSingle i (g i) * mulSingle i x := by ext j rcases eq_or_ne i j with (rfl | h) · simp · simp [Function.update_noteq h.symm, h] @[to_additive] theorem Pi.mulSingle_mul_mulSingle_eq_mulSingle_mul_mulSingle {M : Type*} [CommMonoid M] {k l m n : I} {u v : M} (hu : u ≠ 1) (hv : v ≠ 1) : (mulSingle k u : I → M) * mulSingle l v = mulSingle m u * mulSingle n v ↔ k = m ∧ l = n ∨ u = v ∧ k = n ∧ l = m ∨ u * v = 1 ∧ k = l ∧ m = n := by refine ⟨fun h => ?_, ?_⟩ · have hk := congr_fun h k have hl := congr_fun h l have hm := (congr_fun h m).symm have hn := (congr_fun h n).symm simp only [mul_apply, mulSingle_apply, if_pos rfl] at hk hl hm hn rcases eq_or_ne k m with (rfl | hkm) · refine Or.inl ⟨rfl, not_ne_iff.mp fun hln => (hv ?_).elim⟩ rcases eq_or_ne k l with (rfl | hkl) · rwa [if_neg hln.symm, if_neg hln.symm, one_mul, one_mul] at hn · rwa [if_neg hkl.symm, if_neg hln, one_mul, one_mul] at hl · rcases eq_or_ne m n with (rfl | hmn) · rcases eq_or_ne k l with (rfl | hkl) · rw [if_neg hkm.symm, if_neg hkm.symm, one_mul, if_pos rfl] at hm exact Or.inr (Or.inr ⟨hm, rfl, rfl⟩) · simp only [if_neg hkm, if_neg hkl, mul_one] at hk dsimp at hk contradiction · rw [if_neg hkm.symm, if_neg hmn, one_mul, mul_one] at hm obtain rfl := (ite_ne_right_iff.mp (ne_of_eq_of_ne hm.symm hu)).1 rw [if_neg hkm, if_neg hkm, one_mul, mul_one] at hk obtain rfl := (ite_ne_right_iff.mp (ne_of_eq_of_ne hk.symm hu)).1 exact Or.inr (Or.inl ⟨hk.trans (if_pos rfl), rfl, rfl⟩) · rintro (⟨rfl, rfl⟩ | ⟨rfl, rfl, rfl⟩ | ⟨h, rfl, rfl⟩) · rfl · apply mul_comm · simp_rw [← Pi.mulSingle_mul, h, mulSingle_one] end Single section variable [∀ i, Mul <| f i] @[to_additive] theorem SemiconjBy.pi {x y z : ∀ i, f i} (h : ∀ i, SemiconjBy (x i) (y i) (z i)) : SemiconjBy x y z := funext h @[to_additive] theorem Pi.semiconjBy_iff {x y z : ∀ i, f i} : SemiconjBy x y z ↔ ∀ i, SemiconjBy (x i) (y i) (z i) := Function.funext_iff @[to_additive] theorem Commute.pi {x y : ∀ i, f i} (h : ∀ i, Commute (x i) (y i)) : Commute x y := .pi h @[to_additive] theorem Pi.commute_iff {x y : ∀ i, f i} : Commute x y ↔ ∀ i, Commute (x i) (y i) := semiconjBy_iff end namespace Function @[to_additive (attr := simp)] theorem update_one [∀ i, One (f i)] [DecidableEq I] (i : I) : update (1 : ∀ i, f i) i 1 = 1 := update_eq_self i (1 : (a : I) → f a) @[to_additive] theorem update_mul [∀ i, Mul (f i)] [DecidableEq I] (f₁ f₂ : ∀ i, f i) (i : I) (x₁ : f i) (x₂ : f i) : update (f₁ * f₂) i (x₁ * x₂) = update f₁ i x₁ * update f₂ i x₂ := funext fun j => (apply_update₂ (fun _ => (· * ·)) f₁ f₂ i x₁ x₂ j).symm @[to_additive] theorem update_inv [∀ i, Inv (f i)] [DecidableEq I] (f₁ : ∀ i, f i) (i : I) (x₁ : f i) : update f₁⁻¹ i x₁⁻¹ = (update f₁ i x₁)⁻¹ := funext fun j => (apply_update (fun _ => Inv.inv) f₁ i x₁ j).symm @[to_additive] theorem update_div [∀ i, Div (f i)] [DecidableEq I] (f₁ f₂ : ∀ i, f i) (i : I) (x₁ : f i) (x₂ : f i) : update (f₁ / f₂) i (x₁ / x₂) = update f₁ i x₁ / update f₂ i x₂ := funext fun j => (apply_update₂ (fun _ => (· / ·)) f₁ f₂ i x₁ x₂ j).symm variable [One α] [Nonempty ι] {a : α} @[to_additive (attr := simp)] theorem const_eq_one : const ι a = 1 ↔ a = 1 := @const_inj _ _ _ _ 1 @[to_additive] theorem const_ne_one : const ι a ≠ 1 ↔ a ≠ 1 := Iff.not const_eq_one end Function section Piecewise @[to_additive] theorem Set.piecewise_mul [∀ i, Mul (f i)] (s : Set I) [∀ i, Decidable (i ∈ s)] (f₁ f₂ g₁ g₂ : ∀ i, f i) : s.piecewise (f₁ * f₂) (g₁ * g₂) = s.piecewise f₁ g₁ * s.piecewise f₂ g₂ := s.piecewise_op₂ f₁ _ _ _ fun _ => (· * ·) @[to_additive] theorem Set.piecewise_inv [∀ i, Inv (f i)] (s : Set I) [∀ i, Decidable (i ∈ s)] (f₁ g₁ : ∀ i, f i) : s.piecewise f₁⁻¹ g₁⁻¹ = (s.piecewise f₁ g₁)⁻¹ := s.piecewise_op f₁ g₁ fun _ x => x⁻¹ @[to_additive] theorem Set.piecewise_div [∀ i, Div (f i)] (s : Set I) [∀ i, Decidable (i ∈ s)] (f₁ f₂ g₁ g₂ : ∀ i, f i) : s.piecewise (f₁ / f₂) (g₁ / g₂) = s.piecewise f₁ g₁ / s.piecewise f₂ g₂ := s.piecewise_op₂ f₁ _ _ _ fun _ => (· / ·) end Piecewise section Extend variable {η : Type v} (R : Type w) (s : ι → η) /-- `Function.extend s f 1` as a bundled hom. -/ @[to_additive (attr := simps) Function.ExtendByZero.hom "`Function.extend s f 0` as a bundled hom."] noncomputable def Function.ExtendByOne.hom [MulOneClass R] : (ι → R) →* η → R where toFun f := Function.extend s f 1 map_one' := Function.extend_one s map_mul' f g := by simpa using Function.extend_mul s f g 1 1 end Extend namespace Pi variable [DecidableEq I] [∀ i, Preorder (f i)] [∀ i, One (f i)] @[to_additive] theorem mulSingle_mono : Monotone (Pi.mulSingle i : f i → ∀ i, f i) := Function.update_mono @[to_additive] theorem mulSingle_strictMono : StrictMono (Pi.mulSingle i : f i → ∀ i, f i) := Function.update_strictMono end Pi namespace Sigma variable {α : Type*} {β : α → Type*} {γ : ∀ a, β a → Type*} @[to_additive (attr := simp)] theorem curry_one [∀ a b, One (γ a b)] : Sigma.curry (1 : (i : Σ a, β a) → γ i.1 i.2) = 1 := rfl @[to_additive (attr := simp)] theorem uncurry_one [∀ a b, One (γ a b)] : Sigma.uncurry (1 : ∀ a b, γ a b) = 1 := rfl @[to_additive (attr := simp)] theorem curry_mul [∀ a b, Mul (γ a b)] (x y : (i : Σ a, β a) → γ i.1 i.2) : Sigma.curry (x * y) = Sigma.curry x * Sigma.curry y := rfl @[to_additive (attr := simp)] theorem uncurry_mul [∀ a b, Mul (γ a b)] (x y : ∀ a b, γ a b) : Sigma.uncurry (x * y) = Sigma.uncurry x * Sigma.uncurry y := rfl @[to_additive (attr := simp)] theorem curry_inv [∀ a b, Inv (γ a b)] (x : (i : Σ a, β a) → γ i.1 i.2) : Sigma.curry (x⁻¹) = (Sigma.curry x)⁻¹ := rfl @[to_additive (attr := simp)] theorem uncurry_inv [∀ a b, Inv (γ a b)] (x : ∀ a b, γ a b) : Sigma.uncurry (x⁻¹) = (Sigma.uncurry x)⁻¹ := rfl @[to_additive (attr := simp)] theorem curry_mulSingle [DecidableEq α] [∀ a, DecidableEq (β a)] [∀ a b, One (γ a b)] (i : Σ a, β a) (x : γ i.1 i.2) : Sigma.curry (Pi.mulSingle i x) = Pi.mulSingle i.1 (Pi.mulSingle i.2 x) := by simp only [Pi.mulSingle, Sigma.curry_update, Sigma.curry_one, Pi.one_apply] @[to_additive (attr := simp)] theorem uncurry_mulSingle_mulSingle [DecidableEq α] [∀ a, DecidableEq (β a)] [∀ a b, One (γ a b)] (a : α) (b : β a) (x : γ a b) : Sigma.uncurry (Pi.mulSingle a (Pi.mulSingle b x)) = Pi.mulSingle (Sigma.mk a b) x := by rw [← curry_mulSingle ⟨a, b⟩, uncurry_curry] end Sigma
Algebra\Group\Semiconj\Basic.lean
/- Copyright (c) 2019 Yury Kudryashov. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Yury Kudryashov -/ import Mathlib.Algebra.Group.Semiconj.Defs import Mathlib.Algebra.Group.Basic /-! # Lemmas about semiconjugate elements of a group -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered namespace SemiconjBy variable {G : Type*} section DivisionMonoid variable [DivisionMonoid G] {a x y : G} @[to_additive (attr := simp)] theorem inv_inv_symm_iff : SemiconjBy a⁻¹ x⁻¹ y⁻¹ ↔ SemiconjBy a y x := by simp_rw [SemiconjBy, ← mul_inv_rev, inv_inj, eq_comm] @[to_additive] alias ⟨_, inv_inv_symm⟩ := inv_inv_symm_iff end DivisionMonoid section Group variable [Group G] {a x y : G} @[to_additive (attr := simp)] lemma inv_symm_left_iff : SemiconjBy a⁻¹ y x ↔ SemiconjBy a x y := by simp_rw [SemiconjBy, eq_mul_inv_iff_mul_eq, mul_assoc, inv_mul_eq_iff_eq_mul, eq_comm] @[to_additive] alias ⟨_, inv_symm_left⟩ := inv_symm_left_iff @[to_additive (attr := simp)] lemma inv_right_iff : SemiconjBy a x⁻¹ y⁻¹ ↔ SemiconjBy a x y := by rw [← inv_symm_left_iff, inv_inv_symm_iff] @[to_additive] alias ⟨_, inv_right⟩ := inv_right_iff @[to_additive (attr := simp)] lemma zpow_right (h : SemiconjBy a x y) : ∀ m : ℤ, SemiconjBy a (x ^ m) (y ^ m) | (n : ℕ) => by simp [zpow_natCast, h.pow_right n] | .negSucc n => by simp only [zpow_negSucc, inv_right_iff] apply pow_right h variable (a) in @[to_additive] lemma eq_one_iff (h : SemiconjBy a x y): x = 1 ↔ y = 1 := by rw [← conj_eq_one_iff (a := a) (b := x), h.eq, mul_inv_cancel_right] end Group end SemiconjBy
Algebra\Group\Semiconj\Defs.lean
/- Copyright (c) 2019 Yury Kudryashov. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Yury Kudryashov Some proofs and docs came from `Algebra/Commute` (c) Neil Strickland -/ import Mathlib.Algebra.Group.Defs import Mathlib.Init.Logic import Mathlib.Tactic.Cases /-! # Semiconjugate elements of a semigroup ## Main definitions We say that `x` is semiconjugate to `y` by `a` (`SemiconjBy a x y`), if `a * x = y * a`. In this file we provide operations on `SemiconjBy _ _ _`. In the names of these operations, we treat `a` as the “left” argument, and both `x` and `y` as “right” arguments. This way most names in this file agree with the names of the corresponding lemmas for `Commute a b = SemiconjBy a b b`. As a side effect, some lemmas have only `_right` version. Lean does not immediately recognise these terms as equations, so for rewriting we need syntax like `rw [(h.pow_right 5).eq]` rather than just `rw [h.pow_right 5]`. This file provides only basic operations (`mul_left`, `mul_right`, `inv_right` etc). Other operations (`pow_right`, field inverse etc) are in the files that define corresponding notions. -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered variable {S M G : Type*} /-- `x` is semiconjugate to `y` by `a`, if `a * x = y * a`. -/ @[to_additive "`x` is additive semiconjugate to `y` by `a` if `a + x = y + a`"] def SemiconjBy [Mul M] (a x y : M) : Prop := a * x = y * a namespace SemiconjBy /-- Equality behind `SemiconjBy a x y`; useful for rewriting. -/ @[to_additive "Equality behind `AddSemiconjBy a x y`; useful for rewriting."] protected theorem eq [Mul S] {a x y : S} (h : SemiconjBy a x y) : a * x = y * a := h section Semigroup variable [Semigroup S] {a b x y z x' y' : S} /-- If `a` semiconjugates `x` to `y` and `x'` to `y'`, then it semiconjugates `x * x'` to `y * y'`. -/ @[to_additive (attr := simp) "If `a` semiconjugates `x` to `y` and `x'` to `y'`, then it semiconjugates `x + x'` to `y + y'`."] theorem mul_right (h : SemiconjBy a x y) (h' : SemiconjBy a x' y') : SemiconjBy a (x * x') (y * y') := by unfold SemiconjBy -- TODO this could be done using `assoc_rw` if/when this is ported to mathlib4 rw [← mul_assoc, h.eq, mul_assoc, h'.eq, ← mul_assoc] /-- If `b` semiconjugates `x` to `y` and `a` semiconjugates `y` to `z`, then `a * b` semiconjugates `x` to `z`. -/ @[to_additive "If `b` semiconjugates `x` to `y` and `a` semiconjugates `y` to `z`, then `a + b` semiconjugates `x` to `z`."] theorem mul_left (ha : SemiconjBy a y z) (hb : SemiconjBy b x y) : SemiconjBy (a * b) x z := by unfold SemiconjBy rw [mul_assoc, hb.eq, ← mul_assoc, ha.eq, mul_assoc] /-- The relation “there exists an element that semiconjugates `a` to `b`” on a semigroup is transitive. -/ @[to_additive "The relation “there exists an element that semiconjugates `a` to `b`” on an additive semigroup is transitive."] protected theorem transitive : Transitive fun a b : S ↦ ∃ c, SemiconjBy c a b | _, _, _, ⟨x, hx⟩, ⟨y, hy⟩ => ⟨y * x, hy.mul_left hx⟩ end Semigroup section MulOneClass variable [MulOneClass M] /-- Any element semiconjugates `1` to `1`. -/ @[to_additive (attr := simp) "Any element semiconjugates `0` to `0`."] theorem one_right (a : M) : SemiconjBy a 1 1 := by rw [SemiconjBy, mul_one, one_mul] /-- One semiconjugates any element to itself. -/ @[to_additive (attr := simp) "Zero semiconjugates any element to itself."] theorem one_left (x : M) : SemiconjBy 1 x x := Eq.symm <| one_right x /-- The relation “there exists an element that semiconjugates `a` to `b`” on a monoid (or, more generally, on `MulOneClass` type) is reflexive. -/ @[to_additive "The relation “there exists an element that semiconjugates `a` to `b`” on an additive monoid (or, more generally, on an `AddZeroClass` type) is reflexive."] protected theorem reflexive : Reflexive fun a b : M ↦ ∃ c, SemiconjBy c a b | a => ⟨1, one_left a⟩ end MulOneClass section Monoid variable [Monoid M] @[to_additive (attr := simp)] theorem pow_right {a x y : M} (h : SemiconjBy a x y) (n : ℕ) : SemiconjBy a (x ^ n) (y ^ n) := by induction' n with n ih · rw [pow_zero, pow_zero] exact SemiconjBy.one_right _ · rw [pow_succ, pow_succ] exact ih.mul_right h end Monoid section Group variable [Group G] {a x y : G} /-- `a` semiconjugates `x` to `a * x * a⁻¹`. -/ @[to_additive "`a` semiconjugates `x` to `a + x + -a`."] theorem conj_mk (a x : G) : SemiconjBy a x (a * x * a⁻¹) := by unfold SemiconjBy; rw [mul_assoc, inv_mul_self, mul_one] @[to_additive (attr := simp)] theorem conj_iff {a x y b : G} : SemiconjBy (b * a * b⁻¹) (b * x * b⁻¹) (b * y * b⁻¹) ↔ SemiconjBy a x y := by unfold SemiconjBy simp only [← mul_assoc, inv_mul_cancel_right] repeat rw [mul_assoc] rw [mul_left_cancel_iff, ← mul_assoc, ← mul_assoc, mul_right_cancel_iff] end Group end SemiconjBy @[to_additive (attr := simp)] theorem semiconjBy_iff_eq [CancelCommMonoid M] {a x y : M} : SemiconjBy a x y ↔ x = y := ⟨fun h => mul_left_cancel (h.trans (mul_comm _ _)), fun h => by rw [h, SemiconjBy, mul_comm]⟩
Algebra\Group\Semiconj\Units.lean
/- Copyright (c) 2019 Yury Kudryashov. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Yury Kudryashov Some proofs and docs came from `Algebra/Commute` (c) Neil Strickland -/ import Mathlib.Algebra.Group.Semiconj.Defs import Mathlib.Algebra.Group.Units /-! # Semiconjugate elements of a semigroup ## Main definitions We say that `x` is semiconjugate to `y` by `a` (`SemiconjBy a x y`), if `a * x = y * a`. In this file we provide operations on `SemiconjBy _ _ _`. In the names of these operations, we treat `a` as the “left” argument, and both `x` and `y` as “right” arguments. This way most names in this file agree with the names of the corresponding lemmas for `Commute a b = SemiconjBy a b b`. As a side effect, some lemmas have only `_right` version. Lean does not immediately recognise these terms as equations, so for rewriting we need syntax like `rw [(h.pow_right 5).eq]` rather than just `rw [h.pow_right 5]`. This file provides only basic operations (`mul_left`, `mul_right`, `inv_right` etc). Other operations (`pow_right`, field inverse etc) are in the files that define corresponding notions. -/ assert_not_exists MonoidWithZero assert_not_exists DenselyOrdered open scoped Int variable {M G : Type*} namespace SemiconjBy section Monoid variable [Monoid M] /-- If `a` semiconjugates a unit `x` to a unit `y`, then it semiconjugates `x⁻¹` to `y⁻¹`. -/ @[to_additive "If `a` semiconjugates an additive unit `x` to an additive unit `y`, then it semiconjugates `-x` to `-y`."] theorem units_inv_right {a : M} {x y : Mˣ} (h : SemiconjBy a x y) : SemiconjBy a ↑x⁻¹ ↑y⁻¹ := calc a * ↑x⁻¹ = ↑y⁻¹ * (y * a) * ↑x⁻¹ := by rw [Units.inv_mul_cancel_left] _ = ↑y⁻¹ * a := by rw [← h.eq, mul_assoc, Units.mul_inv_cancel_right] @[to_additive (attr := simp)] theorem units_inv_right_iff {a : M} {x y : Mˣ} : SemiconjBy a ↑x⁻¹ ↑y⁻¹ ↔ SemiconjBy a x y := ⟨units_inv_right, units_inv_right⟩ /-- If a unit `a` semiconjugates `x` to `y`, then `a⁻¹` semiconjugates `y` to `x`. -/ @[to_additive "If an additive unit `a` semiconjugates `x` to `y`, then `-a` semiconjugates `y` to `x`."] theorem units_inv_symm_left {a : Mˣ} {x y : M} (h : SemiconjBy (↑a) x y) : SemiconjBy (↑a⁻¹) y x := calc ↑a⁻¹ * y = ↑a⁻¹ * (y * a * ↑a⁻¹) := by rw [Units.mul_inv_cancel_right] _ = x * ↑a⁻¹ := by rw [← h.eq, ← mul_assoc, Units.inv_mul_cancel_left] @[to_additive (attr := simp)] theorem units_inv_symm_left_iff {a : Mˣ} {x y : M} : SemiconjBy (↑a⁻¹) y x ↔ SemiconjBy (↑a) x y := ⟨units_inv_symm_left, units_inv_symm_left⟩ @[to_additive] theorem units_val {a x y : Mˣ} (h : SemiconjBy a x y) : SemiconjBy (a : M) x y := congr_arg Units.val h @[to_additive] theorem units_of_val {a x y : Mˣ} (h : SemiconjBy (a : M) x y) : SemiconjBy a x y := Units.ext h @[to_additive (attr := simp)] theorem units_val_iff {a x y : Mˣ} : SemiconjBy (a : M) x y ↔ SemiconjBy a x y := ⟨units_of_val, units_val⟩ @[to_additive (attr := simp)] lemma units_zpow_right {a : M} {x y : Mˣ} (h : SemiconjBy a x y) : ∀ m : ℤ, SemiconjBy a ↑(x ^ m) ↑(y ^ m) | (n : ℕ) => by simp only [zpow_natCast, Units.val_pow_eq_pow_val, h, pow_right] | -[n+1] => by simp only [zpow_negSucc, Units.val_pow_eq_pow_val, units_inv_right, h, pow_right] end Monoid end SemiconjBy namespace Units variable [Monoid M] /-- `a` semiconjugates `x` to `a * x * a⁻¹`. -/ @[to_additive "`a` semiconjugates `x` to `a + x + -a`."] lemma mk_semiconjBy (u : Mˣ) (x : M) : SemiconjBy (↑u) x (u * x * ↑u⁻¹) := by unfold SemiconjBy; rw [Units.inv_mul_cancel_right] lemma conj_pow (u : Mˣ) (x : M) (n : ℕ) : ((↑u : M) * x * (↑u⁻¹ : M)) ^ n = (u : M) * x ^ n * (↑u⁻¹ : M) := eq_divp_iff_mul_eq.2 ((u.mk_semiconjBy x).pow_right n).eq.symm lemma conj_pow' (u : Mˣ) (x : M) (n : ℕ) : ((↑u⁻¹ : M) * x * (u : M)) ^ n = (↑u⁻¹ : M) * x ^ n * (u : M) := u⁻¹.conj_pow x n end Units
Algebra\Group\Subgroup\Actions.lean
/- Copyright (c) 2021 Eric Wieser. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Eric Wieser -/ import Mathlib.Algebra.Group.Submonoid.DistribMulAction import Mathlib.GroupTheory.Subgroup.Center /-! # Actions by `Subgroup`s These are just copies of the definitions about `Submonoid` starting from `Submonoid.mulAction`. ## Tags subgroup, subgroups -/ namespace Subgroup variable {G α β : Type*} [Group G] section MulAction variable [MulAction G α] {S : Subgroup G} /-- The action by a subgroup is the action by the underlying group. -/ @[to_additive "The additive action by an add_subgroup is the action by the underlying `AddGroup`. "] instance instMulAction : MulAction S α := inferInstanceAs (MulAction S.toSubmonoid α) @[to_additive] lemma smul_def (g : S) (m : α) : g • m = (g : G) • m := rfl @[to_additive (attr := simp)] lemma mk_smul (g : G) (hg : g ∈ S) (a : α) : (⟨g, hg⟩ : S) • a = g • a := rfl end MulAction @[to_additive] instance smulCommClass_left [MulAction G β] [SMul α β] [SMulCommClass G α β] (S : Subgroup G) : SMulCommClass S α β := S.toSubmonoid.smulCommClass_left @[to_additive] instance smulCommClass_right [SMul α β] [MulAction G β] [SMulCommClass α G β] (S : Subgroup G) : SMulCommClass α S β := S.toSubmonoid.smulCommClass_right /-- Note that this provides `IsScalarTower S G G` which is needed by `smul_mul_assoc`. -/ instance [SMul α β] [MulAction G α] [MulAction G β] [IsScalarTower G α β] (S : Subgroup G) : IsScalarTower S α β := inferInstanceAs (IsScalarTower S.toSubmonoid α β) instance [MulAction G α] [FaithfulSMul G α] (S : Subgroup G) : FaithfulSMul S α := inferInstanceAs (FaithfulSMul S.toSubmonoid α) /-- The action by a subgroup is the action by the underlying group. -/ instance [AddMonoid α] [DistribMulAction G α] (S : Subgroup G) : DistribMulAction S α := inferInstanceAs (DistribMulAction S.toSubmonoid α) /-- The action by a subgroup is the action by the underlying group. -/ instance [Monoid α] [MulDistribMulAction G α] (S : Subgroup G) : MulDistribMulAction S α := inferInstanceAs (MulDistribMulAction S.toSubmonoid α) /-- The center of a group acts commutatively on that group. -/ instance center.smulCommClass_left : SMulCommClass (center G) G G := Submonoid.center.smulCommClass_left /-- The center of a group acts commutatively on that group. -/ instance center.smulCommClass_right : SMulCommClass G (center G) G := Submonoid.center.smulCommClass_right end Subgroup
Algebra\Group\Subgroup\Basic.lean
/- Copyright (c) 2020 Kexing Ying. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Kexing Ying -/ import Mathlib.Algebra.Group.Conj import Mathlib.Algebra.Group.Pi.Lemmas import Mathlib.Algebra.Group.Subsemigroup.Operations import Mathlib.Algebra.Group.Submonoid.Operations import Mathlib.Data.Set.Image import Mathlib.Tactic.ApplyFun /-! # Subgroups This file defines multiplicative and additive subgroups as an extension of submonoids, in a bundled form (unbundled subgroups are in `Deprecated/Subgroups.lean`). We prove subgroups of a group form a complete lattice, and results about images and preimages of subgroups under group homomorphisms. The bundled subgroups use bundled monoid homomorphisms. There are also theorems about the subgroups generated by an element or a subset of a group, defined both inductively and as the infimum of the set of subgroups containing a given element/subset. Special thanks goes to Amelia Livingston and Yury Kudryashov for their help and inspiration. ## Main definitions Notation used here: - `G N` are `Group`s - `A` is an `AddGroup` - `H K` are `Subgroup`s of `G` or `AddSubgroup`s of `A` - `x` is an element of type `G` or type `A` - `f g : N →* G` are group homomorphisms - `s k` are sets of elements of type `G` Definitions in the file: * `Subgroup G` : the type of subgroups of a group `G` * `AddSubgroup A` : the type of subgroups of an additive group `A` * `CompleteLattice (Subgroup G)` : the subgroups of `G` form a complete lattice * `Subgroup.closure k` : the minimal subgroup that includes the set `k` * `Subgroup.subtype` : the natural group homomorphism from a subgroup of group `G` to `G` * `Subgroup.gi` : `closure` forms a Galois insertion with the coercion to set * `Subgroup.comap H f` : the preimage of a subgroup `H` along the group homomorphism `f` is also a subgroup * `Subgroup.map f H` : the image of a subgroup `H` along the group homomorphism `f` is also a subgroup * `Subgroup.prod H K` : the product of subgroups `H`, `K` of groups `G`, `N` respectively, `H × K` is a subgroup of `G × N` * `MonoidHom.range f` : the range of the group homomorphism `f` is a subgroup * `MonoidHom.ker f` : the kernel of a group homomorphism `f` is the subgroup of elements `x : G` such that `f x = 1` * `MonoidHom.eq_locus f g` : given group homomorphisms `f`, `g`, the elements of `G` such that `f x = g x` form a subgroup of `G` ## Implementation notes Subgroup inclusion is denoted `≤` rather than `⊆`, although `∈` is defined as membership of a subgroup's underlying set. ## Tags subgroup, subgroups -/ assert_not_exists OrderedAddCommMonoid open Function open Int variable {G G' G'' : Type*} [Group G] [Group G'] [Group G''] variable {A : Type*} [AddGroup A] section SubgroupClass /-- `InvMemClass S G` states `S` is a type of subsets `s ⊆ G` closed under inverses. -/ class InvMemClass (S G : Type*) [Inv G] [SetLike S G] : Prop where /-- `s` is closed under inverses -/ inv_mem : ∀ {s : S} {x}, x ∈ s → x⁻¹ ∈ s export InvMemClass (inv_mem) /-- `NegMemClass S G` states `S` is a type of subsets `s ⊆ G` closed under negation. -/ class NegMemClass (S G : Type*) [Neg G] [SetLike S G] : Prop where /-- `s` is closed under negation -/ neg_mem : ∀ {s : S} {x}, x ∈ s → -x ∈ s export NegMemClass (neg_mem) /-- `SubgroupClass S G` states `S` is a type of subsets `s ⊆ G` that are subgroups of `G`. -/ class SubgroupClass (S G : Type*) [DivInvMonoid G] [SetLike S G] extends SubmonoidClass S G, InvMemClass S G : Prop /-- `AddSubgroupClass S G` states `S` is a type of subsets `s ⊆ G` that are additive subgroups of `G`. -/ class AddSubgroupClass (S G : Type*) [SubNegMonoid G] [SetLike S G] extends AddSubmonoidClass S G, NegMemClass S G : Prop attribute [to_additive] InvMemClass SubgroupClass attribute [aesop safe apply (rule_sets := [SetLike])] inv_mem neg_mem @[to_additive (attr := simp)] theorem inv_mem_iff {S G} [InvolutiveInv G] {_ : SetLike S G} [InvMemClass S G] {H : S} {x : G} : x⁻¹ ∈ H ↔ x ∈ H := ⟨fun h => inv_inv x ▸ inv_mem h, inv_mem⟩ variable {M S : Type*} [DivInvMonoid M] [SetLike S M] [hSM : SubgroupClass S M] {H K : S} /-- A subgroup is closed under division. -/ @[to_additive (attr := aesop safe apply (rule_sets := [SetLike])) "An additive subgroup is closed under subtraction."] theorem div_mem {x y : M} (hx : x ∈ H) (hy : y ∈ H) : x / y ∈ H := by rw [div_eq_mul_inv]; exact mul_mem hx (inv_mem hy) @[to_additive (attr := aesop safe apply (rule_sets := [SetLike]))] theorem zpow_mem {x : M} (hx : x ∈ K) : ∀ n : ℤ, x ^ n ∈ K | (n : ℕ) => by rw [zpow_natCast] exact pow_mem hx n | -[n+1] => by rw [zpow_negSucc] exact inv_mem (pow_mem hx n.succ) variable [SetLike S G] [SubgroupClass S G] @[to_additive] theorem div_mem_comm_iff {a b : G} : a / b ∈ H ↔ b / a ∈ H := inv_div b a ▸ inv_mem_iff @[to_additive /-(attr := simp)-/] -- Porting note: `simp` cannot simplify LHS theorem exists_inv_mem_iff_exists_mem {P : G → Prop} : (∃ x : G, x ∈ H ∧ P x⁻¹) ↔ ∃ x ∈ H, P x := by constructor <;> · rintro ⟨x, x_in, hx⟩ exact ⟨x⁻¹, inv_mem x_in, by simp [hx]⟩ @[to_additive] theorem mul_mem_cancel_right {x y : G} (h : x ∈ H) : y * x ∈ H ↔ y ∈ H := ⟨fun hba => by simpa using mul_mem hba (inv_mem h), fun hb => mul_mem hb h⟩ @[to_additive] theorem mul_mem_cancel_left {x y : G} (h : x ∈ H) : x * y ∈ H ↔ y ∈ H := ⟨fun hab => by simpa using mul_mem (inv_mem h) hab, mul_mem h⟩ namespace InvMemClass /-- A subgroup of a group inherits an inverse. -/ @[to_additive "An additive subgroup of an `AddGroup` inherits an inverse."] instance inv {G : Type u_1} {S : Type u_2} [Inv G] [SetLike S G] [InvMemClass S G] {H : S} : Inv H := ⟨fun a => ⟨a⁻¹, inv_mem a.2⟩⟩ @[to_additive (attr := simp, norm_cast)] theorem coe_inv (x : H) : (x⁻¹).1 = x.1⁻¹ := rfl end InvMemClass namespace SubgroupClass @[to_additive (attr := deprecated (since := "2024-01-15"))] alias coe_inv := InvMemClass.coe_inv -- Here we assume H, K, and L are subgroups, but in fact any one of them -- could be allowed to be a subsemigroup. -- Counterexample where K and L are submonoids: H = ℤ, K = ℕ, L = -ℕ -- Counterexample where H and K are submonoids: H = {n | n = 0 ∨ 3 ≤ n}, K = 3ℕ + 4ℕ, L = 5ℤ @[to_additive] theorem subset_union {H K L : S} : (H : Set G) ⊆ K ∪ L ↔ H ≤ K ∨ H ≤ L := by refine ⟨fun h ↦ ?_, fun h x xH ↦ h.imp (· xH) (· xH)⟩ rw [or_iff_not_imp_left, SetLike.not_le_iff_exists] exact fun ⟨x, xH, xK⟩ y yH ↦ (h <| mul_mem xH yH).elim ((h yH).resolve_left fun yK ↦ xK <| (mul_mem_cancel_right yK).mp ·) (mul_mem_cancel_left <| (h xH).resolve_left xK).mp /-- A subgroup of a group inherits a division -/ @[to_additive "An additive subgroup of an `AddGroup` inherits a subtraction."] instance div {G : Type u_1} {S : Type u_2} [DivInvMonoid G] [SetLike S G] [SubgroupClass S G] {H : S} : Div H := ⟨fun a b => ⟨a / b, div_mem a.2 b.2⟩⟩ /-- An additive subgroup of an `AddGroup` inherits an integer scaling. -/ instance _root_.AddSubgroupClass.zsmul {M S} [SubNegMonoid M] [SetLike S M] [AddSubgroupClass S M] {H : S} : SMul ℤ H := ⟨fun n a => ⟨n • a.1, zsmul_mem a.2 n⟩⟩ /-- A subgroup of a group inherits an integer power. -/ @[to_additive existing] instance zpow {M S} [DivInvMonoid M] [SetLike S M] [SubgroupClass S M] {H : S} : Pow H ℤ := ⟨fun a n => ⟨a.1 ^ n, zpow_mem a.2 n⟩⟩ @[to_additive (attr := simp, norm_cast)] theorem coe_div (x y : H) : (x / y).1 = x.1 / y.1 := rfl variable (H) -- Prefer subclasses of `Group` over subclasses of `SubgroupClass`. /-- A subgroup of a group inherits a group structure. -/ @[to_additive "An additive subgroup of an `AddGroup` inherits an `AddGroup` structure."] instance (priority := 75) toGroup : Group H := Subtype.coe_injective.group _ rfl (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) fun _ _ => rfl -- Prefer subclasses of `CommGroup` over subclasses of `SubgroupClass`. /-- A subgroup of a `CommGroup` is a `CommGroup`. -/ @[to_additive "An additive subgroup of an `AddCommGroup` is an `AddCommGroup`."] instance (priority := 75) toCommGroup {G : Type*} [CommGroup G] [SetLike S G] [SubgroupClass S G] : CommGroup H := Subtype.coe_injective.commGroup _ rfl (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) fun _ _ => rfl /-- The natural group hom from a subgroup of group `G` to `G`. -/ @[to_additive (attr := coe) "The natural group hom from an additive subgroup of `AddGroup` `G` to `G`."] protected def subtype : H →* G where toFun := ((↑) : H → G); map_one' := rfl; map_mul' := fun _ _ => rfl @[to_additive (attr := simp)] theorem coeSubtype : (SubgroupClass.subtype H : H → G) = ((↑) : H → G) := by rfl variable {H} @[to_additive (attr := simp, norm_cast)] theorem coe_pow (x : H) (n : ℕ) : ((x ^ n : H) : G) = (x : G) ^ n := rfl @[to_additive (attr := simp, norm_cast)] theorem coe_zpow (x : H) (n : ℤ) : ((x ^ n : H) : G) = (x : G) ^ n := rfl /-- The inclusion homomorphism from a subgroup `H` contained in `K` to `K`. -/ @[to_additive "The inclusion homomorphism from an additive subgroup `H` contained in `K` to `K`."] def inclusion {H K : S} (h : H ≤ K) : H →* K := MonoidHom.mk' (fun x => ⟨x, h x.prop⟩) fun _ _=> rfl @[to_additive (attr := simp)] theorem inclusion_self (x : H) : inclusion le_rfl x = x := by cases x rfl @[to_additive (attr := simp)] theorem inclusion_mk {h : H ≤ K} (x : G) (hx : x ∈ H) : inclusion h ⟨x, hx⟩ = ⟨x, h hx⟩ := rfl @[to_additive] theorem inclusion_right (h : H ≤ K) (x : K) (hx : (x : G) ∈ H) : inclusion h ⟨x, hx⟩ = x := by cases x rfl @[simp] theorem inclusion_inclusion {L : S} (hHK : H ≤ K) (hKL : K ≤ L) (x : H) : inclusion hKL (inclusion hHK x) = inclusion (hHK.trans hKL) x := by cases x rfl @[to_additive (attr := simp)] theorem coe_inclusion {H K : S} {h : H ≤ K} (a : H) : (inclusion h a : G) = a := by cases a simp only [inclusion, MonoidHom.mk'_apply] @[to_additive (attr := simp)] theorem subtype_comp_inclusion {H K : S} (hH : H ≤ K) : (SubgroupClass.subtype K).comp (inclusion hH) = SubgroupClass.subtype H := by ext simp only [MonoidHom.comp_apply, coeSubtype, coe_inclusion] end SubgroupClass end SubgroupClass /-- A subgroup of a group `G` is a subset containing 1, closed under multiplication and closed under multiplicative inverse. -/ structure Subgroup (G : Type*) [Group G] extends Submonoid G where /-- `G` is closed under inverses -/ inv_mem' {x} : x ∈ carrier → x⁻¹ ∈ carrier /-- An additive subgroup of an additive group `G` is a subset containing 0, closed under addition and additive inverse. -/ structure AddSubgroup (G : Type*) [AddGroup G] extends AddSubmonoid G where /-- `G` is closed under negation -/ neg_mem' {x} : x ∈ carrier → -x ∈ carrier attribute [to_additive] Subgroup -- Porting note: Removed, translation already exists -- attribute [to_additive AddSubgroup.toAddSubmonoid] Subgroup.toSubmonoid /-- Reinterpret a `Subgroup` as a `Submonoid`. -/ add_decl_doc Subgroup.toSubmonoid /-- Reinterpret an `AddSubgroup` as an `AddSubmonoid`. -/ add_decl_doc AddSubgroup.toAddSubmonoid namespace Subgroup @[to_additive] instance : SetLike (Subgroup G) G where coe s := s.carrier coe_injective' p q h := by obtain ⟨⟨⟨hp,_⟩,_⟩,_⟩ := p obtain ⟨⟨⟨hq,_⟩,_⟩,_⟩ := q congr -- Porting note: Below can probably be written more uniformly @[to_additive] instance : SubgroupClass (Subgroup G) G where inv_mem := Subgroup.inv_mem' _ one_mem _ := (Subgroup.toSubmonoid _).one_mem' mul_mem := (Subgroup.toSubmonoid _).mul_mem' @[to_additive (attr := simp, nolint simpNF)] -- Porting note (#10675): dsimp can not prove this theorem mem_carrier {s : Subgroup G} {x : G} : x ∈ s.carrier ↔ x ∈ s := Iff.rfl @[to_additive (attr := simp)] theorem mem_mk {s : Set G} {x : G} (h_one) (h_mul) (h_inv) : x ∈ mk ⟨⟨s, h_one⟩, h_mul⟩ h_inv ↔ x ∈ s := Iff.rfl @[to_additive (attr := simp, norm_cast)] theorem coe_set_mk {s : Set G} (h_one) (h_mul) (h_inv) : (mk ⟨⟨s, h_one⟩, h_mul⟩ h_inv : Set G) = s := rfl @[to_additive (attr := simp)] theorem mk_le_mk {s t : Set G} (h_one) (h_mul) (h_inv) (h_one') (h_mul') (h_inv') : mk ⟨⟨s, h_one⟩, h_mul⟩ h_inv ≤ mk ⟨⟨t, h_one'⟩, h_mul'⟩ h_inv' ↔ s ⊆ t := Iff.rfl initialize_simps_projections Subgroup (carrier → coe) initialize_simps_projections AddSubgroup (carrier → coe) @[to_additive (attr := simp)] theorem coe_toSubmonoid (K : Subgroup G) : (K.toSubmonoid : Set G) = K := rfl @[to_additive (attr := simp)] theorem mem_toSubmonoid (K : Subgroup G) (x : G) : x ∈ K.toSubmonoid ↔ x ∈ K := Iff.rfl @[to_additive] theorem toSubmonoid_injective : Function.Injective (toSubmonoid : Subgroup G → Submonoid G) := -- fun p q h => SetLike.ext'_iff.2 (show _ from SetLike.ext'_iff.1 h) fun p q h => by have := SetLike.ext'_iff.1 h rw [coe_toSubmonoid, coe_toSubmonoid] at this exact SetLike.ext'_iff.2 this @[to_additive (attr := simp)] theorem toSubmonoid_eq {p q : Subgroup G} : p.toSubmonoid = q.toSubmonoid ↔ p = q := toSubmonoid_injective.eq_iff @[to_additive (attr := mono)] theorem toSubmonoid_strictMono : StrictMono (toSubmonoid : Subgroup G → Submonoid G) := fun _ _ => id @[to_additive (attr := mono)] theorem toSubmonoid_mono : Monotone (toSubmonoid : Subgroup G → Submonoid G) := toSubmonoid_strictMono.monotone @[to_additive (attr := simp)] theorem toSubmonoid_le {p q : Subgroup G} : p.toSubmonoid ≤ q.toSubmonoid ↔ p ≤ q := Iff.rfl @[to_additive (attr := simp)] lemma coe_nonempty (s : Subgroup G) : (s : Set G).Nonempty := ⟨1, one_mem _⟩ end Subgroup /-! ### Conversion to/from `Additive`/`Multiplicative` -/ section mul_add /-- Subgroups of a group `G` are isomorphic to additive subgroups of `Additive G`. -/ @[simps!] def Subgroup.toAddSubgroup : Subgroup G ≃o AddSubgroup (Additive G) where toFun S := { Submonoid.toAddSubmonoid S.toSubmonoid with neg_mem' := S.inv_mem' } invFun S := { AddSubmonoid.toSubmonoid S.toAddSubmonoid with inv_mem' := S.neg_mem' } left_inv x := by cases x; rfl right_inv x := by cases x; rfl map_rel_iff' := Iff.rfl /-- Additive subgroup of an additive group `Additive G` are isomorphic to subgroup of `G`. -/ abbrev AddSubgroup.toSubgroup' : AddSubgroup (Additive G) ≃o Subgroup G := Subgroup.toAddSubgroup.symm /-- Additive subgroups of an additive group `A` are isomorphic to subgroups of `Multiplicative A`. -/ @[simps!] def AddSubgroup.toSubgroup : AddSubgroup A ≃o Subgroup (Multiplicative A) where toFun S := { AddSubmonoid.toSubmonoid S.toAddSubmonoid with inv_mem' := S.neg_mem' } invFun S := { Submonoid.toAddSubmonoid S.toSubmonoid with neg_mem' := S.inv_mem' } left_inv x := by cases x; rfl right_inv x := by cases x; rfl map_rel_iff' := Iff.rfl /-- Subgroups of an additive group `Multiplicative A` are isomorphic to additive subgroups of `A`. -/ abbrev Subgroup.toAddSubgroup' : Subgroup (Multiplicative A) ≃o AddSubgroup A := AddSubgroup.toSubgroup.symm end mul_add namespace Subgroup variable (H K : Subgroup G) /-- Copy of a subgroup with a new `carrier` equal to the old one. Useful to fix definitional equalities. -/ @[to_additive "Copy of an additive subgroup with a new `carrier` equal to the old one. Useful to fix definitional equalities"] protected def copy (K : Subgroup G) (s : Set G) (hs : s = K) : Subgroup G where carrier := s one_mem' := hs.symm ▸ K.one_mem' mul_mem' := hs.symm ▸ K.mul_mem' inv_mem' hx := by simpa [hs] using hx -- Porting note: `▸` didn't work here @[to_additive (attr := simp)] theorem coe_copy (K : Subgroup G) (s : Set G) (hs : s = ↑K) : (K.copy s hs : Set G) = s := rfl @[to_additive] theorem copy_eq (K : Subgroup G) (s : Set G) (hs : s = ↑K) : K.copy s hs = K := SetLike.coe_injective hs /-- Two subgroups are equal if they have the same elements. -/ @[to_additive (attr := ext) "Two `AddSubgroup`s are equal if they have the same elements."] theorem ext {H K : Subgroup G} (h : ∀ x, x ∈ H ↔ x ∈ K) : H = K := SetLike.ext h /-- A subgroup contains the group's 1. -/ @[to_additive "An `AddSubgroup` contains the group's 0."] protected theorem one_mem : (1 : G) ∈ H := one_mem _ /-- A subgroup is closed under multiplication. -/ @[to_additive "An `AddSubgroup` is closed under addition."] protected theorem mul_mem {x y : G} : x ∈ H → y ∈ H → x * y ∈ H := mul_mem /-- A subgroup is closed under inverse. -/ @[to_additive "An `AddSubgroup` is closed under inverse."] protected theorem inv_mem {x : G} : x ∈ H → x⁻¹ ∈ H := inv_mem /-- A subgroup is closed under division. -/ @[to_additive "An `AddSubgroup` is closed under subtraction."] protected theorem div_mem {x y : G} (hx : x ∈ H) (hy : y ∈ H) : x / y ∈ H := div_mem hx hy @[to_additive] protected theorem inv_mem_iff {x : G} : x⁻¹ ∈ H ↔ x ∈ H := inv_mem_iff @[to_additive] protected theorem div_mem_comm_iff {a b : G} : a / b ∈ H ↔ b / a ∈ H := div_mem_comm_iff @[to_additive] protected theorem exists_inv_mem_iff_exists_mem (K : Subgroup G) {P : G → Prop} : (∃ x : G, x ∈ K ∧ P x⁻¹) ↔ ∃ x ∈ K, P x := exists_inv_mem_iff_exists_mem @[to_additive] protected theorem mul_mem_cancel_right {x y : G} (h : x ∈ H) : y * x ∈ H ↔ y ∈ H := mul_mem_cancel_right h @[to_additive] protected theorem mul_mem_cancel_left {x y : G} (h : x ∈ H) : x * y ∈ H ↔ y ∈ H := mul_mem_cancel_left h @[to_additive] protected theorem pow_mem {x : G} (hx : x ∈ K) : ∀ n : ℕ, x ^ n ∈ K := pow_mem hx @[to_additive] protected theorem zpow_mem {x : G} (hx : x ∈ K) : ∀ n : ℤ, x ^ n ∈ K := zpow_mem hx /-- Construct a subgroup from a nonempty set that is closed under division. -/ @[to_additive "Construct a subgroup from a nonempty set that is closed under subtraction"] def ofDiv (s : Set G) (hsn : s.Nonempty) (hs : ∀ᵉ (x ∈ s) (y ∈ s), x * y⁻¹ ∈ s) : Subgroup G := have one_mem : (1 : G) ∈ s := by let ⟨x, hx⟩ := hsn simpa using hs x hx x hx have inv_mem : ∀ x, x ∈ s → x⁻¹ ∈ s := fun x hx => by simpa using hs 1 one_mem x hx { carrier := s one_mem' := one_mem inv_mem' := inv_mem _ mul_mem' := fun hx hy => by simpa using hs _ hx _ (inv_mem _ hy) } /-- A subgroup of a group inherits a multiplication. -/ @[to_additive "An `AddSubgroup` of an `AddGroup` inherits an addition."] instance mul : Mul H := H.toSubmonoid.mul /-- A subgroup of a group inherits a 1. -/ @[to_additive "An `AddSubgroup` of an `AddGroup` inherits a zero."] instance one : One H := H.toSubmonoid.one /-- A subgroup of a group inherits an inverse. -/ @[to_additive "An `AddSubgroup` of an `AddGroup` inherits an inverse."] instance inv : Inv H := ⟨fun a => ⟨a⁻¹, H.inv_mem a.2⟩⟩ /-- A subgroup of a group inherits a division -/ @[to_additive "An `AddSubgroup` of an `AddGroup` inherits a subtraction."] instance div : Div H := ⟨fun a b => ⟨a / b, H.div_mem a.2 b.2⟩⟩ /-- An `AddSubgroup` of an `AddGroup` inherits a natural scaling. -/ instance _root_.AddSubgroup.nsmul {G} [AddGroup G] {H : AddSubgroup G} : SMul ℕ H := ⟨fun n a => ⟨n • a, H.nsmul_mem a.2 n⟩⟩ /-- A subgroup of a group inherits a natural power -/ @[to_additive existing] protected instance npow : Pow H ℕ := ⟨fun a n => ⟨a ^ n, H.pow_mem a.2 n⟩⟩ /-- An `AddSubgroup` of an `AddGroup` inherits an integer scaling. -/ instance _root_.AddSubgroup.zsmul {G} [AddGroup G] {H : AddSubgroup G} : SMul ℤ H := ⟨fun n a => ⟨n • a, H.zsmul_mem a.2 n⟩⟩ /-- A subgroup of a group inherits an integer power -/ @[to_additive existing] instance zpow : Pow H ℤ := ⟨fun a n => ⟨a ^ n, H.zpow_mem a.2 n⟩⟩ @[to_additive (attr := simp, norm_cast)] theorem coe_mul (x y : H) : (↑(x * y) : G) = ↑x * ↑y := rfl @[to_additive (attr := simp, norm_cast)] theorem coe_one : ((1 : H) : G) = 1 := rfl @[to_additive (attr := simp, norm_cast)] theorem coe_inv (x : H) : ↑(x⁻¹ : H) = (x⁻¹ : G) := rfl @[to_additive (attr := simp, norm_cast)] theorem coe_div (x y : H) : (↑(x / y) : G) = ↑x / ↑y := rfl -- Porting note: removed simp, theorem has variable as head symbol @[to_additive (attr := norm_cast)] theorem coe_mk (x : G) (hx : x ∈ H) : ((⟨x, hx⟩ : H) : G) = x := rfl @[to_additive (attr := simp, norm_cast)] theorem coe_pow (x : H) (n : ℕ) : ((x ^ n : H) : G) = (x : G) ^ n := rfl @[to_additive (attr := norm_cast)] -- Porting note (#10685): dsimp can prove this theorem coe_zpow (x : H) (n : ℤ) : ((x ^ n : H) : G) = (x : G) ^ n := rfl @[to_additive] -- This can be proved by `Submonoid.mk_eq_one` theorem mk_eq_one {g : G} {h} : (⟨g, h⟩ : H) = 1 ↔ g = 1 := by simp /-- A subgroup of a group inherits a group structure. -/ @[to_additive "An `AddSubgroup` of an `AddGroup` inherits an `AddGroup` structure."] instance toGroup {G : Type*} [Group G] (H : Subgroup G) : Group H := Subtype.coe_injective.group _ rfl (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) fun _ _ => rfl /-- A subgroup of a `CommGroup` is a `CommGroup`. -/ @[to_additive "An `AddSubgroup` of an `AddCommGroup` is an `AddCommGroup`."] instance toCommGroup {G : Type*} [CommGroup G] (H : Subgroup G) : CommGroup H := Subtype.coe_injective.commGroup _ rfl (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) fun _ _ => rfl /-- The natural group hom from a subgroup of group `G` to `G`. -/ @[to_additive "The natural group hom from an `AddSubgroup` of `AddGroup` `G` to `G`."] protected def subtype : H →* G where toFun := ((↑) : H → G); map_one' := rfl; map_mul' _ _ := rfl @[to_additive (attr := simp)] theorem coeSubtype : ⇑ H.subtype = ((↑) : H → G) := rfl @[to_additive] theorem subtype_injective : Function.Injective (Subgroup.subtype H) := Subtype.coe_injective /-- The inclusion homomorphism from a subgroup `H` contained in `K` to `K`. -/ @[to_additive "The inclusion homomorphism from an additive subgroup `H` contained in `K` to `K`."] def inclusion {H K : Subgroup G} (h : H ≤ K) : H →* K := MonoidHom.mk' (fun x => ⟨x, h x.2⟩) fun _ _ => rfl @[to_additive (attr := simp)] theorem coe_inclusion {H K : Subgroup G} {h : H ≤ K} (a : H) : (inclusion h a : G) = a := by cases a simp only [inclusion, coe_mk, MonoidHom.mk'_apply] @[to_additive] theorem inclusion_injective {H K : Subgroup G} (h : H ≤ K) : Function.Injective <| inclusion h := Set.inclusion_injective h @[to_additive (attr := simp)] theorem subtype_comp_inclusion {H K : Subgroup G} (hH : H ≤ K) : K.subtype.comp (inclusion hH) = H.subtype := rfl /-- The subgroup `G` of the group `G`. -/ @[to_additive "The `AddSubgroup G` of the `AddGroup G`."] instance : Top (Subgroup G) := ⟨{ (⊤ : Submonoid G) with inv_mem' := fun _ => Set.mem_univ _ }⟩ /-- The top subgroup is isomorphic to the group. This is the group version of `Submonoid.topEquiv`. -/ @[to_additive (attr := simps!) "The top additive subgroup is isomorphic to the additive group. This is the additive group version of `AddSubmonoid.topEquiv`."] def topEquiv : (⊤ : Subgroup G) ≃* G := Submonoid.topEquiv /-- The trivial subgroup `{1}` of a group `G`. -/ @[to_additive "The trivial `AddSubgroup` `{0}` of an `AddGroup` `G`."] instance : Bot (Subgroup G) := ⟨{ (⊥ : Submonoid G) with inv_mem' := by simp}⟩ @[to_additive] instance : Inhabited (Subgroup G) := ⟨⊥⟩ @[to_additive (attr := simp)] theorem mem_bot {x : G} : x ∈ (⊥ : Subgroup G) ↔ x = 1 := Iff.rfl @[to_additive (attr := simp)] theorem mem_top (x : G) : x ∈ (⊤ : Subgroup G) := Set.mem_univ x @[to_additive (attr := simp)] theorem coe_top : ((⊤ : Subgroup G) : Set G) = Set.univ := rfl @[to_additive (attr := simp)] theorem coe_bot : ((⊥ : Subgroup G) : Set G) = {1} := rfl @[to_additive] instance : Unique (⊥ : Subgroup G) := ⟨⟨1⟩, fun g => Subtype.ext g.2⟩ @[to_additive (attr := simp)] theorem top_toSubmonoid : (⊤ : Subgroup G).toSubmonoid = ⊤ := rfl @[to_additive (attr := simp)] theorem bot_toSubmonoid : (⊥ : Subgroup G).toSubmonoid = ⊥ := rfl @[to_additive] theorem eq_bot_iff_forall : H = ⊥ ↔ ∀ x ∈ H, x = (1 : G) := toSubmonoid_injective.eq_iff.symm.trans <| Submonoid.eq_bot_iff_forall _ @[to_additive] theorem eq_bot_of_subsingleton [Subsingleton H] : H = ⊥ := by rw [Subgroup.eq_bot_iff_forall] intro y hy rw [← Subgroup.coe_mk H y hy, Subsingleton.elim (⟨y, hy⟩ : H) 1, Subgroup.coe_one] @[to_additive (attr := simp, norm_cast)] theorem coe_eq_univ {H : Subgroup G} : (H : Set G) = Set.univ ↔ H = ⊤ := (SetLike.ext'_iff.trans (by rfl)).symm @[to_additive] theorem coe_eq_singleton {H : Subgroup G} : (∃ g : G, (H : Set G) = {g}) ↔ H = ⊥ := ⟨fun ⟨g, hg⟩ => haveI : Subsingleton (H : Set G) := by rw [hg] infer_instance H.eq_bot_of_subsingleton, fun h => ⟨1, SetLike.ext'_iff.mp h⟩⟩ @[to_additive] theorem nontrivial_iff_exists_ne_one (H : Subgroup G) : Nontrivial H ↔ ∃ x ∈ H, x ≠ (1 : G) := by rw [Subtype.nontrivial_iff_exists_ne (fun x => x ∈ H) (1 : H)] simp @[to_additive] theorem exists_ne_one_of_nontrivial (H : Subgroup G) [Nontrivial H] : ∃ x ∈ H, x ≠ 1 := by rwa [← Subgroup.nontrivial_iff_exists_ne_one] @[to_additive] theorem nontrivial_iff_ne_bot (H : Subgroup G) : Nontrivial H ↔ H ≠ ⊥ := by rw [nontrivial_iff_exists_ne_one, ne_eq, eq_bot_iff_forall] simp only [ne_eq, not_forall, exists_prop] /-- A subgroup is either the trivial subgroup or nontrivial. -/ @[to_additive "A subgroup is either the trivial subgroup or nontrivial."] theorem bot_or_nontrivial (H : Subgroup G) : H = ⊥ ∨ Nontrivial H := by have := nontrivial_iff_ne_bot H tauto /-- A subgroup is either the trivial subgroup or contains a non-identity element. -/ @[to_additive "A subgroup is either the trivial subgroup or contains a nonzero element."] theorem bot_or_exists_ne_one (H : Subgroup G) : H = ⊥ ∨ ∃ x ∈ H, x ≠ (1 : G) := by convert H.bot_or_nontrivial rw [nontrivial_iff_exists_ne_one] @[to_additive] lemma ne_bot_iff_exists_ne_one {H : Subgroup G} : H ≠ ⊥ ↔ ∃ a : ↥H, a ≠ 1 := by rw [← nontrivial_iff_ne_bot, nontrivial_iff_exists_ne_one] simp only [ne_eq, Subtype.exists, mk_eq_one, exists_prop] /-- The inf of two subgroups is their intersection. -/ @[to_additive "The inf of two `AddSubgroup`s is their intersection."] instance : Inf (Subgroup G) := ⟨fun H₁ H₂ => { H₁.toSubmonoid ⊓ H₂.toSubmonoid with inv_mem' := fun ⟨hx, hx'⟩ => ⟨H₁.inv_mem hx, H₂.inv_mem hx'⟩ }⟩ @[to_additive (attr := simp)] theorem coe_inf (p p' : Subgroup G) : ((p ⊓ p' : Subgroup G) : Set G) = (p : Set G) ∩ p' := rfl @[to_additive (attr := simp)] theorem mem_inf {p p' : Subgroup G} {x : G} : x ∈ p ⊓ p' ↔ x ∈ p ∧ x ∈ p' := Iff.rfl @[to_additive] instance : InfSet (Subgroup G) := ⟨fun s => { (⨅ S ∈ s, Subgroup.toSubmonoid S).copy (⋂ S ∈ s, ↑S) (by simp) with inv_mem' := fun {x} hx => Set.mem_biInter fun i h => i.inv_mem (by apply Set.mem_iInter₂.1 hx i h) }⟩ @[to_additive (attr := simp, norm_cast)] theorem coe_sInf (H : Set (Subgroup G)) : ((sInf H : Subgroup G) : Set G) = ⋂ s ∈ H, ↑s := rfl @[to_additive (attr := simp)] theorem mem_sInf {S : Set (Subgroup G)} {x : G} : x ∈ sInf S ↔ ∀ p ∈ S, x ∈ p := Set.mem_iInter₂ @[to_additive] theorem mem_iInf {ι : Sort*} {S : ι → Subgroup G} {x : G} : (x ∈ ⨅ i, S i) ↔ ∀ i, x ∈ S i := by simp only [iInf, mem_sInf, Set.forall_mem_range] @[to_additive (attr := simp, norm_cast)] theorem coe_iInf {ι : Sort*} {S : ι → Subgroup G} : (↑(⨅ i, S i) : Set G) = ⋂ i, S i := by simp only [iInf, coe_sInf, Set.biInter_range] /-- Subgroups of a group form a complete lattice. -/ @[to_additive "The `AddSubgroup`s of an `AddGroup` form a complete lattice."] instance : CompleteLattice (Subgroup G) := { completeLatticeOfInf (Subgroup G) fun _s => IsGLB.of_image SetLike.coe_subset_coe isGLB_biInf with bot := ⊥ bot_le := fun S _x hx => (mem_bot.1 hx).symm ▸ S.one_mem top := ⊤ le_top := fun _S x _hx => mem_top x inf := (· ⊓ ·) le_inf := fun _a _b _c ha hb _x hx => ⟨ha hx, hb hx⟩ inf_le_left := fun _a _b _x => And.left inf_le_right := fun _a _b _x => And.right } @[to_additive] theorem mem_sup_left {S T : Subgroup G} : ∀ {x : G}, x ∈ S → x ∈ S ⊔ T := have : S ≤ S ⊔ T := le_sup_left; fun h ↦ this h @[to_additive] theorem mem_sup_right {S T : Subgroup G} : ∀ {x : G}, x ∈ T → x ∈ S ⊔ T := have : T ≤ S ⊔ T := le_sup_right; fun h ↦ this h @[to_additive] theorem mul_mem_sup {S T : Subgroup G} {x y : G} (hx : x ∈ S) (hy : y ∈ T) : x * y ∈ S ⊔ T := (S ⊔ T).mul_mem (mem_sup_left hx) (mem_sup_right hy) @[to_additive] theorem mem_iSup_of_mem {ι : Sort*} {S : ι → Subgroup G} (i : ι) : ∀ {x : G}, x ∈ S i → x ∈ iSup S := have : S i ≤ iSup S := le_iSup _ _; fun h ↦ this h @[to_additive] theorem mem_sSup_of_mem {S : Set (Subgroup G)} {s : Subgroup G} (hs : s ∈ S) : ∀ {x : G}, x ∈ s → x ∈ sSup S := have : s ≤ sSup S := le_sSup hs; fun h ↦ this h @[to_additive (attr := simp)] theorem subsingleton_iff : Subsingleton (Subgroup G) ↔ Subsingleton G := ⟨fun h => ⟨fun x y => have : ∀ i : G, i = 1 := fun i => mem_bot.mp <| Subsingleton.elim (⊤ : Subgroup G) ⊥ ▸ mem_top i (this x).trans (this y).symm⟩, fun h => ⟨fun x y => Subgroup.ext fun i => Subsingleton.elim 1 i ▸ by simp [Subgroup.one_mem]⟩⟩ @[to_additive (attr := simp)] theorem nontrivial_iff : Nontrivial (Subgroup G) ↔ Nontrivial G := not_iff_not.mp ((not_nontrivial_iff_subsingleton.trans subsingleton_iff).trans not_nontrivial_iff_subsingleton.symm) @[to_additive] instance [Subsingleton G] : Unique (Subgroup G) := ⟨⟨⊥⟩, fun a => @Subsingleton.elim _ (subsingleton_iff.mpr ‹_›) a _⟩ @[to_additive] instance [Nontrivial G] : Nontrivial (Subgroup G) := nontrivial_iff.mpr ‹_› @[to_additive] theorem eq_top_iff' : H = ⊤ ↔ ∀ x : G, x ∈ H := eq_top_iff.trans ⟨fun h m => h <| mem_top m, fun h m _ => h m⟩ /-- The `Subgroup` generated by a set. -/ @[to_additive "The `AddSubgroup` generated by a set"] def closure (k : Set G) : Subgroup G := sInf { K | k ⊆ K } variable {k : Set G} @[to_additive] theorem mem_closure {x : G} : x ∈ closure k ↔ ∀ K : Subgroup G, k ⊆ K → x ∈ K := mem_sInf /-- The subgroup generated by a set includes the set. -/ @[to_additive (attr := simp, aesop safe 20 apply (rule_sets := [SetLike])) "The `AddSubgroup` generated by a set includes the set."] theorem subset_closure : k ⊆ closure k := fun _ hx => mem_closure.2 fun _ hK => hK hx @[to_additive] theorem not_mem_of_not_mem_closure {P : G} (hP : P ∉ closure k) : P ∉ k := fun h => hP (subset_closure h) open Set /-- A subgroup `K` includes `closure k` if and only if it includes `k`. -/ @[to_additive (attr := simp) "An additive subgroup `K` includes `closure k` if and only if it includes `k`"] theorem closure_le : closure k ≤ K ↔ k ⊆ K := ⟨Subset.trans subset_closure, fun h => sInf_le h⟩ @[to_additive] theorem closure_eq_of_le (h₁ : k ⊆ K) (h₂ : K ≤ closure k) : closure k = K := le_antisymm ((closure_le <| K).2 h₁) h₂ /-- An induction principle for closure membership. If `p` holds for `1` and all elements of `k`, and is preserved under multiplication and inverse, then `p` holds for all elements of the closure of `k`. -/ @[to_additive (attr := elab_as_elim) "An induction principle for additive closure membership. If `p` holds for `0` and all elements of `k`, and is preserved under addition and inverses, then `p` holds for all elements of the additive closure of `k`."] theorem closure_induction {p : G → Prop} {x} (h : x ∈ closure k) (mem : ∀ x ∈ k, p x) (one : p 1) (mul : ∀ x y, p x → p y → p (x * y)) (inv : ∀ x, p x → p x⁻¹) : p x := (@closure_le _ _ ⟨⟨⟨setOf p, fun {x y} ↦ mul x y⟩, one⟩, fun {x} ↦ inv x⟩ k).2 mem h /-- A dependent version of `Subgroup.closure_induction`. -/ @[to_additive (attr := elab_as_elim) "A dependent version of `AddSubgroup.closure_induction`. "] theorem closure_induction' {p : ∀ x, x ∈ closure k → Prop} (mem : ∀ (x) (h : x ∈ k), p x (subset_closure h)) (one : p 1 (one_mem _)) (mul : ∀ x hx y hy, p x hx → p y hy → p (x * y) (mul_mem hx hy)) (inv : ∀ x hx, p x hx → p x⁻¹ (inv_mem hx)) {x} (hx : x ∈ closure k) : p x hx := by refine Exists.elim ?_ fun (hx : x ∈ closure k) (hc : p x hx) => hc exact closure_induction hx (fun x hx => ⟨_, mem x hx⟩) ⟨_, one⟩ (fun x y ⟨hx', hx⟩ ⟨hy', hy⟩ => ⟨_, mul _ _ _ _ hx hy⟩) fun x ⟨hx', hx⟩ => ⟨_, inv _ _ hx⟩ /-- An induction principle for closure membership for predicates with two arguments. -/ @[to_additive (attr := elab_as_elim) "An induction principle for additive closure membership, for predicates with two arguments."] theorem closure_induction₂ {p : G → G → Prop} {x} {y : G} (hx : x ∈ closure k) (hy : y ∈ closure k) (Hk : ∀ x ∈ k, ∀ y ∈ k, p x y) (H1_left : ∀ x, p 1 x) (H1_right : ∀ x, p x 1) (Hmul_left : ∀ x₁ x₂ y, p x₁ y → p x₂ y → p (x₁ * x₂) y) (Hmul_right : ∀ x y₁ y₂, p x y₁ → p x y₂ → p x (y₁ * y₂)) (Hinv_left : ∀ x y, p x y → p x⁻¹ y) (Hinv_right : ∀ x y, p x y → p x y⁻¹) : p x y := closure_induction hx (fun x xk => closure_induction hy (Hk x xk) (H1_right x) (Hmul_right x) (Hinv_right x)) (H1_left y) (fun z z' => Hmul_left z z' y) fun z => Hinv_left z y @[to_additive (attr := simp)] theorem closure_closure_coe_preimage {k : Set G} : closure (((↑) : closure k → G) ⁻¹' k) = ⊤ := eq_top_iff.2 fun x => Subtype.recOn x fun x hx _ => by refine closure_induction' (fun g hg => ?_) ?_ (fun g₁ g₂ hg₁ hg₂ => ?_) (fun g hg => ?_) hx · exact subset_closure hg · exact one_mem _ · exact mul_mem · exact inv_mem /-- If all the elements of a set `s` commute, then `closure s` is a commutative group. -/ @[to_additive "If all the elements of a set `s` commute, then `closure s` is an additive commutative group."] def closureCommGroupOfComm {k : Set G} (hcomm : ∀ x ∈ k, ∀ y ∈ k, x * y = y * x) : CommGroup (closure k) := { (closure k).toGroup with mul_comm := fun x y => by ext simp only [Subgroup.coe_mul] refine closure_induction₂ x.prop y.prop hcomm (fun x => by simp only [mul_one, one_mul]) (fun x => by simp only [mul_one, one_mul]) (fun x y z h₁ h₂ => by rw [mul_assoc, h₂, ← mul_assoc, h₁, mul_assoc]) (fun x y z h₁ h₂ => by rw [← mul_assoc, h₁, mul_assoc, h₂, ← mul_assoc]) (fun x y h => by rw [inv_mul_eq_iff_eq_mul, ← mul_assoc, h, mul_assoc, mul_inv_self, mul_one]) fun x y h => by rw [mul_inv_eq_iff_eq_mul, mul_assoc, h, ← mul_assoc, inv_mul_self, one_mul] } variable (G) /-- `closure` forms a Galois insertion with the coercion to set. -/ @[to_additive "`closure` forms a Galois insertion with the coercion to set."] protected def gi : GaloisInsertion (@closure G _) (↑) where choice s _ := closure s gc s t := @closure_le _ _ t s le_l_u _s := subset_closure choice_eq _s _h := rfl variable {G} /-- Subgroup closure of a set is monotone in its argument: if `h ⊆ k`, then `closure h ≤ closure k`. -/ @[to_additive "Additive subgroup closure of a set is monotone in its argument: if `h ⊆ k`, then `closure h ≤ closure k`"] theorem closure_mono ⦃h k : Set G⦄ (h' : h ⊆ k) : closure h ≤ closure k := (Subgroup.gi G).gc.monotone_l h' /-- Closure of a subgroup `K` equals `K`. -/ @[to_additive (attr := simp) "Additive closure of an additive subgroup `K` equals `K`"] theorem closure_eq : closure (K : Set G) = K := (Subgroup.gi G).l_u_eq K @[to_additive (attr := simp)] theorem closure_empty : closure (∅ : Set G) = ⊥ := (Subgroup.gi G).gc.l_bot @[to_additive (attr := simp)] theorem closure_univ : closure (univ : Set G) = ⊤ := @coe_top G _ ▸ closure_eq ⊤ @[to_additive] theorem closure_union (s t : Set G) : closure (s ∪ t) = closure s ⊔ closure t := (Subgroup.gi G).gc.l_sup @[to_additive] theorem sup_eq_closure (H H' : Subgroup G) : H ⊔ H' = closure ((H : Set G) ∪ (H' : Set G)) := by simp_rw [closure_union, closure_eq] @[to_additive] theorem closure_iUnion {ι} (s : ι → Set G) : closure (⋃ i, s i) = ⨆ i, closure (s i) := (Subgroup.gi G).gc.l_iSup @[to_additive (attr := simp)] theorem closure_eq_bot_iff : closure k = ⊥ ↔ k ⊆ {1} := le_bot_iff.symm.trans <| closure_le _ @[to_additive] theorem iSup_eq_closure {ι : Sort*} (p : ι → Subgroup G) : ⨆ i, p i = closure (⋃ i, (p i : Set G)) := by simp_rw [closure_iUnion, closure_eq] /-- The subgroup generated by an element of a group equals the set of integer number powers of the element. -/ @[to_additive "The `AddSubgroup` generated by an element of an `AddGroup` equals the set of natural number multiples of the element."] theorem mem_closure_singleton {x y : G} : y ∈ closure ({x} : Set G) ↔ ∃ n : ℤ, x ^ n = y := by refine ⟨fun hy => closure_induction hy ?_ ?_ ?_ ?_, fun ⟨n, hn⟩ => hn ▸ zpow_mem (subset_closure <| mem_singleton x) n⟩ · intro y hy rw [eq_of_mem_singleton hy] exact ⟨1, zpow_one x⟩ · exact ⟨0, zpow_zero x⟩ · rintro _ _ ⟨n, rfl⟩ ⟨m, rfl⟩ exact ⟨n + m, zpow_add x n m⟩ rintro _ ⟨n, rfl⟩ exact ⟨-n, zpow_neg x n⟩ @[to_additive] theorem closure_singleton_one : closure ({1} : Set G) = ⊥ := by simp [eq_bot_iff_forall, mem_closure_singleton] @[to_additive] theorem le_closure_toSubmonoid (S : Set G) : Submonoid.closure S ≤ (closure S).toSubmonoid := Submonoid.closure_le.2 subset_closure @[to_additive] theorem closure_eq_top_of_mclosure_eq_top {S : Set G} (h : Submonoid.closure S = ⊤) : closure S = ⊤ := (eq_top_iff' _).2 fun _ => le_closure_toSubmonoid _ <| h.symm ▸ trivial @[to_additive] theorem mem_iSup_of_directed {ι} [hι : Nonempty ι] {K : ι → Subgroup G} (hK : Directed (· ≤ ·) K) {x : G} : x ∈ (iSup K : Subgroup G) ↔ ∃ i, x ∈ K i := by refine ⟨?_, fun ⟨i, hi⟩ ↦ le_iSup K i hi⟩ suffices x ∈ closure (⋃ i, (K i : Set G)) → ∃ i, x ∈ K i by simpa only [closure_iUnion, closure_eq (K _)] using this refine fun hx ↦ closure_induction hx (fun _ ↦ mem_iUnion.1) ?_ ?_ ?_ · exact hι.elim fun i ↦ ⟨i, (K i).one_mem⟩ · rintro x y ⟨i, hi⟩ ⟨j, hj⟩ rcases hK i j with ⟨k, hki, hkj⟩ exact ⟨k, mul_mem (hki hi) (hkj hj)⟩ · rintro _ ⟨i, hi⟩ exact ⟨i, inv_mem hi⟩ @[to_additive] theorem coe_iSup_of_directed {ι} [Nonempty ι] {S : ι → Subgroup G} (hS : Directed (· ≤ ·) S) : ((⨆ i, S i : Subgroup G) : Set G) = ⋃ i, S i := Set.ext fun x ↦ by simp [mem_iSup_of_directed hS] @[to_additive] theorem mem_sSup_of_directedOn {K : Set (Subgroup G)} (Kne : K.Nonempty) (hK : DirectedOn (· ≤ ·) K) {x : G} : x ∈ sSup K ↔ ∃ s ∈ K, x ∈ s := by haveI : Nonempty K := Kne.to_subtype simp only [sSup_eq_iSup', mem_iSup_of_directed hK.directed_val, SetCoe.exists, Subtype.coe_mk, exists_prop] variable {N : Type*} [Group N] {P : Type*} [Group P] /-- The preimage of a subgroup along a monoid homomorphism is a subgroup. -/ @[to_additive "The preimage of an `AddSubgroup` along an `AddMonoid` homomorphism is an `AddSubgroup`."] def comap {N : Type*} [Group N] (f : G →* N) (H : Subgroup N) : Subgroup G := { H.toSubmonoid.comap f with carrier := f ⁻¹' H inv_mem' := fun {a} ha => show f a⁻¹ ∈ H by rw [f.map_inv]; exact H.inv_mem ha } @[to_additive (attr := simp)] theorem coe_comap (K : Subgroup N) (f : G →* N) : (K.comap f : Set G) = f ⁻¹' K := rfl @[simp] theorem toAddSubgroup_comap {G₂ : Type*} [Group G₂] (f : G →* G₂) (s : Subgroup G₂) : s.toAddSubgroup.comap (MonoidHom.toAdditive f) = Subgroup.toAddSubgroup (s.comap f) := rfl @[simp] theorem _root_.AddSubgroup.toSubgroup_comap {A A₂ : Type*} [AddGroup A] [AddGroup A₂] (f : A →+ A₂) (s : AddSubgroup A₂) : s.toSubgroup.comap (AddMonoidHom.toMultiplicative f) = AddSubgroup.toSubgroup (s.comap f) := rfl @[to_additive (attr := simp)] theorem mem_comap {K : Subgroup N} {f : G →* N} {x : G} : x ∈ K.comap f ↔ f x ∈ K := Iff.rfl @[to_additive] theorem comap_mono {f : G →* N} {K K' : Subgroup N} : K ≤ K' → comap f K ≤ comap f K' := preimage_mono @[to_additive] theorem comap_comap (K : Subgroup P) (g : N →* P) (f : G →* N) : (K.comap g).comap f = K.comap (g.comp f) := rfl @[to_additive (attr := simp)] theorem comap_id (K : Subgroup N) : K.comap (MonoidHom.id _) = K := by ext rfl /-- The image of a subgroup along a monoid homomorphism is a subgroup. -/ @[to_additive "The image of an `AddSubgroup` along an `AddMonoid` homomorphism is an `AddSubgroup`."] def map (f : G →* N) (H : Subgroup G) : Subgroup N := { H.toSubmonoid.map f with carrier := f '' H inv_mem' := by rintro _ ⟨x, hx, rfl⟩ exact ⟨x⁻¹, H.inv_mem hx, f.map_inv x⟩ } @[to_additive (attr := simp)] theorem coe_map (f : G →* N) (K : Subgroup G) : (K.map f : Set N) = f '' K := rfl @[to_additive (attr := simp)] theorem mem_map {f : G →* N} {K : Subgroup G} {y : N} : y ∈ K.map f ↔ ∃ x ∈ K, f x = y := Iff.rfl @[to_additive] theorem mem_map_of_mem (f : G →* N) {K : Subgroup G} {x : G} (hx : x ∈ K) : f x ∈ K.map f := mem_image_of_mem f hx @[to_additive] theorem apply_coe_mem_map (f : G →* N) (K : Subgroup G) (x : K) : f x ∈ K.map f := mem_map_of_mem f x.prop @[to_additive] theorem map_mono {f : G →* N} {K K' : Subgroup G} : K ≤ K' → map f K ≤ map f K' := image_subset _ @[to_additive (attr := simp)] theorem map_id : K.map (MonoidHom.id G) = K := SetLike.coe_injective <| image_id _ @[to_additive] theorem map_map (g : N →* P) (f : G →* N) : (K.map f).map g = K.map (g.comp f) := SetLike.coe_injective <| image_image _ _ _ @[to_additive (attr := simp)] theorem map_one_eq_bot : K.map (1 : G →* N) = ⊥ := eq_bot_iff.mpr <| by rintro x ⟨y, _, rfl⟩ simp @[to_additive] theorem mem_map_equiv {f : G ≃* N} {K : Subgroup G} {x : N} : x ∈ K.map f.toMonoidHom ↔ f.symm x ∈ K := by erw [@Set.mem_image_equiv _ _ (↑K) f.toEquiv x]; rfl -- The simpNF linter says that the LHS can be simplified via `Subgroup.mem_map`. -- However this is a higher priority lemma. -- https://github.com/leanprover/std4/issues/207 @[to_additive (attr := simp 1100, nolint simpNF)] theorem mem_map_iff_mem {f : G →* N} (hf : Function.Injective f) {K : Subgroup G} {x : G} : f x ∈ K.map f ↔ x ∈ K := hf.mem_set_image @[to_additive] theorem map_equiv_eq_comap_symm' (f : G ≃* N) (K : Subgroup G) : K.map f.toMonoidHom = K.comap f.symm.toMonoidHom := SetLike.coe_injective (f.toEquiv.image_eq_preimage K) @[to_additive] theorem map_equiv_eq_comap_symm (f : G ≃* N) (K : Subgroup G) : K.map f = K.comap (G := N) f.symm := map_equiv_eq_comap_symm' _ _ @[to_additive] theorem comap_equiv_eq_map_symm (f : N ≃* G) (K : Subgroup G) : K.comap (G := N) f = K.map f.symm := (map_equiv_eq_comap_symm f.symm K).symm @[to_additive] theorem comap_equiv_eq_map_symm' (f : N ≃* G) (K : Subgroup G) : K.comap f.toMonoidHom = K.map f.symm.toMonoidHom := (map_equiv_eq_comap_symm f.symm K).symm @[to_additive] theorem map_symm_eq_iff_map_eq {H : Subgroup N} {e : G ≃* N} : H.map ↑e.symm = K ↔ K.map ↑e = H := by constructor <;> rintro rfl · rw [map_map, ← MulEquiv.coe_monoidHom_trans, MulEquiv.symm_trans_self, MulEquiv.coe_monoidHom_refl, map_id] · rw [map_map, ← MulEquiv.coe_monoidHom_trans, MulEquiv.self_trans_symm, MulEquiv.coe_monoidHom_refl, map_id] @[to_additive] theorem map_le_iff_le_comap {f : G →* N} {K : Subgroup G} {H : Subgroup N} : K.map f ≤ H ↔ K ≤ H.comap f := image_subset_iff @[to_additive] theorem gc_map_comap (f : G →* N) : GaloisConnection (map f) (comap f) := fun _ _ => map_le_iff_le_comap @[to_additive] theorem map_sup (H K : Subgroup G) (f : G →* N) : (H ⊔ K).map f = H.map f ⊔ K.map f := (gc_map_comap f).l_sup @[to_additive] theorem map_iSup {ι : Sort*} (f : G →* N) (s : ι → Subgroup G) : (iSup s).map f = ⨆ i, (s i).map f := (gc_map_comap f).l_iSup @[to_additive] theorem comap_sup_comap_le (H K : Subgroup N) (f : G →* N) : comap f H ⊔ comap f K ≤ comap f (H ⊔ K) := Monotone.le_map_sup (fun _ _ => comap_mono) H K @[to_additive] theorem iSup_comap_le {ι : Sort*} (f : G →* N) (s : ι → Subgroup N) : ⨆ i, (s i).comap f ≤ (iSup s).comap f := Monotone.le_map_iSup fun _ _ => comap_mono @[to_additive] theorem comap_inf (H K : Subgroup N) (f : G →* N) : (H ⊓ K).comap f = H.comap f ⊓ K.comap f := (gc_map_comap f).u_inf @[to_additive] theorem comap_iInf {ι : Sort*} (f : G →* N) (s : ι → Subgroup N) : (iInf s).comap f = ⨅ i, (s i).comap f := (gc_map_comap f).u_iInf @[to_additive] theorem map_inf_le (H K : Subgroup G) (f : G →* N) : map f (H ⊓ K) ≤ map f H ⊓ map f K := le_inf (map_mono inf_le_left) (map_mono inf_le_right) @[to_additive] theorem map_inf_eq (H K : Subgroup G) (f : G →* N) (hf : Function.Injective f) : map f (H ⊓ K) = map f H ⊓ map f K := by rw [← SetLike.coe_set_eq] simp [Set.image_inter hf] @[to_additive (attr := simp)] theorem map_bot (f : G →* N) : (⊥ : Subgroup G).map f = ⊥ := (gc_map_comap f).l_bot @[to_additive (attr := simp)] theorem map_top_of_surjective (f : G →* N) (h : Function.Surjective f) : Subgroup.map f ⊤ = ⊤ := by rw [eq_top_iff] intro x _ obtain ⟨y, hy⟩ := h x exact ⟨y, trivial, hy⟩ @[to_additive (attr := simp)] theorem comap_top (f : G →* N) : (⊤ : Subgroup N).comap f = ⊤ := (gc_map_comap f).u_top /-- For any subgroups `H` and `K`, view `H ⊓ K` as a subgroup of `K`. -/ @[to_additive "For any subgroups `H` and `K`, view `H ⊓ K` as a subgroup of `K`."] def subgroupOf (H K : Subgroup G) : Subgroup K := H.comap K.subtype /-- If `H ≤ K`, then `H` as a subgroup of `K` is isomorphic to `H`. -/ @[to_additive (attr := simps) "If `H ≤ K`, then `H` as a subgroup of `K` is isomorphic to `H`."] def subgroupOfEquivOfLe {G : Type*} [Group G] {H K : Subgroup G} (h : H ≤ K) : H.subgroupOf K ≃* H where toFun g := ⟨g.1, g.2⟩ invFun g := ⟨⟨g.1, h g.2⟩, g.2⟩ left_inv _g := Subtype.ext (Subtype.ext rfl) right_inv _g := Subtype.ext rfl map_mul' _g _h := rfl @[to_additive (attr := simp)] theorem comap_subtype (H K : Subgroup G) : H.comap K.subtype = H.subgroupOf K := rfl @[to_additive (attr := simp)] theorem comap_inclusion_subgroupOf {K₁ K₂ : Subgroup G} (h : K₁ ≤ K₂) (H : Subgroup G) : (H.subgroupOf K₂).comap (inclusion h) = H.subgroupOf K₁ := rfl @[to_additive] theorem coe_subgroupOf (H K : Subgroup G) : (H.subgroupOf K : Set K) = K.subtype ⁻¹' H := rfl @[to_additive] theorem mem_subgroupOf {H K : Subgroup G} {h : K} : h ∈ H.subgroupOf K ↔ (h : G) ∈ H := Iff.rfl -- TODO(kmill): use `K ⊓ H` order for RHS to match `Subtype.image_preimage_coe` @[to_additive (attr := simp)] theorem subgroupOf_map_subtype (H K : Subgroup G) : (H.subgroupOf K).map K.subtype = H ⊓ K := SetLike.ext' <| by refine Subtype.image_preimage_coe _ _ |>.trans ?_; apply Set.inter_comm @[to_additive (attr := simp)] theorem bot_subgroupOf : (⊥ : Subgroup G).subgroupOf H = ⊥ := Eq.symm (Subgroup.ext fun _g => Subtype.ext_iff) @[to_additive (attr := simp)] theorem top_subgroupOf : (⊤ : Subgroup G).subgroupOf H = ⊤ := rfl @[to_additive] theorem subgroupOf_bot_eq_bot : H.subgroupOf ⊥ = ⊥ := Subsingleton.elim _ _ @[to_additive] theorem subgroupOf_bot_eq_top : H.subgroupOf ⊥ = ⊤ := Subsingleton.elim _ _ @[to_additive (attr := simp)] theorem subgroupOf_self : H.subgroupOf H = ⊤ := top_unique fun g _hg => g.2 @[to_additive (attr := simp)] theorem subgroupOf_inj {H₁ H₂ K : Subgroup G} : H₁.subgroupOf K = H₂.subgroupOf K ↔ H₁ ⊓ K = H₂ ⊓ K := by simpa only [SetLike.ext_iff, mem_inf, mem_subgroupOf, and_congr_left_iff] using Subtype.forall @[to_additive (attr := simp)] theorem inf_subgroupOf_right (H K : Subgroup G) : (H ⊓ K).subgroupOf K = H.subgroupOf K := subgroupOf_inj.2 (inf_right_idem _ _) @[to_additive (attr := simp)] theorem inf_subgroupOf_left (H K : Subgroup G) : (K ⊓ H).subgroupOf K = H.subgroupOf K := by rw [inf_comm, inf_subgroupOf_right] @[to_additive (attr := simp)] theorem subgroupOf_eq_bot {H K : Subgroup G} : H.subgroupOf K = ⊥ ↔ Disjoint H K := by rw [disjoint_iff, ← bot_subgroupOf, subgroupOf_inj, bot_inf_eq] @[to_additive (attr := simp)] theorem subgroupOf_eq_top {H K : Subgroup G} : H.subgroupOf K = ⊤ ↔ K ≤ H := by rw [← top_subgroupOf, subgroupOf_inj, top_inf_eq, inf_eq_right] /-- Given `Subgroup`s `H`, `K` of groups `G`, `N` respectively, `H × K` as a subgroup of `G × N`. -/ @[to_additive prod "Given `AddSubgroup`s `H`, `K` of `AddGroup`s `A`, `B` respectively, `H × K` as an `AddSubgroup` of `A × B`."] def prod (H : Subgroup G) (K : Subgroup N) : Subgroup (G × N) := { Submonoid.prod H.toSubmonoid K.toSubmonoid with inv_mem' := fun hx => ⟨H.inv_mem' hx.1, K.inv_mem' hx.2⟩ } @[to_additive coe_prod] theorem coe_prod (H : Subgroup G) (K : Subgroup N) : (H.prod K : Set (G × N)) = (H : Set G) ×ˢ (K : Set N) := rfl @[to_additive mem_prod] theorem mem_prod {H : Subgroup G} {K : Subgroup N} {p : G × N} : p ∈ H.prod K ↔ p.1 ∈ H ∧ p.2 ∈ K := Iff.rfl @[to_additive prod_mono] theorem prod_mono : ((· ≤ ·) ⇒ (· ≤ ·) ⇒ (· ≤ ·)) (@prod G _ N _) (@prod G _ N _) := fun _s _s' hs _t _t' ht => Set.prod_mono hs ht @[to_additive prod_mono_right] theorem prod_mono_right (K : Subgroup G) : Monotone fun t : Subgroup N => K.prod t := prod_mono (le_refl K) @[to_additive prod_mono_left] theorem prod_mono_left (H : Subgroup N) : Monotone fun K : Subgroup G => K.prod H := fun _ _ hs => prod_mono hs (le_refl H) @[to_additive prod_top] theorem prod_top (K : Subgroup G) : K.prod (⊤ : Subgroup N) = K.comap (MonoidHom.fst G N) := ext fun x => by simp [mem_prod, MonoidHom.coe_fst] @[to_additive top_prod] theorem top_prod (H : Subgroup N) : (⊤ : Subgroup G).prod H = H.comap (MonoidHom.snd G N) := ext fun x => by simp [mem_prod, MonoidHom.coe_snd] @[to_additive (attr := simp) top_prod_top] theorem top_prod_top : (⊤ : Subgroup G).prod (⊤ : Subgroup N) = ⊤ := (top_prod _).trans <| comap_top _ @[to_additive] theorem bot_prod_bot : (⊥ : Subgroup G).prod (⊥ : Subgroup N) = ⊥ := SetLike.coe_injective <| by simp [coe_prod, Prod.one_eq_mk] @[to_additive le_prod_iff] theorem le_prod_iff {H : Subgroup G} {K : Subgroup N} {J : Subgroup (G × N)} : J ≤ H.prod K ↔ map (MonoidHom.fst G N) J ≤ H ∧ map (MonoidHom.snd G N) J ≤ K := by simpa only [← Subgroup.toSubmonoid_le] using Submonoid.le_prod_iff @[to_additive prod_le_iff] theorem prod_le_iff {H : Subgroup G} {K : Subgroup N} {J : Subgroup (G × N)} : H.prod K ≤ J ↔ map (MonoidHom.inl G N) H ≤ J ∧ map (MonoidHom.inr G N) K ≤ J := by simpa only [← Subgroup.toSubmonoid_le] using Submonoid.prod_le_iff @[to_additive (attr := simp) prod_eq_bot_iff] theorem prod_eq_bot_iff {H : Subgroup G} {K : Subgroup N} : H.prod K = ⊥ ↔ H = ⊥ ∧ K = ⊥ := by simpa only [← Subgroup.toSubmonoid_eq] using Submonoid.prod_eq_bot_iff /-- Product of subgroups is isomorphic to their product as groups. -/ @[to_additive prodEquiv "Product of additive subgroups is isomorphic to their product as additive groups"] def prodEquiv (H : Subgroup G) (K : Subgroup N) : H.prod K ≃* H × K := { Equiv.Set.prod (H : Set G) (K : Set N) with map_mul' := fun _ _ => rfl } section Pi variable {η : Type*} {f : η → Type*} -- defined here and not in Algebra.Group.Submonoid.Operations to have access to Algebra.Group.Pi /-- A version of `Set.pi` for submonoids. Given an index set `I` and a family of submodules `s : Π i, Submonoid f i`, `pi I s` is the submonoid of dependent functions `f : Π i, f i` such that `f i` belongs to `Pi I s` whenever `i ∈ I`. -/ @[to_additive "A version of `Set.pi` for `AddSubmonoid`s. Given an index set `I` and a family of submodules `s : Π i, AddSubmonoid f i`, `pi I s` is the `AddSubmonoid` of dependent functions `f : Π i, f i` such that `f i` belongs to `pi I s` whenever `i ∈ I`."] def _root_.Submonoid.pi [∀ i, MulOneClass (f i)] (I : Set η) (s : ∀ i, Submonoid (f i)) : Submonoid (∀ i, f i) where carrier := I.pi fun i => (s i).carrier one_mem' i _ := (s i).one_mem mul_mem' hp hq i hI := (s i).mul_mem (hp i hI) (hq i hI) variable [∀ i, Group (f i)] /-- A version of `Set.pi` for subgroups. Given an index set `I` and a family of submodules `s : Π i, Subgroup f i`, `pi I s` is the subgroup of dependent functions `f : Π i, f i` such that `f i` belongs to `pi I s` whenever `i ∈ I`. -/ @[to_additive "A version of `Set.pi` for `AddSubgroup`s. Given an index set `I` and a family of submodules `s : Π i, AddSubgroup f i`, `pi I s` is the `AddSubgroup` of dependent functions `f : Π i, f i` such that `f i` belongs to `pi I s` whenever `i ∈ I`."] def pi (I : Set η) (H : ∀ i, Subgroup (f i)) : Subgroup (∀ i, f i) := { Submonoid.pi I fun i => (H i).toSubmonoid with inv_mem' := fun hp i hI => (H i).inv_mem (hp i hI) } @[to_additive] theorem coe_pi (I : Set η) (H : ∀ i, Subgroup (f i)) : (pi I H : Set (∀ i, f i)) = Set.pi I fun i => (H i : Set (f i)) := rfl @[to_additive] theorem mem_pi (I : Set η) {H : ∀ i, Subgroup (f i)} {p : ∀ i, f i} : p ∈ pi I H ↔ ∀ i : η, i ∈ I → p i ∈ H i := Iff.rfl @[to_additive] theorem pi_top (I : Set η) : (pi I fun i => (⊤ : Subgroup (f i))) = ⊤ := ext fun x => by simp [mem_pi] @[to_additive] theorem pi_empty (H : ∀ i, Subgroup (f i)) : pi ∅ H = ⊤ := ext fun x => by simp [mem_pi] @[to_additive] theorem pi_bot : (pi Set.univ fun i => (⊥ : Subgroup (f i))) = ⊥ := (eq_bot_iff_forall _).mpr fun p hp => by simp only [mem_pi, mem_bot] at * ext j exact hp j trivial @[to_additive] theorem le_pi_iff {I : Set η} {H : ∀ i, Subgroup (f i)} {J : Subgroup (∀ i, f i)} : J ≤ pi I H ↔ ∀ i : η, i ∈ I → map (Pi.evalMonoidHom f i) J ≤ H i := by constructor · intro h i hi rintro _ ⟨x, hx, rfl⟩ exact (h hx) _ hi · intro h x hx i hi exact h i hi ⟨_, hx, rfl⟩ @[to_additive (attr := simp)] theorem mulSingle_mem_pi [DecidableEq η] {I : Set η} {H : ∀ i, Subgroup (f i)} (i : η) (x : f i) : Pi.mulSingle i x ∈ pi I H ↔ i ∈ I → x ∈ H i := by constructor · intro h hi simpa using h i hi · intro h j hj by_cases heq : j = i · subst heq simpa using h hj · simp [heq, one_mem] @[to_additive] theorem pi_eq_bot_iff (H : ∀ i, Subgroup (f i)) : pi Set.univ H = ⊥ ↔ ∀ i, H i = ⊥ := by classical simp only [eq_bot_iff_forall] constructor · intro h i x hx have : MonoidHom.mulSingle f i x = 1 := h (MonoidHom.mulSingle f i x) ((mulSingle_mem_pi i x).mpr fun _ => hx) simpa using congr_fun this i · exact fun h x hx => funext fun i => h _ _ (hx i trivial) end Pi /-- A subgroup is normal if whenever `n ∈ H`, then `g * n * g⁻¹ ∈ H` for every `g : G` -/ structure Normal : Prop where /-- `N` is closed under conjugation -/ conj_mem : ∀ n, n ∈ H → ∀ g : G, g * n * g⁻¹ ∈ H attribute [class] Normal end Subgroup namespace AddSubgroup /-- An AddSubgroup is normal if whenever `n ∈ H`, then `g + n - g ∈ H` for every `g : G` -/ structure Normal (H : AddSubgroup A) : Prop where /-- `N` is closed under additive conjugation -/ conj_mem : ∀ n, n ∈ H → ∀ g : A, g + n + -g ∈ H attribute [to_additive] Subgroup.Normal attribute [class] Normal end AddSubgroup namespace Subgroup variable {H K : Subgroup G} @[to_additive] instance (priority := 100) normal_of_comm {G : Type*} [CommGroup G] (H : Subgroup G) : H.Normal := ⟨by simp [mul_comm, mul_left_comm]⟩ namespace Normal @[to_additive] theorem conj_mem' (nH : H.Normal) (n : G) (hn : n ∈ H) (g : G) : g⁻¹ * n * g ∈ H := by convert nH.conj_mem n hn g⁻¹ rw [inv_inv] @[to_additive] theorem mem_comm (nH : H.Normal) {a b : G} (h : a * b ∈ H) : b * a ∈ H := by have : a⁻¹ * (a * b) * a⁻¹⁻¹ ∈ H := nH.conj_mem (a * b) h a⁻¹ -- Porting note: Previous code was: -- simpa simp_all only [inv_mul_cancel_left, inv_inv] @[to_additive] theorem mem_comm_iff (nH : H.Normal) {a b : G} : a * b ∈ H ↔ b * a ∈ H := ⟨nH.mem_comm, nH.mem_comm⟩ end Normal variable (H) /-- A subgroup is characteristic if it is fixed by all automorphisms. Several equivalent conditions are provided by lemmas of the form `Characteristic.iff...` -/ structure Characteristic : Prop where /-- `H` is fixed by all automorphisms -/ fixed : ∀ ϕ : G ≃* G, H.comap ϕ.toMonoidHom = H attribute [class] Characteristic instance (priority := 100) normal_of_characteristic [h : H.Characteristic] : H.Normal := ⟨fun a ha b => (SetLike.ext_iff.mp (h.fixed (MulAut.conj b)) a).mpr ha⟩ end Subgroup namespace AddSubgroup variable (H : AddSubgroup A) /-- An `AddSubgroup` is characteristic if it is fixed by all automorphisms. Several equivalent conditions are provided by lemmas of the form `Characteristic.iff...` -/ structure Characteristic : Prop where /-- `H` is fixed by all automorphisms -/ fixed : ∀ ϕ : A ≃+ A, H.comap ϕ.toAddMonoidHom = H attribute [to_additive] Subgroup.Characteristic attribute [class] Characteristic instance (priority := 100) normal_of_characteristic [h : H.Characteristic] : H.Normal := ⟨fun a ha b => (SetLike.ext_iff.mp (h.fixed (AddAut.conj b)) a).mpr ha⟩ end AddSubgroup namespace Subgroup variable {H K : Subgroup G} @[to_additive] theorem characteristic_iff_comap_eq : H.Characteristic ↔ ∀ ϕ : G ≃* G, H.comap ϕ.toMonoidHom = H := ⟨Characteristic.fixed, Characteristic.mk⟩ @[to_additive] theorem characteristic_iff_comap_le : H.Characteristic ↔ ∀ ϕ : G ≃* G, H.comap ϕ.toMonoidHom ≤ H := characteristic_iff_comap_eq.trans ⟨fun h ϕ => le_of_eq (h ϕ), fun h ϕ => le_antisymm (h ϕ) fun g hg => h ϕ.symm ((congr_arg (· ∈ H) (ϕ.symm_apply_apply g)).mpr hg)⟩ @[to_additive] theorem characteristic_iff_le_comap : H.Characteristic ↔ ∀ ϕ : G ≃* G, H ≤ H.comap ϕ.toMonoidHom := characteristic_iff_comap_eq.trans ⟨fun h ϕ => ge_of_eq (h ϕ), fun h ϕ => le_antisymm (fun g hg => (congr_arg (· ∈ H) (ϕ.symm_apply_apply g)).mp (h ϕ.symm hg)) (h ϕ)⟩ @[to_additive] theorem characteristic_iff_map_eq : H.Characteristic ↔ ∀ ϕ : G ≃* G, H.map ϕ.toMonoidHom = H := by simp_rw [map_equiv_eq_comap_symm'] exact characteristic_iff_comap_eq.trans ⟨fun h ϕ => h ϕ.symm, fun h ϕ => h ϕ.symm⟩ @[to_additive] theorem characteristic_iff_map_le : H.Characteristic ↔ ∀ ϕ : G ≃* G, H.map ϕ.toMonoidHom ≤ H := by simp_rw [map_equiv_eq_comap_symm'] exact characteristic_iff_comap_le.trans ⟨fun h ϕ => h ϕ.symm, fun h ϕ => h ϕ.symm⟩ @[to_additive] theorem characteristic_iff_le_map : H.Characteristic ↔ ∀ ϕ : G ≃* G, H ≤ H.map ϕ.toMonoidHom := by simp_rw [map_equiv_eq_comap_symm'] exact characteristic_iff_le_comap.trans ⟨fun h ϕ => h ϕ.symm, fun h ϕ => h ϕ.symm⟩ @[to_additive] instance botCharacteristic : Characteristic (⊥ : Subgroup G) := characteristic_iff_le_map.mpr fun _ϕ => bot_le @[to_additive] instance topCharacteristic : Characteristic (⊤ : Subgroup G) := characteristic_iff_map_le.mpr fun _ϕ => le_top variable (H) section Normalizer /-- The `normalizer` of `H` is the largest subgroup of `G` inside which `H` is normal. -/ @[to_additive "The `normalizer` of `H` is the largest subgroup of `G` inside which `H` is normal."] def normalizer : Subgroup G where carrier := { g : G | ∀ n, n ∈ H ↔ g * n * g⁻¹ ∈ H } one_mem' := by simp mul_mem' {a b} (ha : ∀ n, n ∈ H ↔ a * n * a⁻¹ ∈ H) (hb : ∀ n, n ∈ H ↔ b * n * b⁻¹ ∈ H) n := by rw [hb, ha] simp only [mul_assoc, mul_inv_rev] inv_mem' {a} (ha : ∀ n, n ∈ H ↔ a * n * a⁻¹ ∈ H) n := by rw [ha (a⁻¹ * n * a⁻¹⁻¹)] simp only [inv_inv, mul_assoc, mul_inv_cancel_left, mul_right_inv, mul_one] -- variant for sets. -- TODO should this replace `normalizer`? /-- The `setNormalizer` of `S` is the subgroup of `G` whose elements satisfy `g*S*g⁻¹=S` -/ @[to_additive "The `setNormalizer` of `S` is the subgroup of `G` whose elements satisfy `g+S-g=S`."] def setNormalizer (S : Set G) : Subgroup G where carrier := { g : G | ∀ n, n ∈ S ↔ g * n * g⁻¹ ∈ S } one_mem' := by simp mul_mem' {a b} (ha : ∀ n, n ∈ S ↔ a * n * a⁻¹ ∈ S) (hb : ∀ n, n ∈ S ↔ b * n * b⁻¹ ∈ S) n := by rw [hb, ha] simp only [mul_assoc, mul_inv_rev] inv_mem' {a} (ha : ∀ n, n ∈ S ↔ a * n * a⁻¹ ∈ S) n := by rw [ha (a⁻¹ * n * a⁻¹⁻¹)] simp only [inv_inv, mul_assoc, mul_inv_cancel_left, mul_right_inv, mul_one] variable {H} @[to_additive] theorem mem_normalizer_iff {g : G} : g ∈ H.normalizer ↔ ∀ h, h ∈ H ↔ g * h * g⁻¹ ∈ H := Iff.rfl @[to_additive] theorem mem_normalizer_iff'' {g : G} : g ∈ H.normalizer ↔ ∀ h : G, h ∈ H ↔ g⁻¹ * h * g ∈ H := by rw [← inv_mem_iff (x := g), mem_normalizer_iff, inv_inv] @[to_additive] theorem mem_normalizer_iff' {g : G} : g ∈ H.normalizer ↔ ∀ n, n * g ∈ H ↔ g * n ∈ H := ⟨fun h n => by rw [h, mul_assoc, mul_inv_cancel_right], fun h n => by rw [mul_assoc, ← h, inv_mul_cancel_right]⟩ @[to_additive] theorem le_normalizer : H ≤ normalizer H := fun x xH n => by rw [H.mul_mem_cancel_right (H.inv_mem xH), H.mul_mem_cancel_left xH] @[to_additive] instance (priority := 100) normal_in_normalizer : (H.subgroupOf H.normalizer).Normal := ⟨fun x xH g => by simpa only [mem_subgroupOf] using (g.2 x.1).1 xH⟩ @[to_additive] theorem normalizer_eq_top : H.normalizer = ⊤ ↔ H.Normal := eq_top_iff.trans ⟨fun h => ⟨fun a ha b => (h (mem_top b) a).mp ha⟩, fun h a _ha b => ⟨fun hb => h.conj_mem b hb a, fun hb => by rwa [h.mem_comm_iff, inv_mul_cancel_left] at hb⟩⟩ @[to_additive] theorem le_normalizer_of_normal [hK : (H.subgroupOf K).Normal] (HK : H ≤ K) : K ≤ H.normalizer := fun x hx y => ⟨fun yH => hK.conj_mem ⟨y, HK yH⟩ yH ⟨x, hx⟩, fun yH => by simpa [mem_subgroupOf, mul_assoc] using hK.conj_mem ⟨x * y * x⁻¹, HK yH⟩ yH ⟨x⁻¹, K.inv_mem hx⟩⟩ variable {N : Type*} [Group N] /-- The preimage of the normalizer is contained in the normalizer of the preimage. -/ @[to_additive "The preimage of the normalizer is contained in the normalizer of the preimage."] theorem le_normalizer_comap (f : N →* G) : H.normalizer.comap f ≤ (H.comap f).normalizer := fun x => by simp only [mem_normalizer_iff, mem_comap] intro h n simp [h (f n)] /-- The image of the normalizer is contained in the normalizer of the image. -/ @[to_additive "The image of the normalizer is contained in the normalizer of the image."] theorem le_normalizer_map (f : G →* N) : H.normalizer.map f ≤ (H.map f).normalizer := fun _ => by simp only [and_imp, exists_prop, mem_map, exists_imp, mem_normalizer_iff] rintro x hx rfl n constructor · rintro ⟨y, hy, rfl⟩ use x * y * x⁻¹, (hx y).1 hy simp · rintro ⟨y, hyH, hy⟩ use x⁻¹ * y * x rw [hx] simp [hy, hyH, mul_assoc] variable (G) /-- Every proper subgroup `H` of `G` is a proper normal subgroup of the normalizer of `H` in `G`. -/ def _root_.NormalizerCondition := ∀ H : Subgroup G, H < ⊤ → H < normalizer H variable {G} /-- Alternative phrasing of the normalizer condition: Only the full group is self-normalizing. This may be easier to work with, as it avoids inequalities and negations. -/ theorem _root_.normalizerCondition_iff_only_full_group_self_normalizing : NormalizerCondition G ↔ ∀ H : Subgroup G, H.normalizer = H → H = ⊤ := by apply forall_congr'; intro H simp only [lt_iff_le_and_ne, le_normalizer, true_and_iff, le_top, Ne] tauto variable (H) end Normalizer /-- Commutativity of a subgroup -/ structure IsCommutative : Prop where /-- `*` is commutative on `H` -/ is_comm : Std.Commutative (α := H) (· * ·) attribute [class] IsCommutative /-- Commutativity of an additive subgroup -/ structure _root_.AddSubgroup.IsCommutative (H : AddSubgroup A) : Prop where /-- `+` is commutative on `H` -/ is_comm : Std.Commutative (α := H) (· + ·) attribute [to_additive] Subgroup.IsCommutative attribute [class] AddSubgroup.IsCommutative /-- A commutative subgroup is commutative. -/ @[to_additive "A commutative subgroup is commutative."] instance IsCommutative.commGroup [h : H.IsCommutative] : CommGroup H := { H.toGroup with mul_comm := h.is_comm.comm } /-- A subgroup of a commutative group is commutative. -/ @[to_additive "A subgroup of a commutative group is commutative."] instance commGroup_isCommutative {G : Type*} [CommGroup G] (H : Subgroup G) : H.IsCommutative := ⟨CommMagma.to_isCommutative⟩ @[to_additive] instance map_isCommutative (f : G →* G') [H.IsCommutative] : (H.map f).IsCommutative := ⟨⟨by rintro ⟨-, a, ha, rfl⟩ ⟨-, b, hb, rfl⟩ rw [Subtype.ext_iff, coe_mul, coe_mul, Subtype.coe_mk, Subtype.coe_mk, ← map_mul, ← map_mul] exact congr_arg f (Subtype.ext_iff.mp (mul_comm (⟨a, ha⟩ : H) ⟨b, hb⟩))⟩⟩ @[to_additive] theorem comap_injective_isCommutative {f : G' →* G} (hf : Injective f) [H.IsCommutative] : (H.comap f).IsCommutative := ⟨⟨fun a b => Subtype.ext (by have := mul_comm (⟨f a, a.2⟩ : H) (⟨f b, b.2⟩ : H) rwa [Subtype.ext_iff, coe_mul, coe_mul, coe_mk, coe_mk, ← map_mul, ← map_mul, hf.eq_iff] at this)⟩⟩ @[to_additive] instance subgroupOf_isCommutative [H.IsCommutative] : (H.subgroupOf K).IsCommutative := H.comap_injective_isCommutative Subtype.coe_injective @[to_additive] lemma mul_comm_of_mem_isCommutative [H.IsCommutative] {a b : G} (ha : a ∈ H) (hb : b ∈ H) : a * b = b * a := by simpa only [Submonoid.mk_mul_mk, Subtype.mk.injEq] using mul_comm (⟨a, ha⟩ : H) (⟨b, hb⟩ : H) end Subgroup namespace MulEquiv variable {H : Type*} [Group H] /-- An isomorphism of groups gives an order isomorphism between the lattices of subgroups, defined by sending subgroups to their inverse images. See also `MulEquiv.mapSubgroup` which maps subgroups to their forward images. -/ @[simps] def comapSubgroup (f : G ≃* H) : Subgroup H ≃o Subgroup G where toFun := Subgroup.comap f invFun := Subgroup.comap f.symm left_inv sg := by simp [Subgroup.comap_comap] right_inv sh := by simp [Subgroup.comap_comap] map_rel_iff' {sg1 sg2} := ⟨fun h => by simpa [Subgroup.comap_comap] using Subgroup.comap_mono (f := (f.symm : H →* G)) h, Subgroup.comap_mono⟩ /-- An isomorphism of groups gives an order isomorphism between the lattices of subgroups, defined by sending subgroups to their forward images. See also `MulEquiv.comapSubgroup` which maps subgroups to their inverse images. -/ @[simps] def mapSubgroup {H : Type*} [Group H] (f : G ≃* H) : Subgroup G ≃o Subgroup H where toFun := Subgroup.map f invFun := Subgroup.map f.symm left_inv sg := by simp [Subgroup.map_map] right_inv sh := by simp [Subgroup.map_map] map_rel_iff' {sg1 sg2} := ⟨fun h => by simpa [Subgroup.map_map] using Subgroup.map_mono (f := (f.symm : H →* G)) h, Subgroup.map_mono⟩ end MulEquiv namespace Group variable {s : Set G} /-- Given a set `s`, `conjugatesOfSet s` is the set of all conjugates of the elements of `s`. -/ def conjugatesOfSet (s : Set G) : Set G := ⋃ a ∈ s, conjugatesOf a theorem mem_conjugatesOfSet_iff {x : G} : x ∈ conjugatesOfSet s ↔ ∃ a ∈ s, IsConj a x := by erw [Set.mem_iUnion₂]; simp only [conjugatesOf, isConj_iff, Set.mem_setOf_eq, exists_prop] theorem subset_conjugatesOfSet : s ⊆ conjugatesOfSet s := fun (x : G) (h : x ∈ s) => mem_conjugatesOfSet_iff.2 ⟨x, h, IsConj.refl _⟩ theorem conjugatesOfSet_mono {s t : Set G} (h : s ⊆ t) : conjugatesOfSet s ⊆ conjugatesOfSet t := Set.biUnion_subset_biUnion_left h theorem conjugates_subset_normal {N : Subgroup G} [tn : N.Normal] {a : G} (h : a ∈ N) : conjugatesOf a ⊆ N := by rintro a hc obtain ⟨c, rfl⟩ := isConj_iff.1 hc exact tn.conj_mem a h c theorem conjugatesOfSet_subset {s : Set G} {N : Subgroup G} [N.Normal] (h : s ⊆ N) : conjugatesOfSet s ⊆ N := Set.iUnion₂_subset fun _x H => conjugates_subset_normal (h H) /-- The set of conjugates of `s` is closed under conjugation. -/ theorem conj_mem_conjugatesOfSet {x c : G} : x ∈ conjugatesOfSet s → c * x * c⁻¹ ∈ conjugatesOfSet s := fun H => by rcases mem_conjugatesOfSet_iff.1 H with ⟨a, h₁, h₂⟩ exact mem_conjugatesOfSet_iff.2 ⟨a, h₁, h₂.trans (isConj_iff.2 ⟨c, rfl⟩)⟩ end Group namespace Subgroup open Group variable {s : Set G} /-- The normal closure of a set `s` is the subgroup closure of all the conjugates of elements of `s`. It is the smallest normal subgroup containing `s`. -/ def normalClosure (s : Set G) : Subgroup G := closure (conjugatesOfSet s) theorem conjugatesOfSet_subset_normalClosure : conjugatesOfSet s ⊆ normalClosure s := subset_closure theorem subset_normalClosure : s ⊆ normalClosure s := Set.Subset.trans subset_conjugatesOfSet conjugatesOfSet_subset_normalClosure theorem le_normalClosure {H : Subgroup G} : H ≤ normalClosure ↑H := fun _ h => subset_normalClosure h /-- The normal closure of `s` is a normal subgroup. -/ instance normalClosure_normal : (normalClosure s).Normal := ⟨fun n h g => by refine Subgroup.closure_induction h (fun x hx => ?_) ?_ (fun x y ihx ihy => ?_) fun x ihx => ?_ · exact conjugatesOfSet_subset_normalClosure (conj_mem_conjugatesOfSet hx) · simpa using (normalClosure s).one_mem · rw [← conj_mul] exact mul_mem ihx ihy · rw [← conj_inv] exact inv_mem ihx⟩ /-- The normal closure of `s` is the smallest normal subgroup containing `s`. -/ theorem normalClosure_le_normal {N : Subgroup G} [N.Normal] (h : s ⊆ N) : normalClosure s ≤ N := by intro a w refine closure_induction w (fun x hx => ?_) ?_ (fun x y ihx ihy => ?_) fun x ihx => ?_ · exact conjugatesOfSet_subset h hx · exact one_mem _ · exact mul_mem ihx ihy · exact inv_mem ihx theorem normalClosure_subset_iff {N : Subgroup G} [N.Normal] : s ⊆ N ↔ normalClosure s ≤ N := ⟨normalClosure_le_normal, Set.Subset.trans subset_normalClosure⟩ theorem normalClosure_mono {s t : Set G} (h : s ⊆ t) : normalClosure s ≤ normalClosure t := normalClosure_le_normal (Set.Subset.trans h subset_normalClosure) theorem normalClosure_eq_iInf : normalClosure s = ⨅ (N : Subgroup G) (_ : Normal N) (_ : s ⊆ N), N := le_antisymm (le_iInf fun N => le_iInf fun hN => le_iInf normalClosure_le_normal) (iInf_le_of_le (normalClosure s) (iInf_le_of_le (by infer_instance) (iInf_le_of_le subset_normalClosure le_rfl))) @[simp] theorem normalClosure_eq_self (H : Subgroup G) [H.Normal] : normalClosure ↑H = H := le_antisymm (normalClosure_le_normal rfl.subset) le_normalClosure -- @[simp] -- Porting note (#10618): simp can prove this theorem normalClosure_idempotent : normalClosure ↑(normalClosure s) = normalClosure s := normalClosure_eq_self _ theorem closure_le_normalClosure {s : Set G} : closure s ≤ normalClosure s := by simp only [subset_normalClosure, closure_le] @[simp] theorem normalClosure_closure_eq_normalClosure {s : Set G} : normalClosure ↑(closure s) = normalClosure s := le_antisymm (normalClosure_le_normal closure_le_normalClosure) (normalClosure_mono subset_closure) /-- The normal core of a subgroup `H` is the largest normal subgroup of `G` contained in `H`, as shown by `Subgroup.normalCore_eq_iSup`. -/ def normalCore (H : Subgroup G) : Subgroup G where carrier := { a : G | ∀ b : G, b * a * b⁻¹ ∈ H } one_mem' a := by rw [mul_one, mul_inv_self]; exact H.one_mem inv_mem' {a} h b := (congr_arg (· ∈ H) conj_inv).mp (H.inv_mem (h b)) mul_mem' {a b} ha hb c := (congr_arg (· ∈ H) conj_mul).mp (H.mul_mem (ha c) (hb c)) theorem normalCore_le (H : Subgroup G) : H.normalCore ≤ H := fun a h => by rw [← mul_one a, ← inv_one, ← one_mul a] exact h 1 instance normalCore_normal (H : Subgroup G) : H.normalCore.Normal := ⟨fun a h b c => by rw [mul_assoc, mul_assoc, ← mul_inv_rev, ← mul_assoc, ← mul_assoc]; exact h (c * b)⟩ theorem normal_le_normalCore {H : Subgroup G} {N : Subgroup G} [hN : N.Normal] : N ≤ H.normalCore ↔ N ≤ H := ⟨ge_trans H.normalCore_le, fun h_le n hn g => h_le (hN.conj_mem n hn g)⟩ theorem normalCore_mono {H K : Subgroup G} (h : H ≤ K) : H.normalCore ≤ K.normalCore := normal_le_normalCore.mpr (H.normalCore_le.trans h) theorem normalCore_eq_iSup (H : Subgroup G) : H.normalCore = ⨆ (N : Subgroup G) (_ : Normal N) (_ : N ≤ H), N := le_antisymm (le_iSup_of_le H.normalCore (le_iSup_of_le H.normalCore_normal (le_iSup_of_le H.normalCore_le le_rfl))) (iSup_le fun _ => iSup_le fun _ => iSup_le normal_le_normalCore.mpr) @[simp] theorem normalCore_eq_self (H : Subgroup G) [H.Normal] : H.normalCore = H := le_antisymm H.normalCore_le (normal_le_normalCore.mpr le_rfl) -- @[simp] -- Porting note (#10618): simp can prove this theorem normalCore_idempotent (H : Subgroup G) : H.normalCore.normalCore = H.normalCore := H.normalCore.normalCore_eq_self end Subgroup namespace MonoidHom variable {N : Type*} {P : Type*} [Group N] [Group P] (K : Subgroup G) open Subgroup /-- The range of a monoid homomorphism from a group is a subgroup. -/ @[to_additive "The range of an `AddMonoidHom` from an `AddGroup` is an `AddSubgroup`."] def range (f : G →* N) : Subgroup N := Subgroup.copy ((⊤ : Subgroup G).map f) (Set.range f) (by simp [Set.ext_iff]) @[to_additive (attr := simp)] theorem coe_range (f : G →* N) : (f.range : Set N) = Set.range f := rfl @[to_additive (attr := simp)] theorem mem_range {f : G →* N} {y : N} : y ∈ f.range ↔ ∃ x, f x = y := Iff.rfl @[to_additive] theorem range_eq_map (f : G →* N) : f.range = (⊤ : Subgroup G).map f := by ext; simp @[to_additive] instance range_isCommutative {G : Type*} [CommGroup G] {N : Type*} [Group N] (f : G →* N) : f.range.IsCommutative := range_eq_map f ▸ Subgroup.map_isCommutative ⊤ f @[to_additive (attr := simp)] theorem restrict_range (f : G →* N) : (f.restrict K).range = K.map f := by simp_rw [SetLike.ext_iff, mem_range, mem_map, restrict_apply, SetLike.exists, exists_prop, forall_const] /-- The canonical surjective group homomorphism `G →* f(G)` induced by a group homomorphism `G →* N`. -/ @[to_additive "The canonical surjective `AddGroup` homomorphism `G →+ f(G)` induced by a group homomorphism `G →+ N`."] def rangeRestrict (f : G →* N) : G →* f.range := codRestrict f _ fun x => ⟨x, rfl⟩ @[to_additive (attr := simp)] theorem coe_rangeRestrict (f : G →* N) (g : G) : (f.rangeRestrict g : N) = f g := rfl @[to_additive] theorem coe_comp_rangeRestrict (f : G →* N) : ((↑) : f.range → N) ∘ (⇑f.rangeRestrict : G → f.range) = f := rfl @[to_additive] theorem subtype_comp_rangeRestrict (f : G →* N) : f.range.subtype.comp f.rangeRestrict = f := ext <| f.coe_rangeRestrict @[to_additive] theorem rangeRestrict_surjective (f : G →* N) : Function.Surjective f.rangeRestrict := fun ⟨_, g, rfl⟩ => ⟨g, rfl⟩ @[to_additive (attr := simp)] lemma rangeRestrict_injective_iff {f : G →* N} : Injective f.rangeRestrict ↔ Injective f := by convert Set.injective_codRestrict _ @[to_additive] theorem map_range (g : N →* P) (f : G →* N) : f.range.map g = (g.comp f).range := by rw [range_eq_map, range_eq_map]; exact (⊤ : Subgroup G).map_map g f @[to_additive] theorem range_top_iff_surjective {N} [Group N] {f : G →* N} : f.range = (⊤ : Subgroup N) ↔ Function.Surjective f := SetLike.ext'_iff.trans <| Iff.trans (by rw [coe_range, coe_top]) Set.range_iff_surjective /-- The range of a surjective monoid homomorphism is the whole of the codomain. -/ @[to_additive (attr := simp) "The range of a surjective `AddMonoid` homomorphism is the whole of the codomain."] theorem range_top_of_surjective {N} [Group N] (f : G →* N) (hf : Function.Surjective f) : f.range = (⊤ : Subgroup N) := range_top_iff_surjective.2 hf @[to_additive (attr := simp)] theorem range_one : (1 : G →* N).range = ⊥ := SetLike.ext fun x => by simpa using @comm _ (· = ·) _ 1 x @[to_additive (attr := simp)] theorem _root_.Subgroup.subtype_range (H : Subgroup G) : H.subtype.range = H := by rw [range_eq_map, ← SetLike.coe_set_eq, coe_map, Subgroup.coeSubtype] ext simp @[to_additive (attr := simp)] theorem _root_.Subgroup.inclusion_range {H K : Subgroup G} (h_le : H ≤ K) : (inclusion h_le).range = H.subgroupOf K := Subgroup.ext fun g => Set.ext_iff.mp (Set.range_inclusion h_le) g @[to_additive] theorem subgroupOf_range_eq_of_le {G₁ G₂ : Type*} [Group G₁] [Group G₂] {K : Subgroup G₂} (f : G₁ →* G₂) (h : f.range ≤ K) : f.range.subgroupOf K = (f.codRestrict K fun x => h ⟨x, rfl⟩).range := by ext k refine exists_congr ?_ simp [Subtype.ext_iff] @[simp] theorem coe_toAdditive_range (f : G →* G') : (MonoidHom.toAdditive f).range = Subgroup.toAddSubgroup f.range := rfl @[simp] theorem coe_toMultiplicative_range {A A' : Type*} [AddGroup A] [AddGroup A'] (f : A →+ A') : (AddMonoidHom.toMultiplicative f).range = AddSubgroup.toSubgroup f.range := rfl /-- Computable alternative to `MonoidHom.ofInjective`. -/ @[to_additive "Computable alternative to `AddMonoidHom.ofInjective`."] def ofLeftInverse {f : G →* N} {g : N →* G} (h : Function.LeftInverse g f) : G ≃* f.range := { f.rangeRestrict with toFun := f.rangeRestrict invFun := g ∘ f.range.subtype left_inv := h right_inv := by rintro ⟨x, y, rfl⟩ apply Subtype.ext rw [coe_rangeRestrict, Function.comp_apply, Subgroup.coeSubtype, Subtype.coe_mk, h] } @[to_additive (attr := simp)] theorem ofLeftInverse_apply {f : G →* N} {g : N →* G} (h : Function.LeftInverse g f) (x : G) : ↑(ofLeftInverse h x) = f x := rfl @[to_additive (attr := simp)] theorem ofLeftInverse_symm_apply {f : G →* N} {g : N →* G} (h : Function.LeftInverse g f) (x : f.range) : (ofLeftInverse h).symm x = g x := rfl /-- The range of an injective group homomorphism is isomorphic to its domain. -/ @[to_additive "The range of an injective additive group homomorphism is isomorphic to its domain."] noncomputable def ofInjective {f : G →* N} (hf : Function.Injective f) : G ≃* f.range := MulEquiv.ofBijective (f.codRestrict f.range fun x => ⟨x, rfl⟩) ⟨fun x y h => hf (Subtype.ext_iff.mp h), by rintro ⟨x, y, rfl⟩ exact ⟨y, rfl⟩⟩ @[to_additive] theorem ofInjective_apply {f : G →* N} (hf : Function.Injective f) {x : G} : ↑(ofInjective hf x) = f x := rfl @[to_additive (attr := simp)] theorem apply_ofInjective_symm {f : G →* N} (hf : Function.Injective f) (x : f.range) : f ((ofInjective hf).symm x) = x := Subtype.ext_iff.1 <| (ofInjective hf).apply_symm_apply x section Ker variable {M : Type*} [MulOneClass M] /-- The multiplicative kernel of a monoid homomorphism is the subgroup of elements `x : G` such that `f x = 1` -/ @[to_additive "The additive kernel of an `AddMonoid` homomorphism is the `AddSubgroup` of elements such that `f x = 0`"] def ker (f : G →* M) : Subgroup G := { MonoidHom.mker f with inv_mem' := fun {x} (hx : f x = 1) => calc f x⁻¹ = f x * f x⁻¹ := by rw [hx, one_mul] _ = 1 := by rw [← map_mul, mul_inv_self, map_one] } @[to_additive] theorem mem_ker (f : G →* M) {x : G} : x ∈ f.ker ↔ f x = 1 := Iff.rfl @[to_additive] theorem coe_ker (f : G →* M) : (f.ker : Set G) = (f : G → M) ⁻¹' {1} := rfl @[to_additive (attr := simp)] theorem ker_toHomUnits {M} [Monoid M] (f : G →* M) : f.toHomUnits.ker = f.ker := by ext x simp [mem_ker, Units.ext_iff] @[to_additive] theorem eq_iff (f : G →* M) {x y : G} : f x = f y ↔ y⁻¹ * x ∈ f.ker := by constructor <;> intro h · rw [mem_ker, map_mul, h, ← map_mul, inv_mul_self, map_one] · rw [← one_mul x, ← mul_inv_self y, mul_assoc, map_mul, f.mem_ker.1 h, mul_one] @[to_additive] instance decidableMemKer [DecidableEq M] (f : G →* M) : DecidablePred (· ∈ f.ker) := fun x => decidable_of_iff (f x = 1) f.mem_ker @[to_additive] theorem comap_ker (g : N →* P) (f : G →* N) : g.ker.comap f = (g.comp f).ker := rfl @[to_additive (attr := simp)] theorem comap_bot (f : G →* N) : (⊥ : Subgroup N).comap f = f.ker := rfl @[to_additive (attr := simp)] theorem ker_restrict (f : G →* N) : (f.restrict K).ker = f.ker.subgroupOf K := rfl @[to_additive (attr := simp)] theorem ker_codRestrict {S} [SetLike S N] [SubmonoidClass S N] (f : G →* N) (s : S) (h : ∀ x, f x ∈ s) : (f.codRestrict s h).ker = f.ker := SetLike.ext fun _x => Subtype.ext_iff @[to_additive (attr := simp)] theorem ker_rangeRestrict (f : G →* N) : ker (rangeRestrict f) = ker f := ker_codRestrict _ _ _ @[to_additive (attr := simp)] theorem ker_one : (1 : G →* M).ker = ⊤ := SetLike.ext fun _x => eq_self_iff_true _ @[to_additive (attr := simp)] theorem ker_id : (MonoidHom.id G).ker = ⊥ := rfl @[to_additive] theorem ker_eq_bot_iff (f : G →* M) : f.ker = ⊥ ↔ Function.Injective f := ⟨fun h x y hxy => by rwa [eq_iff, h, mem_bot, inv_mul_eq_one, eq_comm] at hxy, fun h => bot_unique fun x hx => h (hx.trans f.map_one.symm)⟩ @[to_additive (attr := simp)] theorem _root_.Subgroup.ker_subtype (H : Subgroup G) : H.subtype.ker = ⊥ := H.subtype.ker_eq_bot_iff.mpr Subtype.coe_injective @[to_additive (attr := simp)] theorem _root_.Subgroup.ker_inclusion {H K : Subgroup G} (h : H ≤ K) : (inclusion h).ker = ⊥ := (inclusion h).ker_eq_bot_iff.mpr (Set.inclusion_injective h) @[to_additive] theorem ker_prod {M N : Type*} [MulOneClass M] [MulOneClass N] (f : G →* M) (g : G →* N) : (f.prod g).ker = f.ker ⊓ g.ker := SetLike.ext fun _ => Prod.mk_eq_one @[to_additive] theorem prodMap_comap_prod {G' : Type*} {N' : Type*} [Group G'] [Group N'] (f : G →* N) (g : G' →* N') (S : Subgroup N) (S' : Subgroup N') : (S.prod S').comap (prodMap f g) = (S.comap f).prod (S'.comap g) := SetLike.coe_injective <| Set.preimage_prod_map_prod f g _ _ @[to_additive] theorem ker_prodMap {G' : Type*} {N' : Type*} [Group G'] [Group N'] (f : G →* N) (g : G' →* N') : (prodMap f g).ker = f.ker.prod g.ker := by rw [← comap_bot, ← comap_bot, ← comap_bot, ← prodMap_comap_prod, bot_prod_bot] @[to_additive] theorem range_le_ker_iff (f : G →* G') (g : G' →* G'') : f.range ≤ g.ker ↔ g.comp f = 1 := ⟨fun h => ext fun x => h ⟨x, rfl⟩, by rintro h _ ⟨y, rfl⟩; exact DFunLike.congr_fun h y⟩ @[to_additive] instance (priority := 100) normal_ker (f : G →* M) : f.ker.Normal := ⟨fun x hx y => by rw [mem_ker, map_mul, map_mul, f.mem_ker.1 hx, mul_one, map_mul_eq_one f (mul_inv_self y)]⟩ @[to_additive (attr := simp)] lemma ker_fst : ker (fst G G') = .prod ⊥ ⊤ := SetLike.ext fun _ => (and_true_iff _).symm @[to_additive (attr := simp)] lemma ker_snd : ker (snd G G') = .prod ⊤ ⊥ := SetLike.ext fun _ => (true_and_iff _).symm @[simp] theorem coe_toAdditive_ker (f : G →* G') : (MonoidHom.toAdditive f).ker = Subgroup.toAddSubgroup f.ker := rfl @[simp] theorem coe_toMultiplicative_ker {A A' : Type*} [AddGroup A] [AddGroup A'] (f : A →+ A') : (AddMonoidHom.toMultiplicative f).ker = AddSubgroup.toSubgroup f.ker := rfl end Ker section EqLocus variable {M : Type*} [Monoid M] /-- The subgroup of elements `x : G` such that `f x = g x` -/ @[to_additive "The additive subgroup of elements `x : G` such that `f x = g x`"] def eqLocus (f g : G →* M) : Subgroup G := { eqLocusM f g with inv_mem' := eq_on_inv f g } @[to_additive (attr := simp)] theorem eqLocus_same (f : G →* N) : f.eqLocus f = ⊤ := SetLike.ext fun _ => eq_self_iff_true _ /-- If two monoid homomorphisms are equal on a set, then they are equal on its subgroup closure. -/ @[to_additive "If two monoid homomorphisms are equal on a set, then they are equal on its subgroup closure."] theorem eqOn_closure {f g : G →* M} {s : Set G} (h : Set.EqOn f g s) : Set.EqOn f g (closure s) := show closure s ≤ f.eqLocus g from (closure_le _).2 h @[to_additive] theorem eq_of_eqOn_top {f g : G →* M} (h : Set.EqOn f g (⊤ : Subgroup G)) : f = g := ext fun _x => h trivial @[to_additive] theorem eq_of_eqOn_dense {s : Set G} (hs : closure s = ⊤) {f g : G →* M} (h : s.EqOn f g) : f = g := eq_of_eqOn_top <| hs ▸ eqOn_closure h end EqLocus @[to_additive] theorem closure_preimage_le (f : G →* N) (s : Set N) : closure (f ⁻¹' s) ≤ (closure s).comap f := (closure_le _).2 fun x hx => by rw [SetLike.mem_coe, mem_comap]; exact subset_closure hx /-- The image under a monoid homomorphism of the subgroup generated by a set equals the subgroup generated by the image of the set. -/ @[to_additive "The image under an `AddMonoid` hom of the `AddSubgroup` generated by a set equals the `AddSubgroup` generated by the image of the set."] theorem map_closure (f : G →* N) (s : Set G) : (closure s).map f = closure (f '' s) := Set.image_preimage.l_comm_of_u_comm (Subgroup.gc_map_comap f) (Subgroup.gi N).gc (Subgroup.gi G).gc fun _t => rfl end MonoidHom namespace Subgroup variable {N : Type*} [Group N] (H : Subgroup G) @[to_additive] theorem Normal.map {H : Subgroup G} (h : H.Normal) (f : G →* N) (hf : Function.Surjective f) : (H.map f).Normal := by rw [← normalizer_eq_top, ← top_le_iff, ← f.range_top_of_surjective hf, f.range_eq_map, ← normalizer_eq_top.2 h] exact le_normalizer_map _ @[to_additive] theorem map_eq_bot_iff {f : G →* N} : H.map f = ⊥ ↔ H ≤ f.ker := (gc_map_comap f).l_eq_bot @[to_additive] theorem map_eq_bot_iff_of_injective {f : G →* N} (hf : Function.Injective f) : H.map f = ⊥ ↔ H = ⊥ := by rw [map_eq_bot_iff, f.ker_eq_bot_iff.mpr hf, le_bot_iff] end Subgroup namespace Subgroup open MonoidHom variable {N : Type*} [Group N] (f : G →* N) @[to_additive] theorem map_le_range (H : Subgroup G) : map f H ≤ f.range := (range_eq_map f).symm ▸ map_mono le_top @[to_additive] theorem map_subtype_le {H : Subgroup G} (K : Subgroup H) : K.map H.subtype ≤ H := (K.map_le_range H.subtype).trans (le_of_eq H.subtype_range) @[to_additive] theorem ker_le_comap (H : Subgroup N) : f.ker ≤ comap f H := comap_bot f ▸ comap_mono bot_le @[to_additive] theorem map_comap_le (H : Subgroup N) : map f (comap f H) ≤ H := (gc_map_comap f).l_u_le _ @[to_additive] theorem le_comap_map (H : Subgroup G) : H ≤ comap f (map f H) := (gc_map_comap f).le_u_l _ @[to_additive] theorem map_comap_eq (H : Subgroup N) : map f (comap f H) = f.range ⊓ H := SetLike.ext' <| by rw [coe_map, coe_comap, Set.image_preimage_eq_inter_range, coe_inf, coe_range, Set.inter_comm] @[to_additive] theorem comap_map_eq (H : Subgroup G) : comap f (map f H) = H ⊔ f.ker := by refine le_antisymm ?_ (sup_le (le_comap_map _ _) (ker_le_comap _ _)) intro x hx; simp only [exists_prop, mem_map, mem_comap] at hx rcases hx with ⟨y, hy, hy'⟩ rw [← mul_inv_cancel_left y x] exact mul_mem_sup hy (by simp [mem_ker, hy']) @[to_additive] theorem map_comap_eq_self {f : G →* N} {H : Subgroup N} (h : H ≤ f.range) : map f (comap f H) = H := by rwa [map_comap_eq, inf_eq_right] @[to_additive] theorem map_comap_eq_self_of_surjective {f : G →* N} (h : Function.Surjective f) (H : Subgroup N) : map f (comap f H) = H := map_comap_eq_self ((range_top_of_surjective _ h).symm ▸ le_top) @[to_additive] theorem comap_le_comap_of_le_range {f : G →* N} {K L : Subgroup N} (hf : K ≤ f.range) : K.comap f ≤ L.comap f ↔ K ≤ L := ⟨(map_comap_eq_self hf).ge.trans ∘ map_le_iff_le_comap.mpr, comap_mono⟩ @[to_additive] theorem comap_le_comap_of_surjective {f : G →* N} {K L : Subgroup N} (hf : Function.Surjective f) : K.comap f ≤ L.comap f ↔ K ≤ L := comap_le_comap_of_le_range (le_top.trans (f.range_top_of_surjective hf).ge) @[to_additive] theorem comap_lt_comap_of_surjective {f : G →* N} {K L : Subgroup N} (hf : Function.Surjective f) : K.comap f < L.comap f ↔ K < L := by simp_rw [lt_iff_le_not_le, comap_le_comap_of_surjective hf] @[to_additive] theorem comap_injective {f : G →* N} (h : Function.Surjective f) : Function.Injective (comap f) := fun K L => by simp only [le_antisymm_iff, comap_le_comap_of_surjective h, imp_self] @[to_additive] theorem comap_map_eq_self {f : G →* N} {H : Subgroup G} (h : f.ker ≤ H) : comap f (map f H) = H := by rwa [comap_map_eq, sup_eq_left] @[to_additive] theorem comap_map_eq_self_of_injective {f : G →* N} (h : Function.Injective f) (H : Subgroup G) : comap f (map f H) = H := comap_map_eq_self (((ker_eq_bot_iff _).mpr h).symm ▸ bot_le) @[to_additive] theorem map_le_map_iff {f : G →* N} {H K : Subgroup G} : H.map f ≤ K.map f ↔ H ≤ K ⊔ f.ker := by rw [map_le_iff_le_comap, comap_map_eq] @[to_additive] theorem map_le_map_iff' {f : G →* N} {H K : Subgroup G} : H.map f ≤ K.map f ↔ H ⊔ f.ker ≤ K ⊔ f.ker := by simp only [map_le_map_iff, sup_le_iff, le_sup_right, and_true_iff] @[to_additive] theorem map_eq_map_iff {f : G →* N} {H K : Subgroup G} : H.map f = K.map f ↔ H ⊔ f.ker = K ⊔ f.ker := by simp only [le_antisymm_iff, map_le_map_iff'] @[to_additive] theorem map_eq_range_iff {f : G →* N} {H : Subgroup G} : H.map f = f.range ↔ Codisjoint H f.ker := by rw [f.range_eq_map, map_eq_map_iff, codisjoint_iff, top_sup_eq] @[to_additive] theorem map_le_map_iff_of_injective {f : G →* N} (hf : Function.Injective f) {H K : Subgroup G} : H.map f ≤ K.map f ↔ H ≤ K := by rw [map_le_iff_le_comap, comap_map_eq_self_of_injective hf] @[to_additive (attr := simp)] theorem map_subtype_le_map_subtype {G' : Subgroup G} {H K : Subgroup G'} : H.map G'.subtype ≤ K.map G'.subtype ↔ H ≤ K := map_le_map_iff_of_injective <| by apply Subtype.coe_injective @[to_additive] theorem map_injective {f : G →* N} (h : Function.Injective f) : Function.Injective (map f) := Function.LeftInverse.injective <| comap_map_eq_self_of_injective h @[to_additive] theorem map_eq_comap_of_inverse {f : G →* N} {g : N →* G} (hl : Function.LeftInverse g f) (hr : Function.RightInverse g f) (H : Subgroup G) : map f H = comap g H := SetLike.ext' <| by rw [coe_map, coe_comap, Set.image_eq_preimage_of_inverse hl hr] /-- Given `f(A) = f(B)`, `ker f ≤ A`, and `ker f ≤ B`, deduce that `A = B`. -/ @[to_additive "Given `f(A) = f(B)`, `ker f ≤ A`, and `ker f ≤ B`, deduce that `A = B`."] theorem map_injective_of_ker_le {H K : Subgroup G} (hH : f.ker ≤ H) (hK : f.ker ≤ K) (hf : map f H = map f K) : H = K := by apply_fun comap f at hf rwa [comap_map_eq, comap_map_eq, sup_of_le_left hH, sup_of_le_left hK] at hf @[to_additive] theorem closure_preimage_eq_top (s : Set G) : closure ((closure s).subtype ⁻¹' s) = ⊤ := by apply map_injective (closure s).subtype_injective rw [MonoidHom.map_closure, ← MonoidHom.range_eq_map, subtype_range, Set.image_preimage_eq_of_subset] rw [coeSubtype, Subtype.range_coe_subtype] exact subset_closure @[to_additive] theorem comap_sup_eq_of_le_range {H K : Subgroup N} (hH : H ≤ f.range) (hK : K ≤ f.range) : comap f H ⊔ comap f K = comap f (H ⊔ K) := map_injective_of_ker_le f ((ker_le_comap f H).trans le_sup_left) (ker_le_comap f (H ⊔ K)) (by rw [map_comap_eq, map_sup, map_comap_eq, map_comap_eq, inf_eq_right.mpr hH, inf_eq_right.mpr hK, inf_eq_right.mpr (sup_le hH hK)]) @[to_additive] theorem comap_sup_eq (H K : Subgroup N) (hf : Function.Surjective f) : comap f H ⊔ comap f K = comap f (H ⊔ K) := comap_sup_eq_of_le_range f (le_top.trans (ge_of_eq (f.range_top_of_surjective hf))) (le_top.trans (ge_of_eq (f.range_top_of_surjective hf))) @[to_additive] theorem sup_subgroupOf_eq {H K L : Subgroup G} (hH : H ≤ L) (hK : K ≤ L) : H.subgroupOf L ⊔ K.subgroupOf L = (H ⊔ K).subgroupOf L := comap_sup_eq_of_le_range L.subtype (hH.trans L.subtype_range.ge) (hK.trans L.subtype_range.ge) @[to_additive] theorem codisjoint_subgroupOf_sup (H K : Subgroup G) : Codisjoint (H.subgroupOf (H ⊔ K)) (K.subgroupOf (H ⊔ K)) := by rw [codisjoint_iff, sup_subgroupOf_eq, subgroupOf_self] exacts [le_sup_left, le_sup_right] /-- A subgroup is isomorphic to its image under an injective function. If you have an isomorphism, use `MulEquiv.subgroupMap` for better definitional equalities. -/ @[to_additive "An additive subgroup is isomorphic to its image under an injective function. If you have an isomorphism, use `AddEquiv.addSubgroupMap` for better definitional equalities."] noncomputable def equivMapOfInjective (H : Subgroup G) (f : G →* N) (hf : Function.Injective f) : H ≃* H.map f := { Equiv.Set.image f H hf with map_mul' := fun _ _ => Subtype.ext (f.map_mul _ _) } @[to_additive (attr := simp)] theorem coe_equivMapOfInjective_apply (H : Subgroup G) (f : G →* N) (hf : Function.Injective f) (h : H) : (equivMapOfInjective H f hf h : N) = f h := rfl /-- The preimage of the normalizer is equal to the normalizer of the preimage of a surjective function. -/ @[to_additive "The preimage of the normalizer is equal to the normalizer of the preimage of a surjective function."] theorem comap_normalizer_eq_of_surjective (H : Subgroup G) {f : N →* G} (hf : Function.Surjective f) : H.normalizer.comap f = (H.comap f).normalizer := le_antisymm (le_normalizer_comap f) (by intro x hx simp only [mem_comap, mem_normalizer_iff] at * intro n rcases hf n with ⟨y, rfl⟩ simp [hx y]) @[to_additive] theorem comap_normalizer_eq_of_injective_of_le_range {N : Type*} [Group N] (H : Subgroup G) {f : N →* G} (hf : Function.Injective f) (h : H.normalizer ≤ f.range) : comap f H.normalizer = (comap f H).normalizer := by apply Subgroup.map_injective hf rw [map_comap_eq_self h] apply le_antisymm · refine le_trans (le_of_eq ?_) (map_mono (le_normalizer_comap _)) rw [map_comap_eq_self h] · refine le_trans (le_normalizer_map f) (le_of_eq ?_) rw [map_comap_eq_self (le_trans le_normalizer h)] @[to_additive] theorem subgroupOf_normalizer_eq {H N : Subgroup G} (h : H.normalizer ≤ N) : H.normalizer.subgroupOf N = (H.subgroupOf N).normalizer := by apply comap_normalizer_eq_of_injective_of_le_range · exact Subtype.coe_injective simpa /-- The image of the normalizer is equal to the normalizer of the image of an isomorphism. -/ @[to_additive "The image of the normalizer is equal to the normalizer of the image of an isomorphism."] theorem map_equiv_normalizer_eq (H : Subgroup G) (f : G ≃* N) : H.normalizer.map f.toMonoidHom = (H.map f.toMonoidHom).normalizer := by ext x simp only [mem_normalizer_iff, mem_map_equiv] rw [f.toEquiv.forall_congr] intro erw [f.toEquiv.symm_apply_apply] simp only [map_mul, map_inv] erw [f.toEquiv.symm_apply_apply] /-- The image of the normalizer is equal to the normalizer of the image of a bijective function. -/ @[to_additive "The image of the normalizer is equal to the normalizer of the image of a bijective function."] theorem map_normalizer_eq_of_bijective (H : Subgroup G) {f : G →* N} (hf : Function.Bijective f) : H.normalizer.map f = (H.map f).normalizer := map_equiv_normalizer_eq H (MulEquiv.ofBijective f hf) end Subgroup namespace MonoidHom variable {G₁ G₂ G₃ : Type*} [Group G₁] [Group G₂] [Group G₃] variable (f : G₁ →* G₂) (f_inv : G₂ → G₁) /-- Auxiliary definition used to define `liftOfRightInverse` -/ @[to_additive "Auxiliary definition used to define `liftOfRightInverse`"] def liftOfRightInverseAux (hf : Function.RightInverse f_inv f) (g : G₁ →* G₃) (hg : f.ker ≤ g.ker) : G₂ →* G₃ where toFun b := g (f_inv b) map_one' := hg (hf 1) map_mul' := by intro x y rw [← g.map_mul, ← mul_inv_eq_one, ← g.map_inv, ← g.map_mul, ← g.mem_ker] apply hg rw [f.mem_ker, f.map_mul, f.map_inv, mul_inv_eq_one, f.map_mul] simp only [hf _] @[to_additive (attr := simp)] theorem liftOfRightInverseAux_comp_apply (hf : Function.RightInverse f_inv f) (g : G₁ →* G₃) (hg : f.ker ≤ g.ker) (x : G₁) : (f.liftOfRightInverseAux f_inv hf g hg) (f x) = g x := by dsimp [liftOfRightInverseAux] rw [← mul_inv_eq_one, ← g.map_inv, ← g.map_mul, ← g.mem_ker] apply hg rw [f.mem_ker, f.map_mul, f.map_inv, mul_inv_eq_one] simp only [hf _] /-- `liftOfRightInverse f hf g hg` is the unique group homomorphism `φ` * such that `φ.comp f = g` (`MonoidHom.liftOfRightInverse_comp`), * where `f : G₁ →+* G₂` has a RightInverse `f_inv` (`hf`), * and `g : G₂ →+* G₃` satisfies `hg : f.ker ≤ g.ker`. See `MonoidHom.eq_liftOfRightInverse` for the uniqueness lemma. ``` G₁. | \ f | \ g | \ v \⌟ G₂----> G₃ ∃!φ ``` -/ @[to_additive "`liftOfRightInverse f f_inv hf g hg` is the unique additive group homomorphism `φ` * such that `φ.comp f = g` (`AddMonoidHom.liftOfRightInverse_comp`), * where `f : G₁ →+ G₂` has a RightInverse `f_inv` (`hf`), * and `g : G₂ →+ G₃` satisfies `hg : f.ker ≤ g.ker`. See `AddMonoidHom.eq_liftOfRightInverse` for the uniqueness lemma. ``` G₁. | \\ f | \\ g | \\ v \\⌟ G₂----> G₃ ∃!φ ```"] def liftOfRightInverse (hf : Function.RightInverse f_inv f) : { g : G₁ →* G₃ // f.ker ≤ g.ker } ≃ (G₂ →* G₃) where toFun g := f.liftOfRightInverseAux f_inv hf g.1 g.2 invFun φ := ⟨φ.comp f, fun x hx => (mem_ker _).mpr <| by simp [(mem_ker _).mp hx]⟩ left_inv g := by ext simp only [comp_apply, liftOfRightInverseAux_comp_apply, Subtype.coe_mk] right_inv φ := by ext b simp [liftOfRightInverseAux, hf b] /-- A non-computable version of `MonoidHom.liftOfRightInverse` for when no computable right inverse is available, that uses `Function.surjInv`. -/ @[to_additive (attr := simp) "A non-computable version of `AddMonoidHom.liftOfRightInverse` for when no computable right inverse is available."] noncomputable abbrev liftOfSurjective (hf : Function.Surjective f) : { g : G₁ →* G₃ // f.ker ≤ g.ker } ≃ (G₂ →* G₃) := f.liftOfRightInverse (Function.surjInv hf) (Function.rightInverse_surjInv hf) @[to_additive (attr := simp)] theorem liftOfRightInverse_comp_apply (hf : Function.RightInverse f_inv f) (g : { g : G₁ →* G₃ // f.ker ≤ g.ker }) (x : G₁) : (f.liftOfRightInverse f_inv hf g) (f x) = g.1 x := f.liftOfRightInverseAux_comp_apply f_inv hf g.1 g.2 x @[to_additive (attr := simp)] theorem liftOfRightInverse_comp (hf : Function.RightInverse f_inv f) (g : { g : G₁ →* G₃ // f.ker ≤ g.ker }) : (f.liftOfRightInverse f_inv hf g).comp f = g := MonoidHom.ext <| f.liftOfRightInverse_comp_apply f_inv hf g @[to_additive] theorem eq_liftOfRightInverse (hf : Function.RightInverse f_inv f) (g : G₁ →* G₃) (hg : f.ker ≤ g.ker) (h : G₂ →* G₃) (hh : h.comp f = g) : h = f.liftOfRightInverse f_inv hf ⟨g, hg⟩ := by simp_rw [← hh] exact ((f.liftOfRightInverse f_inv hf).apply_symm_apply _).symm end MonoidHom variable {N : Type*} [Group N] namespace Subgroup -- Here `H.Normal` is an explicit argument so we can use dot notation with `comap`. @[to_additive] theorem Normal.comap {H : Subgroup N} (hH : H.Normal) (f : G →* N) : (H.comap f).Normal := ⟨fun _ => by simp (config := { contextual := true }) [Subgroup.mem_comap, hH.conj_mem]⟩ @[to_additive] instance (priority := 100) normal_comap {H : Subgroup N} [nH : H.Normal] (f : G →* N) : (H.comap f).Normal := nH.comap _ -- Here `H.Normal` is an explicit argument so we can use dot notation with `subgroupOf`. @[to_additive] theorem Normal.subgroupOf {H : Subgroup G} (hH : H.Normal) (K : Subgroup G) : (H.subgroupOf K).Normal := hH.comap _ @[to_additive] instance (priority := 100) normal_subgroupOf {H N : Subgroup G} [N.Normal] : (N.subgroupOf H).Normal := Subgroup.normal_comap _ theorem map_normalClosure (s : Set G) (f : G →* N) (hf : Surjective f) : (normalClosure s).map f = normalClosure (f '' s) := by have : Normal (map f (normalClosure s)) := Normal.map inferInstance f hf apply le_antisymm · simp [map_le_iff_le_comap, normalClosure_le_normal, coe_comap, ← Set.image_subset_iff, subset_normalClosure] · exact normalClosure_le_normal (Set.image_subset f subset_normalClosure) theorem comap_normalClosure (s : Set N) (f : G ≃* N) : normalClosure (f ⁻¹' s) = (normalClosure s).comap f := by have := Set.preimage_equiv_eq_image_symm s f.toEquiv simp_all [comap_equiv_eq_map_symm, map_normalClosure s f.symm f.symm.surjective] lemma Normal.of_map_injective {G H : Type*} [Group G] [Group H] {φ : G →* H} (hφ : Function.Injective φ) {L : Subgroup G} (n : (L.map φ).Normal) : L.Normal := L.comap_map_eq_self_of_injective hφ ▸ n.comap φ theorem Normal.of_map_subtype {K : Subgroup G} {L : Subgroup K} (n : (Subgroup.map K.subtype L).Normal) : L.Normal := n.of_map_injective K.subtype_injective end Subgroup namespace MonoidHom /-- The `MonoidHom` from the preimage of a subgroup to itself. -/ @[to_additive (attr := simps!) "the `AddMonoidHom` from the preimage of an additive subgroup to itself."] def subgroupComap (f : G →* G') (H' : Subgroup G') : H'.comap f →* H' := f.submonoidComap H'.toSubmonoid /-- The `MonoidHom` from a subgroup to its image. -/ @[to_additive (attr := simps!) "the `AddMonoidHom` from an additive subgroup to its image"] def subgroupMap (f : G →* G') (H : Subgroup G) : H →* H.map f := f.submonoidMap H.toSubmonoid @[to_additive] theorem subgroupMap_surjective (f : G →* G') (H : Subgroup G) : Function.Surjective (f.subgroupMap H) := f.submonoidMap_surjective H.toSubmonoid end MonoidHom namespace MulEquiv variable {H K : Subgroup G} /-- Makes the identity isomorphism from a proof two subgroups of a multiplicative group are equal. -/ @[to_additive "Makes the identity additive isomorphism from a proof two subgroups of an additive group are equal."] def subgroupCongr (h : H = K) : H ≃* K := { Equiv.setCongr <| congr_arg _ h with map_mul' := fun _ _ => rfl } @[to_additive (attr := simp)] lemma subgroupCongr_apply (h : H = K) (x) : (MulEquiv.subgroupCongr h x : G) = x := rfl @[to_additive (attr := simp)] lemma subgroupCongr_symm_apply (h : H = K) (x) : ((MulEquiv.subgroupCongr h).symm x : G) = x := rfl /-- A subgroup is isomorphic to its image under an isomorphism. If you only have an injective map, use `Subgroup.equiv_map_of_injective`. -/ @[to_additive "An additive subgroup is isomorphic to its image under an isomorphism. If you only have an injective map, use `AddSubgroup.equiv_map_of_injective`."] def subgroupMap (e : G ≃* G') (H : Subgroup G) : H ≃* H.map (e : G →* G') := MulEquiv.submonoidMap (e : G ≃* G') H.toSubmonoid @[to_additive (attr := simp)] theorem coe_subgroupMap_apply (e : G ≃* G') (H : Subgroup G) (g : H) : ((subgroupMap e H g : H.map (e : G →* G')) : G') = e g := rfl @[to_additive (attr := simp)] theorem subgroupMap_symm_apply (e : G ≃* G') (H : Subgroup G) (g : H.map (e : G →* G')) : (e.subgroupMap H).symm g = ⟨e.symm g, SetLike.mem_coe.1 <| Set.mem_image_equiv.1 g.2⟩ := rfl end MulEquiv namespace Subgroup @[to_additive (attr := simp)] theorem equivMapOfInjective_coe_mulEquiv (H : Subgroup G) (e : G ≃* G') : H.equivMapOfInjective (e : G →* G') (EquivLike.injective e) = e.subgroupMap H := by ext rfl variable {C : Type*} [CommGroup C] {s t : Subgroup C} {x : C} @[to_additive] theorem mem_sup : x ∈ s ⊔ t ↔ ∃ y ∈ s, ∃ z ∈ t, y * z = x := ⟨fun h => by rw [sup_eq_closure] at h refine Subgroup.closure_induction h ?_ ?_ ?_ ?_ · rintro y (h | h) · exact ⟨y, h, 1, t.one_mem, by simp⟩ · exact ⟨1, s.one_mem, y, h, by simp⟩ · exact ⟨1, s.one_mem, 1, ⟨t.one_mem, mul_one 1⟩⟩ · rintro _ _ ⟨y₁, hy₁, z₁, hz₁, rfl⟩ ⟨y₂, hy₂, z₂, hz₂, rfl⟩ exact ⟨_, mul_mem hy₁ hy₂, _, mul_mem hz₁ hz₂, by simp [mul_assoc, mul_left_comm]⟩ · rintro _ ⟨y, hy, z, hz, rfl⟩ exact ⟨_, inv_mem hy, _, inv_mem hz, mul_comm z y ▸ (mul_inv_rev z y).symm⟩, by rintro ⟨y, hy, z, hz, rfl⟩; exact mul_mem_sup hy hz⟩ @[to_additive] theorem mem_sup' : x ∈ s ⊔ t ↔ ∃ (y : s) (z : t), (y : C) * z = x := mem_sup.trans <| by simp only [SetLike.exists, coe_mk, exists_prop] @[to_additive] theorem mem_closure_pair {x y z : C} : z ∈ closure ({x, y} : Set C) ↔ ∃ m n : ℤ, x ^ m * y ^ n = z := by rw [← Set.singleton_union, Subgroup.closure_union, mem_sup] simp_rw [mem_closure_singleton, exists_exists_eq_and] end Subgroup namespace Subgroup section SubgroupNormal @[to_additive] theorem normal_subgroupOf_iff {H K : Subgroup G} (hHK : H ≤ K) : (H.subgroupOf K).Normal ↔ ∀ h k, h ∈ H → k ∈ K → k * h * k⁻¹ ∈ H := ⟨fun hN h k hH hK => hN.conj_mem ⟨h, hHK hH⟩ hH ⟨k, hK⟩, fun hN => { conj_mem := fun h hm k => hN h.1 k.1 hm k.2 }⟩ @[to_additive] instance prod_subgroupOf_prod_normal {H₁ K₁ : Subgroup G} {H₂ K₂ : Subgroup N} [h₁ : (H₁.subgroupOf K₁).Normal] [h₂ : (H₂.subgroupOf K₂).Normal] : ((H₁.prod H₂).subgroupOf (K₁.prod K₂)).Normal where conj_mem n hgHK g := ⟨h₁.conj_mem ⟨(n : G × N).fst, (mem_prod.mp n.2).1⟩ hgHK.1 ⟨(g : G × N).fst, (mem_prod.mp g.2).1⟩, h₂.conj_mem ⟨(n : G × N).snd, (mem_prod.mp n.2).2⟩ hgHK.2 ⟨(g : G × N).snd, (mem_prod.mp g.2).2⟩⟩ @[to_additive] instance prod_normal (H : Subgroup G) (K : Subgroup N) [hH : H.Normal] [hK : K.Normal] : (H.prod K).Normal where conj_mem n hg g := ⟨hH.conj_mem n.fst (Subgroup.mem_prod.mp hg).1 g.fst, hK.conj_mem n.snd (Subgroup.mem_prod.mp hg).2 g.snd⟩ @[to_additive] theorem inf_subgroupOf_inf_normal_of_right (A B' B : Subgroup G) (hB : B' ≤ B) [hN : (B'.subgroupOf B).Normal] : ((A ⊓ B').subgroupOf (A ⊓ B)).Normal := { conj_mem := fun {n} hn g => ⟨mul_mem (mul_mem (mem_inf.1 g.2).1 (mem_inf.1 n.2).1) <| show ↑g⁻¹ ∈ A from (inv_mem (mem_inf.1 g.2).1), (normal_subgroupOf_iff hB).mp hN n g hn.2 (mem_inf.mp g.2).2⟩ } @[to_additive] theorem inf_subgroupOf_inf_normal_of_left {A' A : Subgroup G} (B : Subgroup G) (hA : A' ≤ A) [hN : (A'.subgroupOf A).Normal] : ((A' ⊓ B).subgroupOf (A ⊓ B)).Normal := { conj_mem := fun n hn g => ⟨(normal_subgroupOf_iff hA).mp hN n g hn.1 (mem_inf.mp g.2).1, mul_mem (mul_mem (mem_inf.1 g.2).2 (mem_inf.1 n.2).2) <| show ↑g⁻¹ ∈ B from (inv_mem (mem_inf.1 g.2).2)⟩ } @[to_additive] instance normal_inf_normal (H K : Subgroup G) [hH : H.Normal] [hK : K.Normal] : (H ⊓ K).Normal := ⟨fun n hmem g => ⟨hH.conj_mem n hmem.1 g, hK.conj_mem n hmem.2 g⟩⟩ @[to_additive] theorem subgroupOf_sup (A A' B : Subgroup G) (hA : A ≤ B) (hA' : A' ≤ B) : (A ⊔ A').subgroupOf B = A.subgroupOf B ⊔ A'.subgroupOf B := by refine map_injective_of_ker_le B.subtype (ker_le_comap _ _) (le_trans (ker_le_comap B.subtype _) le_sup_left) ?_ simp only [subgroupOf, map_comap_eq, map_sup, subtype_range] rw [inf_of_le_right (sup_le hA hA'), inf_of_le_right hA', inf_of_le_right hA] @[to_additive] theorem SubgroupNormal.mem_comm {H K : Subgroup G} (hK : H ≤ K) [hN : (H.subgroupOf K).Normal] {a b : G} (hb : b ∈ K) (h : a * b ∈ H) : b * a ∈ H := by have := (normal_subgroupOf_iff hK).mp hN (a * b) b h hb rwa [mul_assoc, mul_assoc, mul_right_inv, mul_one] at this /-- Elements of disjoint, normal subgroups commute. -/ @[to_additive "Elements of disjoint, normal subgroups commute."] theorem commute_of_normal_of_disjoint (H₁ H₂ : Subgroup G) (hH₁ : H₁.Normal) (hH₂ : H₂.Normal) (hdis : Disjoint H₁ H₂) (x y : G) (hx : x ∈ H₁) (hy : y ∈ H₂) : Commute x y := by suffices x * y * x⁻¹ * y⁻¹ = 1 by show x * y = y * x · rw [mul_assoc, mul_eq_one_iff_eq_inv] at this -- Porting note: Previous code was: -- simpa simp only [this, mul_inv_rev, inv_inv] apply hdis.le_bot constructor · suffices x * (y * x⁻¹ * y⁻¹) ∈ H₁ by simpa [mul_assoc] exact H₁.mul_mem hx (hH₁.conj_mem _ (H₁.inv_mem hx) _) · show x * y * x⁻¹ * y⁻¹ ∈ H₂ apply H₂.mul_mem _ (H₂.inv_mem hy) apply hH₂.conj_mem _ hy end SubgroupNormal @[to_additive] theorem disjoint_def {H₁ H₂ : Subgroup G} : Disjoint H₁ H₂ ↔ ∀ {x : G}, x ∈ H₁ → x ∈ H₂ → x = 1 := disjoint_iff_inf_le.trans <| by simp only [Disjoint, SetLike.le_def, mem_inf, mem_bot, and_imp] @[to_additive] theorem disjoint_def' {H₁ H₂ : Subgroup G} : Disjoint H₁ H₂ ↔ ∀ {x y : G}, x ∈ H₁ → y ∈ H₂ → x = y → x = 1 := disjoint_def.trans ⟨fun h _x _y hx hy hxy ↦ h hx <| hxy.symm ▸ hy, fun h _x hx hx' ↦ h hx hx' rfl⟩ @[to_additive] theorem disjoint_iff_mul_eq_one {H₁ H₂ : Subgroup G} : Disjoint H₁ H₂ ↔ ∀ {x y : G}, x ∈ H₁ → y ∈ H₂ → x * y = 1 → x = 1 ∧ y = 1 := disjoint_def'.trans ⟨fun h x y hx hy hxy => let hx1 : x = 1 := h hx (H₂.inv_mem hy) (eq_inv_iff_mul_eq_one.mpr hxy) ⟨hx1, by simpa [hx1] using hxy⟩, fun h x y hx hy hxy => (h hx (H₂.inv_mem hy) (mul_inv_eq_one.mpr hxy)).1⟩ @[to_additive] theorem mul_injective_of_disjoint {H₁ H₂ : Subgroup G} (h : Disjoint H₁ H₂) : Function.Injective (fun g => g.1 * g.2 : H₁ × H₂ → G) := by intro x y hxy rw [← inv_mul_eq_iff_eq_mul, ← mul_assoc, ← mul_inv_eq_one, mul_assoc] at hxy replace hxy := disjoint_iff_mul_eq_one.mp h (y.1⁻¹ * x.1).prop (x.2 * y.2⁻¹).prop hxy rwa [coe_mul, coe_mul, coe_inv, coe_inv, inv_mul_eq_one, mul_inv_eq_one, ← Subtype.ext_iff, ← Subtype.ext_iff, eq_comm, ← Prod.ext_iff] at hxy end Subgroup namespace IsConj open Subgroup theorem normalClosure_eq_top_of {N : Subgroup G} [hn : N.Normal] {g g' : G} {hg : g ∈ N} {hg' : g' ∈ N} (hc : IsConj g g') (ht : normalClosure ({⟨g, hg⟩} : Set N) = ⊤) : normalClosure ({⟨g', hg'⟩} : Set N) = ⊤ := by obtain ⟨c, rfl⟩ := isConj_iff.1 hc have h : ∀ x : N, (MulAut.conj c) x ∈ N := by rintro ⟨x, hx⟩ exact hn.conj_mem _ hx c have hs : Function.Surjective (((MulAut.conj c).toMonoidHom.restrict N).codRestrict _ h) := by rintro ⟨x, hx⟩ refine ⟨⟨c⁻¹ * x * c, ?_⟩, ?_⟩ · have h := hn.conj_mem _ hx c⁻¹ rwa [inv_inv] at h simp only [MonoidHom.codRestrict_apply, MulEquiv.coe_toMonoidHom, MulAut.conj_apply, coe_mk, MonoidHom.restrict_apply, Subtype.mk_eq_mk, ← mul_assoc, mul_inv_self, one_mul] rw [mul_assoc, mul_inv_self, mul_one] rw [eq_top_iff, ← MonoidHom.range_top_of_surjective _ hs, MonoidHom.range_eq_map] refine le_trans (map_mono (eq_top_iff.1 ht)) (map_le_iff_le_comap.2 (normalClosure_le_normal ?_)) rw [Set.singleton_subset_iff, SetLike.mem_coe] simp only [MonoidHom.codRestrict_apply, MulEquiv.coe_toMonoidHom, MulAut.conj_apply, coe_mk, MonoidHom.restrict_apply, mem_comap] exact subset_normalClosure (Set.mem_singleton _) end IsConj namespace ConjClasses /-- The conjugacy classes that are not trivial. -/ def noncenter (G : Type*) [Monoid G] : Set (ConjClasses G) := {x | x.carrier.Nontrivial} @[simp] lemma mem_noncenter {G} [Monoid G] (g : ConjClasses G) : g ∈ noncenter G ↔ g.carrier.Nontrivial := Iff.rfl end ConjClasses assert_not_exists Multiset assert_not_exists Ring
Algebra\Group\Subgroup\Finite.lean
/- Copyright (c) 2020 Kexing Ying. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Kexing Ying -/ import Mathlib.Algebra.Group.Subgroup.Basic import Mathlib.Algebra.Group.Submonoid.Membership import Mathlib.Data.Finite.Card /-! # Subgroups This file provides some result on multiplicative and additive subgroups in the finite context. ## Tags subgroup, subgroups -/ variable {G : Type*} [Group G] variable {A : Type*} [AddGroup A] namespace Subgroup @[to_additive] instance (K : Subgroup G) [DecidablePred (· ∈ K)] [Fintype G] : Fintype K := show Fintype { g : G // g ∈ K } from inferInstance @[to_additive] instance (K : Subgroup G) [Finite G] : Finite K := Subtype.finite end Subgroup /-! ### Conversion to/from `Additive`/`Multiplicative` -/ namespace Subgroup variable (H K : Subgroup G) /-- Product of a list of elements in a subgroup is in the subgroup. -/ @[to_additive "Sum of a list of elements in an `AddSubgroup` is in the `AddSubgroup`."] protected theorem list_prod_mem {l : List G} : (∀ x ∈ l, x ∈ K) → l.prod ∈ K := list_prod_mem /-- Product of a multiset of elements in a subgroup of a `CommGroup` is in the subgroup. -/ @[to_additive "Sum of a multiset of elements in an `AddSubgroup` of an `AddCommGroup` is in the `AddSubgroup`."] protected theorem multiset_prod_mem {G} [CommGroup G] (K : Subgroup G) (g : Multiset G) : (∀ a ∈ g, a ∈ K) → g.prod ∈ K := multiset_prod_mem g @[to_additive] theorem multiset_noncommProd_mem (K : Subgroup G) (g : Multiset G) (comm) : (∀ a ∈ g, a ∈ K) → g.noncommProd comm ∈ K := K.toSubmonoid.multiset_noncommProd_mem g comm /-- Product of elements of a subgroup of a `CommGroup` indexed by a `Finset` is in the subgroup. -/ @[to_additive "Sum of elements in an `AddSubgroup` of an `AddCommGroup` indexed by a `Finset` is in the `AddSubgroup`."] protected theorem prod_mem {G : Type*} [CommGroup G] (K : Subgroup G) {ι : Type*} {t : Finset ι} {f : ι → G} (h : ∀ c ∈ t, f c ∈ K) : (∏ c ∈ t, f c) ∈ K := prod_mem h @[to_additive] theorem noncommProd_mem (K : Subgroup G) {ι : Type*} {t : Finset ι} {f : ι → G} (comm) : (∀ c ∈ t, f c ∈ K) → t.noncommProd f comm ∈ K := K.toSubmonoid.noncommProd_mem t f comm -- Porting note: increased priority to appease `simpNF`, otherwise left-hand side reduces @[to_additive (attr := simp 1100, norm_cast)] theorem val_list_prod (l : List H) : (l.prod : G) = (l.map Subtype.val).prod := SubmonoidClass.coe_list_prod l -- Porting note: increased priority to appease `simpNF`, otherwise left-hand side reduces @[to_additive (attr := simp 1100, norm_cast)] theorem val_multiset_prod {G} [CommGroup G] (H : Subgroup G) (m : Multiset H) : (m.prod : G) = (m.map Subtype.val).prod := SubmonoidClass.coe_multiset_prod m -- Porting note: increased priority to appease `simpNF`, otherwise `simp` can prove it. @[to_additive (attr := simp 1100, norm_cast)] theorem val_finset_prod {ι G} [CommGroup G] (H : Subgroup G) (f : ι → H) (s : Finset ι) : ↑(∏ i ∈ s, f i) = (∏ i ∈ s, f i : G) := SubmonoidClass.coe_finset_prod f s @[to_additive] instance fintypeBot : Fintype (⊥ : Subgroup G) := ⟨{1}, by rintro ⟨x, ⟨hx⟩⟩ exact Finset.mem_singleton_self _⟩ @[to_additive] -- Porting note: removed `simp` because `simpNF` says it can prove it. theorem card_bot : Nat.card (⊥ : Subgroup G) = 1 := Nat.card_unique @[to_additive] theorem card_top : Nat.card (⊤ : Subgroup G) = Nat.card G := Nat.card_congr Subgroup.topEquiv.toEquiv @[to_additive] theorem eq_top_of_card_eq [Finite H] (h : Nat.card H = Nat.card G) : H = ⊤ := by have : Nonempty H := ⟨1, one_mem H⟩ have h' : Nat.card H ≠ 0 := Nat.card_pos.ne' have : Finite G := (Nat.finite_of_card_ne_zero (h ▸ h')) have : Fintype G := Fintype.ofFinite G have : Fintype H := Fintype.ofFinite H rw [Nat.card_eq_fintype_card, Nat.card_eq_fintype_card] at h rw [SetLike.ext'_iff, coe_top, ← Finset.coe_univ, ← (H : Set G).coe_toFinset, Finset.coe_inj, ← Finset.card_eq_iff_eq_univ, ← h, Set.toFinset_card] congr @[to_additive (attr := simp)] theorem card_eq_iff_eq_top [Finite H] : Nat.card H = Nat.card G ↔ H = ⊤ := Iff.intro (eq_top_of_card_eq H) (fun h ↦ by simpa only [h] using card_top) @[to_additive] theorem eq_top_of_le_card [Finite G] (h : Nat.card G ≤ Nat.card H) : H = ⊤ := eq_top_of_card_eq H (le_antisymm (Nat.card_le_card_of_injective H.subtype H.subtype_injective) h) @[to_additive] theorem eq_bot_of_card_le [Finite H] (h : Nat.card H ≤ 1) : H = ⊥ := let _ := Finite.card_le_one_iff_subsingleton.mp h eq_bot_of_subsingleton H @[to_additive] theorem eq_bot_of_card_eq (h : Nat.card H = 1) : H = ⊥ := let _ := (Nat.card_eq_one_iff_unique.mp h).1 eq_bot_of_subsingleton H @[to_additive card_le_one_iff_eq_bot] theorem card_le_one_iff_eq_bot [Finite H] : Nat.card H ≤ 1 ↔ H = ⊥ := ⟨H.eq_bot_of_card_le, fun h => by simp [h]⟩ @[to_additive] lemma eq_bot_iff_card : H = ⊥ ↔ Nat.card H = 1 := ⟨by rintro rfl; exact card_bot, eq_bot_of_card_eq _⟩ @[to_additive one_lt_card_iff_ne_bot] theorem one_lt_card_iff_ne_bot [Finite H] : 1 < Nat.card H ↔ H ≠ ⊥ := lt_iff_not_le.trans H.card_le_one_iff_eq_bot.not @[to_additive] theorem card_le_card_group [Finite G] : Nat.card H ≤ Nat.card G := Nat.card_le_card_of_injective _ Subtype.coe_injective end Subgroup namespace Subgroup section Pi open Set variable {η : Type*} {f : η → Type*} [∀ i, Group (f i)] @[to_additive] theorem pi_mem_of_mulSingle_mem_aux [DecidableEq η] (I : Finset η) {H : Subgroup (∀ i, f i)} (x : ∀ i, f i) (h1 : ∀ i, i ∉ I → x i = 1) (h2 : ∀ i, i ∈ I → Pi.mulSingle i (x i) ∈ H) : x ∈ H := by induction' I using Finset.induction_on with i I hnmem ih generalizing x · convert one_mem H ext i exact h1 i (Finset.not_mem_empty i) · have : x = Function.update x i 1 * Pi.mulSingle i (x i) := by ext j by_cases heq : j = i · subst heq simp · simp [heq] rw [this] clear this apply mul_mem · apply ih <;> clear ih · intro j hj by_cases heq : j = i · subst heq simp · simp [heq] apply h1 j simpa [heq] using hj · intro j hj have : j ≠ i := by rintro rfl contradiction simp only [ne_eq, this, not_false_eq_true, Function.update_noteq] exact h2 _ (Finset.mem_insert_of_mem hj) · apply h2 simp @[to_additive] theorem pi_mem_of_mulSingle_mem [Finite η] [DecidableEq η] {H : Subgroup (∀ i, f i)} (x : ∀ i, f i) (h : ∀ i, Pi.mulSingle i (x i) ∈ H) : x ∈ H := by cases nonempty_fintype η exact pi_mem_of_mulSingle_mem_aux Finset.univ x (by simp) fun i _ => h i /-- For finite index types, the `Subgroup.pi` is generated by the embeddings of the groups. -/ @[to_additive "For finite index types, the `Subgroup.pi` is generated by the embeddings of the additive groups."] theorem pi_le_iff [DecidableEq η] [Finite η] {H : ∀ i, Subgroup (f i)} {J : Subgroup (∀ i, f i)} : pi univ H ≤ J ↔ ∀ i : η, map (MonoidHom.mulSingle f i) (H i) ≤ J := by constructor · rintro h i _ ⟨x, hx, rfl⟩ apply h simpa using hx · exact fun h x hx => pi_mem_of_mulSingle_mem x fun i => h i (mem_map_of_mem _ (hx i trivial)) end Pi end Subgroup namespace Subgroup section Normalizer theorem mem_normalizer_fintype {S : Set G} [Finite S] {x : G} (h : ∀ n, n ∈ S → x * n * x⁻¹ ∈ S) : x ∈ Subgroup.setNormalizer S := by haveI := Classical.propDecidable; cases nonempty_fintype S haveI := Set.fintypeImage S fun n => x * n * x⁻¹ exact fun n => ⟨h n, fun h₁ => have heq : (fun n => x * n * x⁻¹) '' S = S := Set.eq_of_subset_of_card_le (fun n ⟨y, hy⟩ => hy.2 ▸ h y hy.1) (by rw [Set.card_image_of_injective S conj_injective]) have : x * n * x⁻¹ ∈ (fun n => x * n * x⁻¹) '' S := heq.symm ▸ h₁ let ⟨y, hy⟩ := this conj_injective hy.2 ▸ hy.1⟩ end Normalizer end Subgroup namespace MonoidHom variable {N : Type*} [Group N] open Subgroup @[to_additive] instance decidableMemRange (f : G →* N) [Fintype G] [DecidableEq N] : DecidablePred (· ∈ f.range) := fun _ => Fintype.decidableExistsFintype -- this instance can't go just after the definition of `mrange` because `Fintype` is -- not imported at that stage /-- The range of a finite monoid under a monoid homomorphism is finite. Note: this instance can form a diamond with `Subtype.fintype` in the presence of `Fintype N`. -/ @[to_additive "The range of a finite additive monoid under an additive monoid homomorphism is finite. Note: this instance can form a diamond with `Subtype.fintype` or `Subgroup.fintype` in the presence of `Fintype N`."] instance fintypeMrange {M N : Type*} [Monoid M] [Monoid N] [Fintype M] [DecidableEq N] (f : M →* N) : Fintype (mrange f) := Set.fintypeRange f /-- The range of a finite group under a group homomorphism is finite. Note: this instance can form a diamond with `Subtype.fintype` or `Subgroup.fintype` in the presence of `Fintype N`. -/ @[to_additive "The range of a finite additive group under an additive group homomorphism is finite. Note: this instance can form a diamond with `Subtype.fintype` or `Subgroup.fintype` in the presence of `Fintype N`."] instance fintypeRange [Fintype G] [DecidableEq N] (f : G →* N) : Fintype (range f) := Set.fintypeRange f end MonoidHom
Algebra\Group\Subgroup\MulOpposite.lean
/- Copyright (c) 2022 Alex Kontorovich. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Alex Kontorovich, Eric Wieser -/ import Mathlib.Algebra.Group.Subgroup.Basic import Mathlib.Algebra.Group.Submonoid.MulOpposite import Mathlib.Logic.Encodable.Basic /-! # Mul-opposite subgroups ## Tags subgroup, subgroups -/ variable {ι : Sort*} {G : Type*} [Group G] namespace Subgroup /-- Pull a subgroup back to an opposite subgroup along `MulOpposite.unop`-/ @[to_additive (attr := simps) "Pull an additive subgroup back to an opposite additive subgroup along `AddOpposite.unop`"] protected def op (H : Subgroup G) : Subgroup Gᵐᵒᵖ where carrier := MulOpposite.unop ⁻¹' (H : Set G) one_mem' := H.one_mem mul_mem' ha hb := H.mul_mem hb ha inv_mem' := H.inv_mem @[to_additive (attr := simp)] theorem mem_op {x : Gᵐᵒᵖ} {S : Subgroup G} : x ∈ S.op ↔ x.unop ∈ S := Iff.rfl @[to_additive (attr := simp)] lemma op_toSubmonoid (H : Subgroup G) : H.op.toSubmonoid = H.toSubmonoid.op := rfl /-- Pull an opposite subgroup back to a subgroup along `MulOpposite.op`-/ @[to_additive (attr := simps) "Pull an opposite additive subgroup back to an additive subgroup along `AddOpposite.op`"] protected def unop (H : Subgroup Gᵐᵒᵖ) : Subgroup G where carrier := MulOpposite.op ⁻¹' (H : Set Gᵐᵒᵖ) one_mem' := H.one_mem mul_mem' := fun ha hb => H.mul_mem hb ha inv_mem' := H.inv_mem @[to_additive (attr := simp)] theorem mem_unop {x : G} {S : Subgroup Gᵐᵒᵖ} : x ∈ S.unop ↔ MulOpposite.op x ∈ S := Iff.rfl @[to_additive (attr := simp)] lemma unop_toSubmonoid (H : Subgroup Gᵐᵒᵖ) : H.unop.toSubmonoid = H.toSubmonoid.unop := rfl @[to_additive (attr := simp)] theorem unop_op (S : Subgroup G) : S.op.unop = S := rfl @[to_additive (attr := simp)] theorem op_unop (S : Subgroup Gᵐᵒᵖ) : S.unop.op = S := rfl /-! ### Lattice results -/ @[to_additive] theorem op_le_iff {S₁ : Subgroup G} {S₂ : Subgroup Gᵐᵒᵖ} : S₁.op ≤ S₂ ↔ S₁ ≤ S₂.unop := MulOpposite.op_surjective.forall @[to_additive] theorem le_op_iff {S₁ : Subgroup Gᵐᵒᵖ} {S₂ : Subgroup G} : S₁ ≤ S₂.op ↔ S₁.unop ≤ S₂ := MulOpposite.op_surjective.forall @[to_additive (attr := simp)] theorem op_le_op_iff {S₁ S₂ : Subgroup G} : S₁.op ≤ S₂.op ↔ S₁ ≤ S₂ := MulOpposite.op_surjective.forall @[to_additive (attr := simp)] theorem unop_le_unop_iff {S₁ S₂ : Subgroup Gᵐᵒᵖ} : S₁.unop ≤ S₂.unop ↔ S₁ ≤ S₂ := MulOpposite.unop_surjective.forall /-- A subgroup `H` of `G` determines a subgroup `H.op` of the opposite group `Gᵐᵒᵖ`. -/ @[to_additive (attr := simps) "An additive subgroup `H` of `G` determines an additive subgroup `H.op` of the opposite additive group `Gᵃᵒᵖ`."] def opEquiv : Subgroup G ≃o Subgroup Gᵐᵒᵖ where toFun := Subgroup.op invFun := Subgroup.unop left_inv := unop_op right_inv := op_unop map_rel_iff' := op_le_op_iff @[to_additive (attr := simp)] theorem op_bot : (⊥ : Subgroup G).op = ⊥ := opEquiv.map_bot @[to_additive (attr := simp)] theorem unop_bot : (⊥ : Subgroup Gᵐᵒᵖ).unop = ⊥ := opEquiv.symm.map_bot @[to_additive (attr := simp)] theorem op_top : (⊤ : Subgroup G).op = ⊤ := opEquiv.map_top @[to_additive (attr := simp)] theorem unop_top : (⊤ : Subgroup Gᵐᵒᵖ).unop = ⊤ := opEquiv.symm.map_top @[to_additive] theorem op_sup (S₁ S₂ : Subgroup G) : (S₁ ⊔ S₂).op = S₁.op ⊔ S₂.op := opEquiv.map_sup _ _ @[to_additive] theorem unop_sup (S₁ S₂ : Subgroup Gᵐᵒᵖ) : (S₁ ⊔ S₂).unop = S₁.unop ⊔ S₂.unop := opEquiv.symm.map_sup _ _ @[to_additive] theorem op_inf (S₁ S₂ : Subgroup G) : (S₁ ⊓ S₂).op = S₁.op ⊓ S₂.op := opEquiv.map_inf _ _ @[to_additive] theorem unop_inf (S₁ S₂ : Subgroup Gᵐᵒᵖ) : (S₁ ⊓ S₂).unop = S₁.unop ⊓ S₂.unop := opEquiv.symm.map_inf _ _ @[to_additive] theorem op_sSup (S : Set (Subgroup G)) : (sSup S).op = sSup (.unop ⁻¹' S) := opEquiv.map_sSup_eq_sSup_symm_preimage _ @[to_additive] theorem unop_sSup (S : Set (Subgroup Gᵐᵒᵖ)) : (sSup S).unop = sSup (.op ⁻¹' S) := opEquiv.symm.map_sSup_eq_sSup_symm_preimage _ @[to_additive] theorem op_sInf (S : Set (Subgroup G)) : (sInf S).op = sInf (.unop ⁻¹' S) := opEquiv.map_sInf_eq_sInf_symm_preimage _ @[to_additive] theorem unop_sInf (S : Set (Subgroup Gᵐᵒᵖ)) : (sInf S).unop = sInf (.op ⁻¹' S) := opEquiv.symm.map_sInf_eq_sInf_symm_preimage _ @[to_additive] theorem op_iSup (S : ι → Subgroup G) : (iSup S).op = ⨆ i, (S i).op := opEquiv.map_iSup _ @[to_additive] theorem unop_iSup (S : ι → Subgroup Gᵐᵒᵖ) : (iSup S).unop = ⨆ i, (S i).unop := opEquiv.symm.map_iSup _ @[to_additive] theorem op_iInf (S : ι → Subgroup G) : (iInf S).op = ⨅ i, (S i).op := opEquiv.map_iInf _ @[to_additive] theorem unop_iInf (S : ι → Subgroup Gᵐᵒᵖ) : (iInf S).unop = ⨅ i, (S i).unop := opEquiv.symm.map_iInf _ @[to_additive] theorem op_closure (s : Set G) : (closure s).op = closure (MulOpposite.unop ⁻¹' s) := by simp_rw [closure, op_sInf, Set.preimage_setOf_eq, Subgroup.unop_coe] congr with a exact MulOpposite.unop_surjective.forall @[to_additive] theorem unop_closure (s : Set Gᵐᵒᵖ) : (closure s).unop = closure (MulOpposite.op ⁻¹' s) := by simp_rw [closure, unop_sInf, Set.preimage_setOf_eq, Subgroup.op_coe] congr with a exact MulOpposite.op_surjective.forall /-- Bijection between a subgroup `H` and its opposite. -/ @[to_additive (attr := simps!) "Bijection between an additive subgroup `H` and its opposite."] def equivOp (H : Subgroup G) : H ≃ H.op := MulOpposite.opEquiv.subtypeEquiv fun _ => Iff.rfl @[to_additive] instance (H : Subgroup G) [Encodable H] : Encodable H.op := Encodable.ofEquiv H H.equivOp.symm @[to_additive] instance (H : Subgroup G) [Countable H] : Countable H.op := Countable.of_equiv H H.equivOp @[to_additive] theorem smul_opposite_mul {H : Subgroup G} (x g : G) (h : H.op) : h • (g * x) = g * h • x := mul_assoc _ _ _ end Subgroup
Algebra\Group\Subgroup\Order.lean
/- Copyright (c) 2021 Damiano Testa. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Damiano Testa, Ruben Van de Velde -/ import Mathlib.Order.Atoms import Mathlib.Algebra.Group.Subgroup.Basic import Mathlib.Algebra.Order.Group.InjSurj import Mathlib.Algebra.Order.Group.Unbundled.Abs /-! # Facts about ordered structures and ordered instances on subgroups -/ open Subgroup @[simp] theorem abs_mem_iff {S G} [AddGroup G] [LinearOrder G] {_ : SetLike S G} [NegMemClass S G] {H : S} {x : G} : |x| ∈ H ↔ x ∈ H := by cases abs_choice x <;> simp [*] section ModularLattice variable {C : Type*} [CommGroup C] {s t : Subgroup C} {x : C} @[to_additive] instance : IsModularLattice (Subgroup C) := ⟨fun {x} y z xz a ha => by rw [mem_inf, mem_sup] at ha rcases ha with ⟨⟨b, hb, c, hc, rfl⟩, haz⟩ rw [mem_sup] exact ⟨b, hb, c, mem_inf.2 ⟨hc, (mul_mem_cancel_left (xz hb)).1 haz⟩, rfl⟩⟩ end ModularLattice section Coatom namespace Subgroup variable {G : Type*} [Group G] (H : Subgroup G) /-- In a group that satisfies the normalizer condition, every maximal subgroup is normal -/ theorem NormalizerCondition.normal_of_coatom (hnc : NormalizerCondition G) (hmax : IsCoatom H) : H.Normal := normalizer_eq_top.mp (hmax.2 _ (hnc H (lt_top_iff_ne_top.mpr hmax.1))) @[simp] theorem isCoatom_comap {H : Type*} [Group H] (f : G ≃* H) {K : Subgroup H} : IsCoatom (Subgroup.comap (f : G →* H) K) ↔ IsCoatom K := OrderIso.isCoatom_iff (f.comapSubgroup) K @[simp] theorem isCoatom_map (f : G ≃* H) {K : Subgroup G} : IsCoatom (Subgroup.map (f : G →* H) K) ↔ IsCoatom K := OrderIso.isCoatom_iff (f.mapSubgroup) K lemma isCoatom_comap_of_surjective {H : Type*} [Group H] {φ : G →* H} (hφ : Function.Surjective φ) {M : Subgroup H} (hM : IsCoatom M) : IsCoatom (M.comap φ) := by refine And.imp (fun hM ↦ ?_) (fun hM ↦ ?_) hM · rwa [← (comap_injective hφ).ne_iff, comap_top] at hM · intro K hK specialize hM (K.map φ) rw [← comap_lt_comap_of_surjective hφ, ← (comap_injective hφ).eq_iff] at hM rw [comap_map_eq_self ((M.ker_le_comap φ).trans hK.le), comap_top] at hM exact hM hK end Subgroup end Coatom namespace SubgroupClass variable {G S : Type*} [SetLike S G] -- Prefer subclasses of `Group` over subclasses of `SubgroupClass`. /-- A subgroup of an `OrderedCommGroup` is an `OrderedCommGroup`. -/ @[to_additive "An additive subgroup of an `AddOrderedCommGroup` is an `AddOrderedCommGroup`."] instance (priority := 75) toOrderedCommGroup [OrderedCommGroup G] [SubgroupClass S G] (H : S) : OrderedCommGroup H := Subtype.coe_injective.orderedCommGroup _ rfl (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) fun _ _ => rfl -- Prefer subclasses of `Group` over subclasses of `SubgroupClass`. /-- A subgroup of a `LinearOrderedCommGroup` is a `LinearOrderedCommGroup`. -/ @[to_additive "An additive subgroup of a `LinearOrderedAddCommGroup` is a `LinearOrderedAddCommGroup`."] instance (priority := 75) toLinearOrderedCommGroup [LinearOrderedCommGroup G] [SubgroupClass S G] (H : S) : LinearOrderedCommGroup H := Subtype.coe_injective.linearOrderedCommGroup _ rfl (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) fun _ _ => rfl end SubgroupClass namespace Subgroup variable {G : Type*} /-- A subgroup of an `OrderedCommGroup` is an `OrderedCommGroup`. -/ @[to_additive "An `AddSubgroup` of an `AddOrderedCommGroup` is an `AddOrderedCommGroup`."] instance toOrderedCommGroup [OrderedCommGroup G] (H : Subgroup G) : OrderedCommGroup H := Subtype.coe_injective.orderedCommGroup _ rfl (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) fun _ _ => rfl /-- A subgroup of a `LinearOrderedCommGroup` is a `LinearOrderedCommGroup`. -/ @[to_additive "An `AddSubgroup` of a `LinearOrderedAddCommGroup` is a `LinearOrderedAddCommGroup`."] instance toLinearOrderedCommGroup [LinearOrderedCommGroup G] (H : Subgroup G) : LinearOrderedCommGroup H := Subtype.coe_injective.linearOrderedCommGroup _ rfl (fun _ _ => rfl) (fun _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) (fun _ _ => rfl) fun _ _ => rfl end Subgroup
Algebra\Group\Subgroup\Pointwise.lean
/- Copyright (c) 2021 Eric Wieser. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Eric Wieser -/ import Mathlib.Algebra.Group.Subgroup.MulOpposite import Mathlib.Algebra.Group.Submonoid.Pointwise import Mathlib.GroupTheory.GroupAction.ConjAct /-! # Pointwise instances on `Subgroup` and `AddSubgroup`s This file provides the actions * `Subgroup.pointwiseMulAction` * `AddSubgroup.pointwiseMulAction` which matches the action of `Set.mulActionSet`. These actions are available in the `Pointwise` locale. ## Implementation notes The pointwise section of this file is almost identical to the file `Mathlib.Algebra.Group.Submonoid.Pointwise`. Where possible, try to keep them in sync. -/ open Set open Pointwise variable {α G A S : Type*} @[to_additive (attr := simp, norm_cast)] theorem inv_coe_set [InvolutiveInv G] [SetLike S G] [InvMemClass S G] {H : S} : (H : Set G)⁻¹ = H := Set.ext fun _ => inv_mem_iff @[to_additive (attr := simp)] lemma smul_coe_set [Group G] [SetLike S G] [SubgroupClass S G] {s : S} {a : G} (ha : a ∈ s) : a • (s : Set G) = s := by ext; simp [Set.mem_smul_set_iff_inv_smul_mem, mul_mem_cancel_left, ha] @[to_additive (attr := simp)] lemma op_smul_coe_set [Group G] [SetLike S G] [SubgroupClass S G] {s : S} {a : G} (ha : a ∈ s) : MulOpposite.op a • (s : Set G) = s := by ext; simp [Set.mem_smul_set_iff_inv_smul_mem, mul_mem_cancel_right, ha] @[to_additive (attr := simp, norm_cast)] lemma coe_mul_coe [SetLike S G] [DivInvMonoid G] [SubgroupClass S G] (H : S) : H * H = (H : Set G) := by aesop (add simp mem_mul) @[to_additive (attr := simp, norm_cast)] lemma coe_div_coe [SetLike S G] [DivisionMonoid G] [SubgroupClass S G] (H : S) : H / H = (H : Set G) := by simp [div_eq_mul_inv] variable [Group G] [AddGroup A] {s : Set G} namespace Subgroup @[to_additive (attr := simp)] theorem inv_subset_closure (S : Set G) : S⁻¹ ⊆ closure S := fun s hs => by rw [SetLike.mem_coe, ← Subgroup.inv_mem_iff] exact subset_closure (mem_inv.mp hs) @[to_additive] theorem closure_toSubmonoid (S : Set G) : (closure S).toSubmonoid = Submonoid.closure (S ∪ S⁻¹) := by refine le_antisymm (fun x hx => ?_) (Submonoid.closure_le.2 ?_) · refine closure_induction hx (fun x hx => Submonoid.closure_mono subset_union_left (Submonoid.subset_closure hx)) (Submonoid.one_mem _) (fun x y hx hy => Submonoid.mul_mem _ hx hy) fun x hx => ?_ rwa [← Submonoid.mem_closure_inv, Set.union_inv, inv_inv, Set.union_comm] · simp only [true_and_iff, coe_toSubmonoid, union_subset_iff, subset_closure, inv_subset_closure] /-- For subgroups generated by a single element, see the simpler `zpow_induction_left`. -/ @[to_additive (attr := elab_as_elim) "For additive subgroups generated by a single element, see the simpler `zsmul_induction_left`."] theorem closure_induction_left {p : (x : G) → x ∈ closure s → Prop} (one : p 1 (one_mem _)) (mul_left : ∀ x (hx : x ∈ s), ∀ (y) hy, p y hy → p (x * y) (mul_mem (subset_closure hx) hy)) (mul_left_inv : ∀ x (hx : x ∈ s), ∀ (y) hy, p y hy → p (x⁻¹ * y) (mul_mem (inv_mem (subset_closure hx)) hy)) {x : G} (h : x ∈ closure s) : p x h := by revert h simp_rw [← mem_toSubmonoid, closure_toSubmonoid] at * intro h induction h using Submonoid.closure_induction_left with | one => exact one | mul_left x hx y hy ih => cases hx with | inl hx => exact mul_left _ hx _ hy ih | inr hx => simpa only [inv_inv] using mul_left_inv _ hx _ hy ih /-- For subgroups generated by a single element, see the simpler `zpow_induction_right`. -/ @[to_additive (attr := elab_as_elim) "For additive subgroups generated by a single element, see the simpler `zsmul_induction_right`."] theorem closure_induction_right {p : (x : G) → x ∈ closure s → Prop} (one : p 1 (one_mem _)) (mul_right : ∀ (x) hx, ∀ y (hy : y ∈ s), p x hx → p (x * y) (mul_mem hx (subset_closure hy))) (mul_right_inv : ∀ (x) hx, ∀ y (hy : y ∈ s), p x hx → p (x * y⁻¹) (mul_mem hx (inv_mem (subset_closure hy)))) {x : G} (h : x ∈ closure s) : p x h := closure_induction_left (s := MulOpposite.unop ⁻¹' s) (p := fun m hm => p m.unop <| by rwa [← op_closure] at hm) one (fun _x hx _y hy => mul_right _ _ _ hx) (fun _x hx _y hy => mul_right_inv _ _ _ hx) (by rwa [← op_closure]) @[to_additive (attr := simp)] theorem closure_inv (s : Set G) : closure s⁻¹ = closure s := by simp only [← toSubmonoid_eq, closure_toSubmonoid, inv_inv, union_comm] /-- An induction principle for closure membership. If `p` holds for `1` and all elements of `k` and their inverse, and is preserved under multiplication, then `p` holds for all elements of the closure of `k`. -/ @[to_additive (attr := elab_as_elim) "An induction principle for additive closure membership. If `p` holds for `0` and all elements of `k` and their negation, and is preserved under addition, then `p` holds for all elements of the additive closure of `k`."] theorem closure_induction'' {p : (g : G) → g ∈ closure s → Prop} (mem : ∀ x (hx : x ∈ s), p x (subset_closure hx)) (inv_mem : ∀ x (hx : x ∈ s), p x⁻¹ (inv_mem (subset_closure hx))) (one : p 1 (one_mem _)) (mul : ∀ x y hx hy, p x hx → p y hy → p (x * y) (mul_mem hx hy)) {x} (h : x ∈ closure s) : p x h := closure_induction_left one (fun x hx y _ hy => mul x y _ _ (mem x hx) hy) (fun x hx y _ => mul x⁻¹ y _ _ <| inv_mem x hx) h /-- An induction principle for elements of `⨆ i, S i`. If `C` holds for `1` and all elements of `S i` for all `i`, and is preserved under multiplication, then it holds for all elements of the supremum of `S`. -/ @[to_additive (attr := elab_as_elim) " An induction principle for elements of `⨆ i, S i`. If `C` holds for `0` and all elements of `S i` for all `i`, and is preserved under addition, then it holds for all elements of the supremum of `S`. "] theorem iSup_induction {ι : Sort*} (S : ι → Subgroup G) {C : G → Prop} {x : G} (hx : x ∈ ⨆ i, S i) (mem : ∀ (i), ∀ x ∈ S i, C x) (one : C 1) (mul : ∀ x y, C x → C y → C (x * y)) : C x := by rw [iSup_eq_closure] at hx induction hx using closure_induction'' with | one => exact one | mem x hx => obtain ⟨i, hi⟩ := Set.mem_iUnion.mp hx exact mem _ _ hi | inv_mem x hx => obtain ⟨i, hi⟩ := Set.mem_iUnion.mp hx exact mem _ _ (inv_mem hi) | mul x y _ _ ihx ihy => exact mul x y ihx ihy /-- A dependent version of `Subgroup.iSup_induction`. -/ @[to_additive (attr := elab_as_elim) "A dependent version of `AddSubgroup.iSup_induction`. "] theorem iSup_induction' {ι : Sort*} (S : ι → Subgroup G) {C : ∀ x, (x ∈ ⨆ i, S i) → Prop} (hp : ∀ (i), ∀ x (hx : x ∈ S i), C x (mem_iSup_of_mem i hx)) (h1 : C 1 (one_mem _)) (hmul : ∀ x y hx hy, C x hx → C y hy → C (x * y) (mul_mem ‹_› ‹_›)) {x : G} (hx : x ∈ ⨆ i, S i) : C x hx := by suffices ∃ h, C x h from this.snd refine iSup_induction S (C := fun x => ∃ h, C x h) hx (fun i x hx => ?_) ?_ fun x y => ?_ · exact ⟨_, hp i _ hx⟩ · exact ⟨_, h1⟩ · rintro ⟨_, Cx⟩ ⟨_, Cy⟩ exact ⟨_, hmul _ _ _ _ Cx Cy⟩ @[to_additive] theorem closure_mul_le (S T : Set G) : closure (S * T) ≤ closure S ⊔ closure T := sInf_le fun _x ⟨_s, hs, _t, ht, hx⟩ => hx ▸ (closure S ⊔ closure T).mul_mem (SetLike.le_def.mp le_sup_left <| subset_closure hs) (SetLike.le_def.mp le_sup_right <| subset_closure ht) @[to_additive] theorem sup_eq_closure_mul (H K : Subgroup G) : H ⊔ K = closure ((H : Set G) * (K : Set G)) := le_antisymm (sup_le (fun h hh => subset_closure ⟨h, hh, 1, K.one_mem, mul_one h⟩) fun k hk => subset_closure ⟨1, H.one_mem, k, hk, one_mul k⟩) ((closure_mul_le _ _).trans <| by rw [closure_eq, closure_eq]) @[to_additive] theorem set_mul_normal_comm (s : Set G) (N : Subgroup G) [hN : N.Normal] : s * (N : Set G) = (N : Set G) * s := by rw [← iUnion_mul_left_image, ← iUnion_mul_right_image] simp only [image_mul_left, image_mul_right, Set.preimage, SetLike.mem_coe, hN.mem_comm_iff] /-- The carrier of `H ⊔ N` is just `↑H * ↑N` (pointwise set product) when `N` is normal. -/ @[to_additive "The carrier of `H ⊔ N` is just `↑H + ↑N` (pointwise set addition) when `N` is normal."] theorem mul_normal (H N : Subgroup G) [hN : N.Normal] : (↑(H ⊔ N) : Set G) = H * N := by rw [sup_eq_closure_mul] refine Set.Subset.antisymm (fun x hx => ?_) subset_closure induction hx using closure_induction'' with | one => exact ⟨1, one_mem _, 1, one_mem _, mul_one 1⟩ | mem _ hx => exact hx | inv_mem x hx => obtain ⟨x, hx, y, hy, rfl⟩ := hx simpa only [mul_inv_rev, mul_assoc, inv_inv, inv_mul_cancel_left] using mul_mem_mul (inv_mem hx) (hN.conj_mem _ (inv_mem hy) x) | mul x' x' _ _ hx hx' => obtain ⟨x, hx, y, hy, rfl⟩ := hx obtain ⟨x', hx', y', hy', rfl⟩ := hx' refine ⟨x * x', mul_mem hx hx', x'⁻¹ * y * x' * y', mul_mem ?_ hy', ?_⟩ · simpa using hN.conj_mem _ hy x'⁻¹ · simp only [mul_assoc, mul_inv_cancel_left] /-- The carrier of `N ⊔ H` is just `↑N * ↑H` (pointwise set product) when `N` is normal. -/ @[to_additive "The carrier of `N ⊔ H` is just `↑N + ↑H` (pointwise set addition) when `N` is normal."] theorem normal_mul (N H : Subgroup G) [N.Normal] : (↑(N ⊔ H) : Set G) = N * H := by rw [← set_mul_normal_comm, sup_comm, mul_normal] @[to_additive] theorem mul_inf_assoc (A B C : Subgroup G) (h : A ≤ C) : (A : Set G) * ↑(B ⊓ C) = (A : Set G) * (B : Set G) ∩ C := by ext simp only [coe_inf, Set.mem_mul, Set.mem_inter_iff] constructor · rintro ⟨y, hy, z, ⟨hzB, hzC⟩, rfl⟩ refine ⟨?_, mul_mem (h hy) hzC⟩ exact ⟨y, hy, z, hzB, rfl⟩ rintro ⟨⟨y, hy, z, hz, rfl⟩, hyz⟩ refine ⟨y, hy, z, ⟨hz, ?_⟩, rfl⟩ suffices y⁻¹ * (y * z) ∈ C by simpa exact mul_mem (inv_mem (h hy)) hyz @[to_additive] theorem inf_mul_assoc (A B C : Subgroup G) (h : C ≤ A) : ((A ⊓ B : Subgroup G) : Set G) * C = (A : Set G) ∩ (↑B * ↑C) := by ext simp only [coe_inf, Set.mem_mul, Set.mem_inter_iff] constructor · rintro ⟨y, ⟨hyA, hyB⟩, z, hz, rfl⟩ refine ⟨A.mul_mem hyA (h hz), ?_⟩ exact ⟨y, hyB, z, hz, rfl⟩ rintro ⟨hyz, y, hy, z, hz, rfl⟩ refine ⟨y, ⟨?_, hy⟩, z, hz, rfl⟩ suffices y * z * z⁻¹ ∈ A by simpa exact mul_mem hyz (inv_mem (h hz)) @[to_additive] instance sup_normal (H K : Subgroup G) [hH : H.Normal] [hK : K.Normal] : (H ⊔ K).Normal where conj_mem n hmem g := by rw [← SetLike.mem_coe, normal_mul] at hmem ⊢ rcases hmem with ⟨h, hh, k, hk, rfl⟩ refine ⟨g * h * g⁻¹, hH.conj_mem h hh g, g * k * g⁻¹, hK.conj_mem k hk g, ?_⟩ simp only [mul_assoc, inv_mul_cancel_left] @[to_additive] theorem smul_opposite_image_mul_preimage' (g : G) (h : Gᵐᵒᵖ) (s : Set G) : (fun y => h • y) '' ((g * ·) ⁻¹' s) = (g * ·) ⁻¹' ((fun y => h • y) '' s) := by simp [preimage_preimage, mul_assoc] -- Porting note: deprecate? @[to_additive] theorem smul_opposite_image_mul_preimage {H : Subgroup G} (g : G) (h : H.op) (s : Set G) : (fun y => h • y) '' ((g * ·) ⁻¹' s) = (g * ·) ⁻¹' ((fun y => h • y) '' s) := smul_opposite_image_mul_preimage' g h s /-! ### Pointwise action -/ section Monoid variable [Monoid α] [MulDistribMulAction α G] /-- The action on a subgroup corresponding to applying the action to every element. This is available as an instance in the `Pointwise` locale. -/ protected def pointwiseMulAction : MulAction α (Subgroup G) where smul a S := S.map (MulDistribMulAction.toMonoidEnd _ _ a) one_smul S := by change S.map _ = S simpa only [map_one] using S.map_id mul_smul a₁ a₂ S := (congr_arg (fun f : Monoid.End G => S.map f) (MonoidHom.map_mul _ _ _)).trans (S.map_map _ _).symm scoped[Pointwise] attribute [instance] Subgroup.pointwiseMulAction theorem pointwise_smul_def {a : α} (S : Subgroup G) : a • S = S.map (MulDistribMulAction.toMonoidEnd _ _ a) := rfl @[simp] theorem coe_pointwise_smul (a : α) (S : Subgroup G) : ↑(a • S) = a • (S : Set G) := rfl @[simp] theorem pointwise_smul_toSubmonoid (a : α) (S : Subgroup G) : (a • S).toSubmonoid = a • S.toSubmonoid := rfl theorem smul_mem_pointwise_smul (m : G) (a : α) (S : Subgroup G) : m ∈ S → a • m ∈ a • S := (Set.smul_mem_smul_set : _ → _ ∈ a • (S : Set G)) instance : CovariantClass α (Subgroup G) HSMul.hSMul LE.le := ⟨fun _ _ => image_subset _⟩ theorem mem_smul_pointwise_iff_exists (m : G) (a : α) (S : Subgroup G) : m ∈ a • S ↔ ∃ s : G, s ∈ S ∧ a • s = m := (Set.mem_smul_set : m ∈ a • (S : Set G) ↔ _) @[simp] theorem smul_bot (a : α) : a • (⊥ : Subgroup G) = ⊥ := map_bot _ theorem smul_sup (a : α) (S T : Subgroup G) : a • (S ⊔ T) = a • S ⊔ a • T := map_sup _ _ _ theorem smul_closure (a : α) (s : Set G) : a • closure s = closure (a • s) := MonoidHom.map_closure _ _ instance pointwise_isCentralScalar [MulDistribMulAction αᵐᵒᵖ G] [IsCentralScalar α G] : IsCentralScalar α (Subgroup G) := ⟨fun _ S => (congr_arg fun f => S.map f) <| MonoidHom.ext <| op_smul_eq_smul _⟩ theorem conj_smul_le_of_le {P H : Subgroup G} (hP : P ≤ H) (h : H) : MulAut.conj (h : G) • P ≤ H := by rintro - ⟨g, hg, rfl⟩ exact H.mul_mem (H.mul_mem h.2 (hP hg)) (H.inv_mem h.2) theorem conj_smul_subgroupOf {P H : Subgroup G} (hP : P ≤ H) (h : H) : MulAut.conj h • P.subgroupOf H = (MulAut.conj (h : G) • P).subgroupOf H := by refine le_antisymm ?_ ?_ · rintro - ⟨g, hg, rfl⟩ exact ⟨g, hg, rfl⟩ · rintro p ⟨g, hg, hp⟩ exact ⟨⟨g, hP hg⟩, hg, Subtype.ext hp⟩ end Monoid section Group variable [Group α] [MulDistribMulAction α G] @[simp] theorem smul_mem_pointwise_smul_iff {a : α} {S : Subgroup G} {x : G} : a • x ∈ a • S ↔ x ∈ S := smul_mem_smul_set_iff theorem mem_pointwise_smul_iff_inv_smul_mem {a : α} {S : Subgroup G} {x : G} : x ∈ a • S ↔ a⁻¹ • x ∈ S := mem_smul_set_iff_inv_smul_mem theorem mem_inv_pointwise_smul_iff {a : α} {S : Subgroup G} {x : G} : x ∈ a⁻¹ • S ↔ a • x ∈ S := mem_inv_smul_set_iff @[simp] theorem pointwise_smul_le_pointwise_smul_iff {a : α} {S T : Subgroup G} : a • S ≤ a • T ↔ S ≤ T := set_smul_subset_set_smul_iff theorem pointwise_smul_subset_iff {a : α} {S T : Subgroup G} : a • S ≤ T ↔ S ≤ a⁻¹ • T := set_smul_subset_iff theorem subset_pointwise_smul_iff {a : α} {S T : Subgroup G} : S ≤ a • T ↔ a⁻¹ • S ≤ T := subset_set_smul_iff @[simp] theorem smul_inf (a : α) (S T : Subgroup G) : a • (S ⊓ T) = a • S ⊓ a • T := by simp [SetLike.ext_iff, mem_pointwise_smul_iff_inv_smul_mem] /-- Applying a `MulDistribMulAction` results in an isomorphic subgroup -/ @[simps!] def equivSMul (a : α) (H : Subgroup G) : H ≃* (a • H : Subgroup G) := (MulDistribMulAction.toMulEquiv G a).subgroupMap H theorem subgroup_mul_singleton {H : Subgroup G} {h : G} (hh : h ∈ H) : (H : Set G) * {h} = H := suffices { x : G | x ∈ H } = ↑H by simpa [preimage, mul_mem_cancel_right (inv_mem hh)] rfl theorem singleton_mul_subgroup {H : Subgroup G} {h : G} (hh : h ∈ H) : {h} * (H : Set G) = H := suffices { x : G | x ∈ H } = ↑H by simpa [preimage, mul_mem_cancel_left (inv_mem hh)] rfl theorem Normal.conjAct {G : Type*} [Group G] {H : Subgroup G} (hH : H.Normal) (g : ConjAct G) : g • H = H := have : ∀ g : ConjAct G, g • H ≤ H := fun _ => map_le_iff_le_comap.2 fun _ h => hH.conj_mem _ h _ (this g).antisymm <| (smul_inv_smul g H).symm.trans_le (map_mono <| this _) @[simp] theorem smul_normal (g : G) (H : Subgroup G) [h : Normal H] : MulAut.conj g • H = H := h.conjAct g end Group section GroupWithZero variable [GroupWithZero α] [MulDistribMulAction α G] @[simp] theorem smul_mem_pointwise_smul_iff₀ {a : α} (ha : a ≠ 0) (S : Subgroup G) (x : G) : a • x ∈ a • S ↔ x ∈ S := smul_mem_smul_set_iff₀ ha (S : Set G) x theorem mem_pointwise_smul_iff_inv_smul_mem₀ {a : α} (ha : a ≠ 0) (S : Subgroup G) (x : G) : x ∈ a • S ↔ a⁻¹ • x ∈ S := mem_smul_set_iff_inv_smul_mem₀ ha (S : Set G) x theorem mem_inv_pointwise_smul_iff₀ {a : α} (ha : a ≠ 0) (S : Subgroup G) (x : G) : x ∈ a⁻¹ • S ↔ a • x ∈ S := mem_inv_smul_set_iff₀ ha (S : Set G) x @[simp] theorem pointwise_smul_le_pointwise_smul_iff₀ {a : α} (ha : a ≠ 0) {S T : Subgroup G} : a • S ≤ a • T ↔ S ≤ T := set_smul_subset_set_smul_iff₀ ha theorem pointwise_smul_le_iff₀ {a : α} (ha : a ≠ 0) {S T : Subgroup G} : a • S ≤ T ↔ S ≤ a⁻¹ • T := set_smul_subset_iff₀ ha theorem le_pointwise_smul_iff₀ {a : α} (ha : a ≠ 0) {S T : Subgroup G} : S ≤ a • T ↔ a⁻¹ • S ≤ T := subset_set_smul_iff₀ ha end GroupWithZero end Subgroup namespace AddSubgroup section Monoid variable [Monoid α] [DistribMulAction α A] /-- The action on an additive subgroup corresponding to applying the action to every element. This is available as an instance in the `Pointwise` locale. -/ protected def pointwiseMulAction : MulAction α (AddSubgroup A) where smul a S := S.map (DistribMulAction.toAddMonoidEnd _ _ a) one_smul S := by change S.map _ = S simpa only [map_one] using S.map_id mul_smul _ _ S := (congr_arg (fun f : AddMonoid.End A => S.map f) (MonoidHom.map_mul _ _ _)).trans (S.map_map _ _).symm scoped[Pointwise] attribute [instance] AddSubgroup.pointwiseMulAction theorem pointwise_smul_def {a : α} (S : AddSubgroup A) : a • S = S.map (DistribMulAction.toAddMonoidEnd _ _ a) := rfl @[simp] theorem coe_pointwise_smul (a : α) (S : AddSubgroup A) : ↑(a • S) = a • (S : Set A) := rfl @[simp] theorem pointwise_smul_toAddSubmonoid (a : α) (S : AddSubgroup A) : (a • S).toAddSubmonoid = a • S.toAddSubmonoid := rfl theorem smul_mem_pointwise_smul (m : A) (a : α) (S : AddSubgroup A) : m ∈ S → a • m ∈ a • S := (Set.smul_mem_smul_set : _ → _ ∈ a • (S : Set A)) theorem mem_smul_pointwise_iff_exists (m : A) (a : α) (S : AddSubgroup A) : m ∈ a • S ↔ ∃ s : A, s ∈ S ∧ a • s = m := (Set.mem_smul_set : m ∈ a • (S : Set A) ↔ _) instance pointwise_isCentralScalar [DistribMulAction αᵐᵒᵖ A] [IsCentralScalar α A] : IsCentralScalar α (AddSubgroup A) := ⟨fun _ S => (congr_arg fun f => S.map f) <| AddMonoidHom.ext <| op_smul_eq_smul _⟩ end Monoid section Group variable [Group α] [DistribMulAction α A] open Pointwise @[simp] theorem smul_mem_pointwise_smul_iff {a : α} {S : AddSubgroup A} {x : A} : a • x ∈ a • S ↔ x ∈ S := smul_mem_smul_set_iff theorem mem_pointwise_smul_iff_inv_smul_mem {a : α} {S : AddSubgroup A} {x : A} : x ∈ a • S ↔ a⁻¹ • x ∈ S := mem_smul_set_iff_inv_smul_mem theorem mem_inv_pointwise_smul_iff {a : α} {S : AddSubgroup A} {x : A} : x ∈ a⁻¹ • S ↔ a • x ∈ S := mem_inv_smul_set_iff @[simp] theorem pointwise_smul_le_pointwise_smul_iff {a : α} {S T : AddSubgroup A} : a • S ≤ a • T ↔ S ≤ T := set_smul_subset_set_smul_iff theorem pointwise_smul_le_iff {a : α} {S T : AddSubgroup A} : a • S ≤ T ↔ S ≤ a⁻¹ • T := set_smul_subset_iff theorem le_pointwise_smul_iff {a : α} {S T : AddSubgroup A} : S ≤ a • T ↔ a⁻¹ • S ≤ T := subset_set_smul_iff end Group section GroupWithZero variable [GroupWithZero α] [DistribMulAction α A] open Pointwise @[simp] theorem smul_mem_pointwise_smul_iff₀ {a : α} (ha : a ≠ 0) (S : AddSubgroup A) (x : A) : a • x ∈ a • S ↔ x ∈ S := smul_mem_smul_set_iff₀ ha (S : Set A) x theorem mem_pointwise_smul_iff_inv_smul_mem₀ {a : α} (ha : a ≠ 0) (S : AddSubgroup A) (x : A) : x ∈ a • S ↔ a⁻¹ • x ∈ S := mem_smul_set_iff_inv_smul_mem₀ ha (S : Set A) x theorem mem_inv_pointwise_smul_iff₀ {a : α} (ha : a ≠ 0) (S : AddSubgroup A) (x : A) : x ∈ a⁻¹ • S ↔ a • x ∈ S := mem_inv_smul_set_iff₀ ha (S : Set A) x @[simp] theorem pointwise_smul_le_pointwise_smul_iff₀ {a : α} (ha : a ≠ 0) {S T : AddSubgroup A} : a • S ≤ a • T ↔ S ≤ T := set_smul_subset_set_smul_iff₀ ha theorem pointwise_smul_le_iff₀ {a : α} (ha : a ≠ 0) {S T : AddSubgroup A} : a • S ≤ T ↔ S ≤ a⁻¹ • T := set_smul_subset_iff₀ ha theorem le_pointwise_smul_iff₀ {a : α} (ha : a ≠ 0) {S T : AddSubgroup A} : S ≤ a • T ↔ a⁻¹ • S ≤ T := subset_set_smul_iff₀ ha end GroupWithZero end AddSubgroup
Algebra\Group\Subgroup\ZPowers.lean
/- Copyright (c) 2020 Chris Hughes. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Chris Hughes -/ import Mathlib.Algebra.Group.Subgroup.Basic import Mathlib.Data.Countable.Basic import Mathlib.Data.Set.Image import Mathlib.Data.Set.Subsingleton import Mathlib.Data.Int.Cast.Lemmas import Mathlib.GroupTheory.Subgroup.Centralizer /-! # Subgroups generated by an element ## Tags subgroup, subgroups -/ variable {G : Type*} [Group G] variable {A : Type*} [AddGroup A] variable {N : Type*} [Group N] namespace Subgroup /-- The subgroup generated by an element. -/ def zpowers (g : G) : Subgroup G := Subgroup.copy (zpowersHom G g).range (Set.range (g ^ · : ℤ → G)) rfl theorem mem_zpowers (g : G) : g ∈ zpowers g := ⟨1, zpow_one _⟩ theorem coe_zpowers (g : G) : ↑(zpowers g) = Set.range (g ^ · : ℤ → G) := rfl noncomputable instance decidableMemZPowers {a : G} : DecidablePred (· ∈ Subgroup.zpowers a) := Classical.decPred _ theorem zpowers_eq_closure (g : G) : zpowers g = closure {g} := by ext exact mem_closure_singleton.symm theorem range_zpowersHom (g : G) : (zpowersHom G g).range = zpowers g := rfl theorem mem_zpowers_iff {g h : G} : h ∈ zpowers g ↔ ∃ k : ℤ, g ^ k = h := Iff.rfl theorem zpow_mem_zpowers (g : G) (k : ℤ) : g ^ k ∈ zpowers g := mem_zpowers_iff.mpr ⟨k, rfl⟩ theorem npow_mem_zpowers (g : G) (k : ℕ) : g ^ k ∈ zpowers g := zpow_natCast g k ▸ zpow_mem_zpowers g k theorem forall_zpowers {x : G} {p : zpowers x → Prop} : (∀ g, p g) ↔ ∀ m : ℤ, p ⟨x ^ m, m, rfl⟩ := Set.forall_subtype_range_iff theorem exists_zpowers {x : G} {p : zpowers x → Prop} : (∃ g, p g) ↔ ∃ m : ℤ, p ⟨x ^ m, m, rfl⟩ := Set.exists_subtype_range_iff theorem forall_mem_zpowers {x : G} {p : G → Prop} : (∀ g ∈ zpowers x, p g) ↔ ∀ m : ℤ, p (x ^ m) := Set.forall_mem_range theorem exists_mem_zpowers {x : G} {p : G → Prop} : (∃ g ∈ zpowers x, p g) ↔ ∃ m : ℤ, p (x ^ m) := Set.exists_range_iff instance (a : G) : Countable (zpowers a) := ((zpowersHom G a).rangeRestrict_surjective.comp Multiplicative.ofAdd.surjective).countable end Subgroup namespace AddSubgroup /-- The subgroup generated by an element. -/ def zmultiples (a : A) : AddSubgroup A := AddSubgroup.copy (zmultiplesHom A a).range (Set.range ((· • a) : ℤ → A)) rfl @[simp] theorem range_zmultiplesHom (a : A) : (zmultiplesHom A a).range = zmultiples a := rfl attribute [to_additive existing] Subgroup.zpowers attribute [to_additive (attr := simp)] Subgroup.mem_zpowers attribute [to_additive (attr := norm_cast)] Subgroup.coe_zpowers attribute [to_additive] Subgroup.decidableMemZPowers attribute [to_additive] Subgroup.zpowers_eq_closure attribute [to_additive existing (attr := simp)] Subgroup.range_zpowersHom attribute [to_additive] Subgroup.mem_zpowers_iff attribute [to_additive (attr := simp)] Subgroup.zpow_mem_zpowers attribute [to_additive (attr := simp)] Subgroup.npow_mem_zpowers -- Porting note: increasing simp priority. Better lemma than `Subtype.forall` attribute [to_additive (attr := simp 1100)] Subgroup.forall_zpowers attribute [to_additive] Subgroup.forall_mem_zpowers -- Porting note: increasing simp priority. Better lemma than `Subtype.exists` attribute [to_additive (attr := simp 1100)] Subgroup.exists_zpowers attribute [to_additive] Subgroup.exists_mem_zpowers instance (a : A) : Countable (zmultiples a) := (zmultiplesHom A a).rangeRestrict_surjective.countable section Ring variable {R : Type*} [Ring R] (r : R) (k : ℤ) @[simp] theorem intCast_mul_mem_zmultiples : ↑(k : ℤ) * r ∈ zmultiples r := by simpa only [← zsmul_eq_mul] using zsmul_mem_zmultiples r k @[deprecated (since := "2024-04-17")] alias int_cast_mul_mem_zmultiples := intCast_mul_mem_zmultiples @[simp] theorem intCast_mem_zmultiples_one : ↑(k : ℤ) ∈ zmultiples (1 : R) := mem_zmultiples_iff.mp ⟨k, by simp⟩ @[deprecated (since := "2024-04-17")] alias int_cast_mem_zmultiples_one := intCast_mem_zmultiples_one end Ring end AddSubgroup @[simp] lemma Int.range_castAddHom {A : Type*} [AddGroupWithOne A] : (Int.castAddHom A).range = AddSubgroup.zmultiples 1 := by ext a simp_rw [AddMonoidHom.mem_range, Int.coe_castAddHom, AddSubgroup.mem_zmultiples_iff, zsmul_one] @[to_additive (attr := simp)] theorem MonoidHom.map_zpowers (f : G →* N) (x : G) : (Subgroup.zpowers x).map f = Subgroup.zpowers (f x) := by rw [Subgroup.zpowers_eq_closure, Subgroup.zpowers_eq_closure, f.map_closure, Set.image_singleton] theorem Int.mem_zmultiples_iff {a b : ℤ} : b ∈ AddSubgroup.zmultiples a ↔ a ∣ b := exists_congr fun k => by rw [mul_comm, eq_comm, ← smul_eq_mul] @[simp] lemma Int.zmultiples_one : AddSubgroup.zmultiples (1 : ℤ) = ⊤ := by ext z simpa only [AddSubgroup.mem_top, iff_true] using ⟨z, zsmul_int_one z⟩ theorem ofMul_image_zpowers_eq_zmultiples_ofMul {x : G} : Additive.ofMul '' (Subgroup.zpowers x : Set G) = AddSubgroup.zmultiples (Additive.ofMul x) := by ext y constructor · rintro ⟨z, ⟨m, hm⟩, hz2⟩ use m simp only at * rwa [← ofMul_zpow, hm] · rintro ⟨n, hn⟩ refine ⟨x ^ n, ⟨n, rfl⟩, ?_⟩ rwa [ofMul_zpow] theorem ofAdd_image_zmultiples_eq_zpowers_ofAdd {x : A} : Multiplicative.ofAdd '' (AddSubgroup.zmultiples x : Set A) = Subgroup.zpowers (Multiplicative.ofAdd x) := by symm rw [Equiv.eq_image_iff_symm_image_eq] exact ofMul_image_zpowers_eq_zmultiples_ofMul namespace Subgroup variable {s : Set G} {g : G} @[to_additive] instance zpowers_isCommutative (g : G) : (zpowers g).IsCommutative := ⟨⟨fun ⟨_, _, h₁⟩ ⟨_, _, h₂⟩ => by rw [Subtype.ext_iff, coe_mul, coe_mul, Subtype.coe_mk, Subtype.coe_mk, ← h₁, ← h₂, zpow_mul_comm]⟩⟩ @[to_additive (attr := simp)] theorem zpowers_le {g : G} {H : Subgroup G} : zpowers g ≤ H ↔ g ∈ H := by rw [zpowers_eq_closure, closure_le, Set.singleton_subset_iff, SetLike.mem_coe] alias ⟨_, zpowers_le_of_mem⟩ := zpowers_le alias ⟨_, _root_.AddSubgroup.zmultiples_le_of_mem⟩ := AddSubgroup.zmultiples_le attribute [to_additive existing] zpowers_le_of_mem @[to_additive (attr := simp)] theorem zpowers_eq_bot {g : G} : zpowers g = ⊥ ↔ g = 1 := by rw [eq_bot_iff, zpowers_le, mem_bot] @[to_additive] theorem zpowers_ne_bot : zpowers g ≠ ⊥ ↔ g ≠ 1 := zpowers_eq_bot.not @[to_additive (attr := simp)] theorem zpowers_one_eq_bot : Subgroup.zpowers (1 : G) = ⊥ := Subgroup.zpowers_eq_bot.mpr rfl @[to_additive (attr := simp)] theorem zpowers_inv : zpowers g⁻¹ = zpowers g := eq_of_forall_ge_iff fun _ ↦ by simp only [zpowers_le, inv_mem_iff] @[to_additive] theorem centralizer_closure (S : Set G) : centralizer (closure S : Set G) = ⨅ g ∈ S, centralizer (zpowers g : Set G) := le_antisymm (le_iInf fun _ => le_iInf fun hg => centralizer_le <| zpowers_le.2 <| subset_closure hg) <| le_centralizer_iff.1 <| (closure_le _).2 fun g => SetLike.mem_coe.2 ∘ zpowers_le.1 ∘ le_centralizer_iff.1 ∘ iInf_le_of_le g ∘ iInf_le _ @[to_additive] theorem center_eq_iInf (S : Set G) (hS : closure S = ⊤) : center G = ⨅ g ∈ S, centralizer (zpowers g) := by rw [← centralizer_univ, ← coe_top, ← hS, centralizer_closure] @[to_additive] theorem center_eq_infi' (S : Set G) (hS : closure S = ⊤) : center G = ⨅ g : S, centralizer (zpowers (g : G)) := by rw [center_eq_iInf S hS, ← iInf_subtype''] end Subgroup
Algebra\Group\Submonoid\Basic.lean
/- Copyright (c) 2018 Johannes Hölzl. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Johannes Hölzl, Kenny Lau, Johan Commelin, Mario Carneiro, Kevin Buzzard, Amelia Livingston, Yury Kudryashov -/ import Mathlib.Algebra.Group.Hom.Defs import Mathlib.Algebra.Group.Subsemigroup.Basic import Mathlib.Algebra.Group.Units /-! # Submonoids: definition and `CompleteLattice` structure This file defines bundled multiplicative and additive submonoids. We also define a `CompleteLattice` structure on `Submonoid`s, define the closure of a set as the minimal submonoid that includes this set, and prove a few results about extending properties from a dense set (i.e. a set with `closure s = ⊤`) to the whole monoid, see `Submonoid.dense_induction` and `MonoidHom.ofClosureEqTopLeft`/`MonoidHom.ofClosureEqTopRight`. ## Main definitions * `Submonoid M`: the type of bundled submonoids of a monoid `M`; the underlying set is given in the `carrier` field of the structure, and should be accessed through coercion as in `(S : Set M)`. * `AddSubmonoid M` : the type of bundled submonoids of an additive monoid `M`. For each of the following definitions in the `Submonoid` namespace, there is a corresponding definition in the `AddSubmonoid` namespace. * `Submonoid.copy` : copy of a submonoid with `carrier` replaced by a set that is equal but possibly not definitionally equal to the carrier of the original `Submonoid`. * `Submonoid.closure` : monoid closure of a set, i.e., the least submonoid that includes the set. * `Submonoid.gi` : `closure : Set M → Submonoid M` and coercion `coe : Submonoid M → Set M` form a `GaloisInsertion`; * `MonoidHom.eqLocus`: the submonoid of elements `x : M` such that `f x = g x`; * `MonoidHom.ofClosureEqTopRight`: if a map `f : M → N` between two monoids satisfies `f 1 = 1` and `f (x * y) = f x * f y` for `y` from some dense set `s`, then `f` is a monoid homomorphism. E.g., if `f : ℕ → M` satisfies `f 0 = 0` and `f (x + 1) = f x + f 1`, then `f` is an additive monoid homomorphism. ## Implementation notes Submonoid inclusion is denoted `≤` rather than `⊆`, although `∈` is defined as membership of a submonoid's underlying set. Note that `Submonoid M` does not actually require `Monoid M`, instead requiring only the weaker `MulOneClass M`. This file is designed to have very few dependencies. In particular, it should not use natural numbers. `Submonoid` is implemented by extending `Subsemigroup` requiring `one_mem'`. ## Tags submonoid, submonoids -/ assert_not_exists MonoidWithZero -- Only needed for notation -- Only needed for notation variable {M : Type*} {N : Type*} variable {A : Type*} section NonAssoc variable [MulOneClass M] {s : Set M} variable [AddZeroClass A] {t : Set A} /-- `OneMemClass S M` says `S` is a type of subsets `s ≤ M`, such that `1 ∈ s` for all `s`. -/ class OneMemClass (S : Type*) (M : Type*) [One M] [SetLike S M] : Prop where /-- By definition, if we have `OneMemClass S M`, we have `1 ∈ s` for all `s : S`. -/ one_mem : ∀ s : S, (1 : M) ∈ s export OneMemClass (one_mem) /-- `ZeroMemClass S M` says `S` is a type of subsets `s ≤ M`, such that `0 ∈ s` for all `s`. -/ class ZeroMemClass (S : Type*) (M : Type*) [Zero M] [SetLike S M] : Prop where /-- By definition, if we have `ZeroMemClass S M`, we have `0 ∈ s` for all `s : S`. -/ zero_mem : ∀ s : S, (0 : M) ∈ s export ZeroMemClass (zero_mem) attribute [to_additive] OneMemClass attribute [aesop safe apply (rule_sets := [SetLike])] one_mem zero_mem section /-- A submonoid of a monoid `M` is a subset containing 1 and closed under multiplication. -/ structure Submonoid (M : Type*) [MulOneClass M] extends Subsemigroup M where /-- A submonoid contains `1`. -/ one_mem' : (1 : M) ∈ carrier end /-- A submonoid of a monoid `M` can be considered as a subsemigroup of that monoid. -/ add_decl_doc Submonoid.toSubsemigroup /-- `SubmonoidClass S M` says `S` is a type of subsets `s ≤ M` that contain `1` and are closed under `(*)` -/ class SubmonoidClass (S : Type*) (M : Type*) [MulOneClass M] [SetLike S M] extends MulMemClass S M, OneMemClass S M : Prop section /-- An additive submonoid of an additive monoid `M` is a subset containing 0 and closed under addition. -/ structure AddSubmonoid (M : Type*) [AddZeroClass M] extends AddSubsemigroup M where /-- An additive submonoid contains `0`. -/ zero_mem' : (0 : M) ∈ carrier end /-- An additive submonoid of an additive monoid `M` can be considered as an additive subsemigroup of that additive monoid. -/ add_decl_doc AddSubmonoid.toAddSubsemigroup /-- `AddSubmonoidClass S M` says `S` is a type of subsets `s ≤ M` that contain `0` and are closed under `(+)` -/ class AddSubmonoidClass (S : Type*) (M : Type*) [AddZeroClass M] [SetLike S M] extends AddMemClass S M, ZeroMemClass S M : Prop attribute [to_additive] Submonoid SubmonoidClass @[to_additive (attr := aesop safe apply (rule_sets := [SetLike]))] theorem pow_mem {M A} [Monoid M] [SetLike A M] [SubmonoidClass A M] {S : A} {x : M} (hx : x ∈ S) : ∀ n : ℕ, x ^ n ∈ S | 0 => by rw [pow_zero] exact OneMemClass.one_mem S | n + 1 => by rw [pow_succ] exact mul_mem (pow_mem hx n) hx namespace Submonoid @[to_additive] instance : SetLike (Submonoid M) M where coe s := s.carrier coe_injective' p q h := by cases p; cases q; congr; exact SetLike.coe_injective' h @[to_additive] instance : SubmonoidClass (Submonoid M) M where one_mem := Submonoid.one_mem' mul_mem {s} := s.mul_mem' initialize_simps_projections Submonoid (carrier → coe) initialize_simps_projections AddSubmonoid (carrier → coe) @[to_additive (attr := simp)] theorem mem_toSubsemigroup {s : Submonoid M} {x : M} : x ∈ s.toSubsemigroup ↔ x ∈ s := Iff.rfl -- Porting note: `x ∈ s.carrier` is now syntactically `x ∈ s.toSubsemigroup.carrier`, -- which `simp` already simplifies to `x ∈ s.toSubsemigroup`. So we remove the `@[simp]` attribute -- here, and instead add the simp lemma `mem_toSubsemigroup` to allow `simp` to do this exact -- simplification transitively. @[to_additive] theorem mem_carrier {s : Submonoid M} {x : M} : x ∈ s.carrier ↔ x ∈ s := Iff.rfl @[to_additive (attr := simp)] theorem mem_mk {s : Subsemigroup M} {x : M} (h_one) : x ∈ mk s h_one ↔ x ∈ s := Iff.rfl @[to_additive (attr := simp)] theorem coe_set_mk {s : Subsemigroup M} (h_one) : (mk s h_one : Set M) = s := rfl @[to_additive (attr := simp)] theorem mk_le_mk {s t : Subsemigroup M} (h_one) (h_one') : mk s h_one ≤ mk t h_one' ↔ s ≤ t := Iff.rfl /-- Two submonoids are equal if they have the same elements. -/ @[to_additive (attr := ext) "Two `AddSubmonoid`s are equal if they have the same elements."] theorem ext {S T : Submonoid M} (h : ∀ x, x ∈ S ↔ x ∈ T) : S = T := SetLike.ext h /-- Copy a submonoid replacing `carrier` with a set that is equal to it. -/ @[to_additive "Copy an additive submonoid replacing `carrier` with a set that is equal to it."] protected def copy (S : Submonoid M) (s : Set M) (hs : s = S) : Submonoid M where carrier := s one_mem' := show 1 ∈ s from hs.symm ▸ S.one_mem' mul_mem' := hs.symm ▸ S.mul_mem' variable {S : Submonoid M} @[to_additive (attr := simp)] theorem coe_copy {s : Set M} (hs : s = S) : (S.copy s hs : Set M) = s := rfl @[to_additive] theorem copy_eq {s : Set M} (hs : s = S) : S.copy s hs = S := SetLike.coe_injective hs variable (S) /-- A submonoid contains the monoid's 1. -/ @[to_additive "An `AddSubmonoid` contains the monoid's 0."] protected theorem one_mem : (1 : M) ∈ S := one_mem S /-- A submonoid is closed under multiplication. -/ @[to_additive "An `AddSubmonoid` is closed under addition."] protected theorem mul_mem {x y : M} : x ∈ S → y ∈ S → x * y ∈ S := mul_mem /-- The submonoid `M` of the monoid `M`. -/ @[to_additive "The additive submonoid `M` of the `AddMonoid M`."] instance : Top (Submonoid M) := ⟨{ carrier := Set.univ one_mem' := Set.mem_univ 1 mul_mem' := fun _ _ => Set.mem_univ _ }⟩ /-- The trivial submonoid `{1}` of a monoid `M`. -/ @[to_additive "The trivial `AddSubmonoid` `{0}` of an `AddMonoid` `M`."] instance : Bot (Submonoid M) := ⟨{ carrier := {1} one_mem' := Set.mem_singleton 1 mul_mem' := fun ha hb => by simp only [Set.mem_singleton_iff] at * rw [ha, hb, mul_one] }⟩ @[to_additive] instance : Inhabited (Submonoid M) := ⟨⊥⟩ @[to_additive (attr := simp)] theorem mem_bot {x : M} : x ∈ (⊥ : Submonoid M) ↔ x = 1 := Set.mem_singleton_iff @[to_additive (attr := simp)] theorem mem_top (x : M) : x ∈ (⊤ : Submonoid M) := Set.mem_univ x @[to_additive (attr := simp)] theorem coe_top : ((⊤ : Submonoid M) : Set M) = Set.univ := rfl @[to_additive (attr := simp)] theorem coe_bot : ((⊥ : Submonoid M) : Set M) = {1} := rfl /-- The inf of two submonoids is their intersection. -/ @[to_additive "The inf of two `AddSubmonoid`s is their intersection."] instance : Inf (Submonoid M) := ⟨fun S₁ S₂ => { carrier := S₁ ∩ S₂ one_mem' := ⟨S₁.one_mem, S₂.one_mem⟩ mul_mem' := fun ⟨hx, hx'⟩ ⟨hy, hy'⟩ => ⟨S₁.mul_mem hx hy, S₂.mul_mem hx' hy'⟩ }⟩ @[to_additive (attr := simp)] theorem coe_inf (p p' : Submonoid M) : ((p ⊓ p' : Submonoid M) : Set M) = (p : Set M) ∩ p' := rfl @[to_additive (attr := simp)] theorem mem_inf {p p' : Submonoid M} {x : M} : x ∈ p ⊓ p' ↔ x ∈ p ∧ x ∈ p' := Iff.rfl @[to_additive] instance : InfSet (Submonoid M) := ⟨fun s => { carrier := ⋂ t ∈ s, ↑t one_mem' := Set.mem_biInter fun i _ => i.one_mem mul_mem' := fun hx hy => Set.mem_biInter fun i h => i.mul_mem (by apply Set.mem_iInter₂.1 hx i h) (by apply Set.mem_iInter₂.1 hy i h) }⟩ @[to_additive (attr := simp, norm_cast)] theorem coe_sInf (S : Set (Submonoid M)) : ((sInf S : Submonoid M) : Set M) = ⋂ s ∈ S, ↑s := rfl @[to_additive] theorem mem_sInf {S : Set (Submonoid M)} {x : M} : x ∈ sInf S ↔ ∀ p ∈ S, x ∈ p := Set.mem_iInter₂ @[to_additive] theorem mem_iInf {ι : Sort*} {S : ι → Submonoid M} {x : M} : (x ∈ ⨅ i, S i) ↔ ∀ i, x ∈ S i := by simp only [iInf, mem_sInf, Set.forall_mem_range] @[to_additive (attr := simp, norm_cast)] theorem coe_iInf {ι : Sort*} {S : ι → Submonoid M} : (↑(⨅ i, S i) : Set M) = ⋂ i, S i := by simp only [iInf, coe_sInf, Set.biInter_range] /-- Submonoids of a monoid form a complete lattice. -/ @[to_additive "The `AddSubmonoid`s of an `AddMonoid` form a complete lattice."] instance : CompleteLattice (Submonoid M) := { (completeLatticeOfInf (Submonoid M)) fun _ => IsGLB.of_image (f := (SetLike.coe : Submonoid M → Set M)) (@fun S T => show (S : Set M) ≤ T ↔ S ≤ T from SetLike.coe_subset_coe) isGLB_biInf with le := (· ≤ ·) lt := (· < ·) bot := ⊥ bot_le := fun S _ hx => (mem_bot.1 hx).symm ▸ S.one_mem top := ⊤ le_top := fun _ x _ => mem_top x inf := (· ⊓ ·) sInf := InfSet.sInf le_inf := fun _ _ _ ha hb _ hx => ⟨ha hx, hb hx⟩ inf_le_left := fun _ _ _ => And.left inf_le_right := fun _ _ _ => And.right } @[to_additive (attr := simp)] theorem subsingleton_iff : Subsingleton (Submonoid M) ↔ Subsingleton M := ⟨fun h => ⟨fun x y => have : ∀ i : M, i = 1 := fun i => mem_bot.mp <| Subsingleton.elim (⊤ : Submonoid M) ⊥ ▸ mem_top i (this x).trans (this y).symm⟩, fun h => ⟨fun x y => Submonoid.ext fun i => Subsingleton.elim 1 i ▸ by simp [Submonoid.one_mem]⟩⟩ @[to_additive (attr := simp)] theorem nontrivial_iff : Nontrivial (Submonoid M) ↔ Nontrivial M := not_iff_not.mp ((not_nontrivial_iff_subsingleton.trans subsingleton_iff).trans not_nontrivial_iff_subsingleton.symm) @[to_additive] instance [Subsingleton M] : Unique (Submonoid M) := ⟨⟨⊥⟩, fun a => @Subsingleton.elim _ (subsingleton_iff.mpr ‹_›) a _⟩ @[to_additive] instance [Nontrivial M] : Nontrivial (Submonoid M) := nontrivial_iff.mpr ‹_› /-- The `Submonoid` generated by a set. -/ @[to_additive "The `AddSubmonoid` generated by a set"] def closure (s : Set M) : Submonoid M := sInf { S | s ⊆ S } @[to_additive] theorem mem_closure {x : M} : x ∈ closure s ↔ ∀ S : Submonoid M, s ⊆ S → x ∈ S := mem_sInf /-- The submonoid generated by a set includes the set. -/ @[to_additive (attr := simp, aesop safe 20 apply (rule_sets := [SetLike])) "The `AddSubmonoid` generated by a set includes the set."] theorem subset_closure : s ⊆ closure s := fun _ hx => mem_closure.2 fun _ hS => hS hx @[to_additive] theorem not_mem_of_not_mem_closure {P : M} (hP : P ∉ closure s) : P ∉ s := fun h => hP (subset_closure h) variable {S} open Set /-- A submonoid `S` includes `closure s` if and only if it includes `s`. -/ @[to_additive (attr := simp) "An additive submonoid `S` includes `closure s` if and only if it includes `s`"] theorem closure_le : closure s ≤ S ↔ s ⊆ S := ⟨Subset.trans subset_closure, fun h => sInf_le h⟩ /-- Submonoid closure of a set is monotone in its argument: if `s ⊆ t`, then `closure s ≤ closure t`. -/ @[to_additive "Additive submonoid closure of a set is monotone in its argument: if `s ⊆ t`, then `closure s ≤ closure t`"] theorem closure_mono ⦃s t : Set M⦄ (h : s ⊆ t) : closure s ≤ closure t := closure_le.2 <| Subset.trans h subset_closure @[to_additive] theorem closure_eq_of_le (h₁ : s ⊆ S) (h₂ : S ≤ closure s) : closure s = S := le_antisymm (closure_le.2 h₁) h₂ variable (S) /-- An induction principle for closure membership. If `p` holds for `1` and all elements of `s`, and is preserved under multiplication, then `p` holds for all elements of the closure of `s`. -/ @[to_additive (attr := elab_as_elim) "An induction principle for additive closure membership. If `p` holds for `0` and all elements of `s`, and is preserved under addition, then `p` holds for all elements of the additive closure of `s`."] theorem closure_induction {p : M → Prop} {x} (h : x ∈ closure s) (mem : ∀ x ∈ s, p x) (one : p 1) (mul : ∀ x y, p x → p y → p (x * y)) : p x := (@closure_le _ _ _ ⟨⟨p, mul _ _⟩, one⟩).2 mem h /-- A dependent version of `Submonoid.closure_induction`. -/ @[to_additive (attr := elab_as_elim) "A dependent version of `AddSubmonoid.closure_induction`. "] theorem closure_induction' (s : Set M) {p : ∀ x, x ∈ closure s → Prop} (mem : ∀ (x) (h : x ∈ s), p x (subset_closure h)) (one : p 1 (one_mem _)) (mul : ∀ x hx y hy, p x hx → p y hy → p (x * y) (mul_mem hx hy)) {x} (hx : x ∈ closure s) : p x hx := by refine Exists.elim ?_ fun (hx : x ∈ closure s) (hc : p x hx) => hc exact closure_induction hx (fun x hx => ⟨_, mem x hx⟩) ⟨_, one⟩ fun x y ⟨hx', hx⟩ ⟨hy', hy⟩ => ⟨_, mul _ _ _ _ hx hy⟩ /-- An induction principle for closure membership for predicates with two arguments. -/ @[to_additive (attr := elab_as_elim) "An induction principle for additive closure membership for predicates with two arguments."] theorem closure_induction₂ {p : M → M → Prop} {x} {y : M} (hx : x ∈ closure s) (hy : y ∈ closure s) (Hs : ∀ x ∈ s, ∀ y ∈ s, p x y) (H1_left : ∀ x, p 1 x) (H1_right : ∀ x, p x 1) (Hmul_left : ∀ x y z, p x z → p y z → p (x * y) z) (Hmul_right : ∀ x y z, p z x → p z y → p z (x * y)) : p x y := closure_induction hx (fun x xs => closure_induction hy (Hs x xs) (H1_right x) fun z _ h₁ h₂ => Hmul_right z _ _ h₁ h₂) (H1_left y) fun _ _ h₁ h₂ => Hmul_left _ _ _ h₁ h₂ /-- If `s` is a dense set in a monoid `M`, `Submonoid.closure s = ⊤`, then in order to prove that some predicate `p` holds for all `x : M` it suffices to verify `p x` for `x ∈ s`, verify `p 1`, and verify that `p x` and `p y` imply `p (x * y)`. -/ @[to_additive (attr := elab_as_elim) "If `s` is a dense set in an additive monoid `M`, `AddSubmonoid.closure s = ⊤`, then in order to prove that some predicate `p` holds for all `x : M` it suffices to verify `p x` for `x ∈ s`, verify `p 0`, and verify that `p x` and `p y` imply `p (x + y)`."] theorem dense_induction {p : M → Prop} (x : M) {s : Set M} (hs : closure s = ⊤) (mem : ∀ x ∈ s, p x) (one : p 1) (mul : ∀ x y, p x → p y → p (x * y)) : p x := by have : ∀ x ∈ closure s, p x := fun x hx => closure_induction hx mem one mul simpa [hs] using this x /-- The `Submonoid.closure` of a set is the union of `{1}` and its `Subsemigroup.closure`. -/ lemma closure_eq_one_union (s : Set M) : closure s = {(1 : M)} ∪ (Subsemigroup.closure s : Set M) := by apply le_antisymm · intro x hx induction hx using closure_induction' with | mem x hx => exact Or.inr <| Subsemigroup.subset_closure hx | one => exact Or.inl <| by simp | mul x hx y hy hx hy => simp only [singleton_union, mem_insert_iff, SetLike.mem_coe] at hx hy obtain ⟨(rfl | hx), (rfl | hy)⟩ := And.intro hx hy all_goals simp_all exact Or.inr <| mul_mem hx hy · rintro x (hx | hx) · exact (show x = 1 by simpa using hx) ▸ one_mem (closure s) · exact Subsemigroup.closure_le.mpr subset_closure hx variable (M) /-- `closure` forms a Galois insertion with the coercion to set. -/ @[to_additive "`closure` forms a Galois insertion with the coercion to set."] protected def gi : GaloisInsertion (@closure M _) SetLike.coe where choice s _ := closure s gc _ _ := closure_le le_l_u _ := subset_closure choice_eq _ _ := rfl variable {M} /-- Closure of a submonoid `S` equals `S`. -/ @[to_additive (attr := simp) "Additive closure of an additive submonoid `S` equals `S`"] theorem closure_eq : closure (S : Set M) = S := (Submonoid.gi M).l_u_eq S @[to_additive (attr := simp)] theorem closure_empty : closure (∅ : Set M) = ⊥ := (Submonoid.gi M).gc.l_bot @[to_additive (attr := simp)] theorem closure_univ : closure (univ : Set M) = ⊤ := @coe_top M _ ▸ closure_eq ⊤ @[to_additive] theorem closure_union (s t : Set M) : closure (s ∪ t) = closure s ⊔ closure t := (Submonoid.gi M).gc.l_sup @[to_additive] theorem sup_eq_closure (N N' : Submonoid M) : N ⊔ N' = closure ((N : Set M) ∪ (N' : Set M)) := by simp_rw [closure_union, closure_eq] @[to_additive] theorem closure_iUnion {ι} (s : ι → Set M) : closure (⋃ i, s i) = ⨆ i, closure (s i) := (Submonoid.gi M).gc.l_iSup -- Porting note (#10618): `simp` can now prove this, so we remove the `@[simp]` attribute @[to_additive] theorem closure_singleton_le_iff_mem (m : M) (p : Submonoid M) : closure {m} ≤ p ↔ m ∈ p := by rw [closure_le, singleton_subset_iff, SetLike.mem_coe] @[to_additive] theorem mem_iSup {ι : Sort*} (p : ι → Submonoid M) {m : M} : (m ∈ ⨆ i, p i) ↔ ∀ N, (∀ i, p i ≤ N) → m ∈ N := by rw [← closure_singleton_le_iff_mem, le_iSup_iff] simp only [closure_singleton_le_iff_mem] @[to_additive] theorem iSup_eq_closure {ι : Sort*} (p : ι → Submonoid M) : ⨆ i, p i = Submonoid.closure (⋃ i, (p i : Set M)) := by simp_rw [Submonoid.closure_iUnion, Submonoid.closure_eq] @[to_additive] theorem disjoint_def {p₁ p₂ : Submonoid M} : Disjoint p₁ p₂ ↔ ∀ {x : M}, x ∈ p₁ → x ∈ p₂ → x = 1 := by simp_rw [disjoint_iff_inf_le, SetLike.le_def, mem_inf, and_imp, mem_bot] @[to_additive] theorem disjoint_def' {p₁ p₂ : Submonoid M} : Disjoint p₁ p₂ ↔ ∀ {x y : M}, x ∈ p₁ → y ∈ p₂ → x = y → x = 1 := disjoint_def.trans ⟨fun h _ _ hx hy hxy => h hx <| hxy.symm ▸ hy, fun h _ hx hx' => h hx hx' rfl⟩ end Submonoid namespace MonoidHom variable [MulOneClass N] open Submonoid /-- The submonoid of elements `x : M` such that `f x = g x` -/ @[to_additive "The additive submonoid of elements `x : M` such that `f x = g x`"] def eqLocusM (f g : M →* N) : Submonoid M where carrier := { x | f x = g x } one_mem' := by rw [Set.mem_setOf_eq, f.map_one, g.map_one] mul_mem' (hx : _ = _) (hy : _ = _) := by simp [*] @[to_additive (attr := simp)] theorem eqLocusM_same (f : M →* N) : f.eqLocusM f = ⊤ := SetLike.ext fun _ => eq_self_iff_true _ /-- If two monoid homomorphisms are equal on a set, then they are equal on its submonoid closure. -/ @[to_additive "If two monoid homomorphisms are equal on a set, then they are equal on its submonoid closure."] theorem eqOn_closureM {f g : M →* N} {s : Set M} (h : Set.EqOn f g s) : Set.EqOn f g (closure s) := show closure s ≤ f.eqLocusM g from closure_le.2 h @[to_additive] theorem eq_of_eqOn_topM {f g : M →* N} (h : Set.EqOn f g (⊤ : Submonoid M)) : f = g := ext fun _ => h trivial @[to_additive] theorem eq_of_eqOn_denseM {s : Set M} (hs : closure s = ⊤) {f g : M →* N} (h : s.EqOn f g) : f = g := eq_of_eqOn_topM <| hs ▸ eqOn_closureM h end MonoidHom end NonAssoc section Assoc variable [Monoid M] [Monoid N] {s : Set M} section IsUnit /-- The submonoid consisting of the units of a monoid -/ @[to_additive "The additive submonoid consisting of the additive units of an additive monoid"] def IsUnit.submonoid (M : Type*) [Monoid M] : Submonoid M where carrier := setOf IsUnit one_mem' := by simp only [isUnit_one, Set.mem_setOf_eq] mul_mem' := by intro a b ha hb rw [Set.mem_setOf_eq] at * exact IsUnit.mul ha hb @[to_additive] theorem IsUnit.mem_submonoid_iff {M : Type*} [Monoid M] (a : M) : a ∈ IsUnit.submonoid M ↔ IsUnit a := by change a ∈ setOf IsUnit ↔ IsUnit a rw [Set.mem_setOf_eq] end IsUnit namespace MonoidHom open Submonoid /-- Let `s` be a subset of a monoid `M` such that the closure of `s` is the whole monoid. Then `MonoidHom.ofClosureEqTopLeft` defines a monoid homomorphism from `M` asking for a proof of `f (x * y) = f x * f y` only for `x ∈ s`. -/ @[to_additive "Let `s` be a subset of an additive monoid `M` such that the closure of `s` is the whole monoid. Then `AddMonoidHom.ofClosureEqTopLeft` defines an additive monoid homomorphism from `M` asking for a proof of `f (x + y) = f x + f y` only for `x ∈ s`. "] def ofClosureMEqTopLeft {M N} [Monoid M] [Monoid N] {s : Set M} (f : M → N) (hs : closure s = ⊤) (h1 : f 1 = 1) (hmul : ∀ x ∈ s, ∀ (y), f (x * y) = f x * f y) : M →* N where toFun := f map_one' := h1 map_mul' x := (dense_induction (p := _) x hs hmul fun y => by rw [one_mul, h1, one_mul]) fun a b ha hb y => by rw [mul_assoc, ha, ha, hb, mul_assoc] @[to_additive (attr := simp, norm_cast)] theorem coe_ofClosureMEqTopLeft (f : M → N) (hs : closure s = ⊤) (h1 hmul) : ⇑(ofClosureMEqTopLeft f hs h1 hmul) = f := rfl /-- Let `s` be a subset of a monoid `M` such that the closure of `s` is the whole monoid. Then `MonoidHom.ofClosureEqTopRight` defines a monoid homomorphism from `M` asking for a proof of `f (x * y) = f x * f y` only for `y ∈ s`. -/ @[to_additive "Let `s` be a subset of an additive monoid `M` such that the closure of `s` is the whole monoid. Then `AddMonoidHom.ofClosureEqTopRight` defines an additive monoid homomorphism from `M` asking for a proof of `f (x + y) = f x + f y` only for `y ∈ s`. "] def ofClosureMEqTopRight {M N} [Monoid M] [Monoid N] {s : Set M} (f : M → N) (hs : closure s = ⊤) (h1 : f 1 = 1) (hmul : ∀ (x), ∀ y ∈ s, f (x * y) = f x * f y) : M →* N where toFun := f map_one' := h1 map_mul' x y := dense_induction y hs (fun y hy x => hmul x y hy) (by simp [h1]) (fun y₁ y₂ (h₁ : ∀ x, f _ = f _ * f _) (h₂ : ∀ x, f _ = f _ * f _) x => by simp [← mul_assoc, h₁, h₂]) x @[to_additive (attr := simp, norm_cast)] theorem coe_ofClosureMEqTopRight (f : M → N) (hs : closure s = ⊤) (h1 hmul) : ⇑(ofClosureMEqTopRight f hs h1 hmul) = f := rfl end MonoidHom end Assoc
Algebra\Group\Submonoid\DistribMulAction.lean
/- Copyright (c) 2022 Yaël Dillies. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Yaël Dillies -/ import Mathlib.Algebra.Group.Submonoid.Operations import Mathlib.Algebra.GroupWithZero.Action.Defs /-! # Distributive actions by submonoids -/ namespace Submonoid variable {M α : Type*} [Monoid M] /-- The action by a submonoid is the action by the underlying monoid. -/ instance distribMulAction [AddMonoid α] [DistribMulAction M α] (S : Submonoid M) : DistribMulAction S α := DistribMulAction.compHom _ S.subtype /-- The action by a submonoid is the action by the underlying monoid. -/ instance mulDistribMulAction [Monoid α] [MulDistribMulAction M α] (S : Submonoid M) : MulDistribMulAction S α := MulDistribMulAction.compHom _ S.subtype end Submonoid
Algebra\Group\Submonoid\Membership.lean
/- Copyright (c) 2018 Johannes Hölzl. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Johannes Hölzl, Kenny Lau, Johan Commelin, Mario Carneiro, Kevin Buzzard, Amelia Livingston, Yury Kudryashov -/ import Mathlib.Algebra.FreeMonoid.Basic import Mathlib.Algebra.Group.Submonoid.MulOpposite import Mathlib.Algebra.Group.Submonoid.Operations import Mathlib.Algebra.GroupWithZero.Divisibility import Mathlib.Algebra.Ring.Int import Mathlib.Data.Finset.NoncommProd import Mathlib.Data.Nat.Cast.Basic import Mathlib.Util.AssertExists /-! # Submonoids: membership criteria In this file we prove various facts about membership in a submonoid: * `list_prod_mem`, `multiset_prod_mem`, `prod_mem`: if each element of a collection belongs to a multiplicative submonoid, then so does their product; * `list_sum_mem`, `multiset_sum_mem`, `sum_mem`: if each element of a collection belongs to an additive submonoid, then so does their sum; * `pow_mem`, `nsmul_mem`: if `x ∈ S` where `S` is a multiplicative (resp., additive) submonoid and `n` is a natural number, then `x^n` (resp., `n • x`) belongs to `S`; * `mem_iSup_of_directed`, `coe_iSup_of_directed`, `mem_sSup_of_directedOn`, `coe_sSup_of_directedOn`: the supremum of a directed collection of submonoid is their union. * `sup_eq_range`, `mem_sup`: supremum of two submonoids `S`, `T` of a commutative monoid is the set of products; * `closure_singleton_eq`, `mem_closure_singleton`, `mem_closure_pair`: the multiplicative (resp., additive) closure of `{x}` consists of powers (resp., natural multiples) of `x`, and a similar result holds for the closure of `{x, y}`. ## Tags submonoid, submonoids -/ -- We don't need ordered structures to establish basic membership facts for submonoids assert_not_exists OrderedSemiring variable {M A B : Type*} section Assoc variable [Monoid M] [SetLike B M] [SubmonoidClass B M] {S : B} namespace SubmonoidClass @[to_additive (attr := norm_cast, simp)] theorem coe_list_prod (l : List S) : (l.prod : M) = (l.map (↑)).prod := map_list_prod (SubmonoidClass.subtype S : _ →* M) l @[to_additive (attr := norm_cast, simp)] theorem coe_multiset_prod {M} [CommMonoid M] [SetLike B M] [SubmonoidClass B M] (m : Multiset S) : (m.prod : M) = (m.map (↑)).prod := (SubmonoidClass.subtype S : _ →* M).map_multiset_prod m @[to_additive (attr := norm_cast)] -- Porting note (#10618): removed `simp`, `simp` can prove it theorem coe_finset_prod {ι M} [CommMonoid M] [SetLike B M] [SubmonoidClass B M] (f : ι → S) (s : Finset ι) : ↑(∏ i ∈ s, f i) = (∏ i ∈ s, f i : M) := map_prod (SubmonoidClass.subtype S) f s end SubmonoidClass open SubmonoidClass /-- Product of a list of elements in a submonoid is in the submonoid. -/ @[to_additive "Sum of a list of elements in an `AddSubmonoid` is in the `AddSubmonoid`."] theorem list_prod_mem {l : List M} (hl : ∀ x ∈ l, x ∈ S) : l.prod ∈ S := by lift l to List S using hl rw [← coe_list_prod] exact l.prod.coe_prop /-- Product of a multiset of elements in a submonoid of a `CommMonoid` is in the submonoid. -/ @[to_additive "Sum of a multiset of elements in an `AddSubmonoid` of an `AddCommMonoid` is in the `AddSubmonoid`."] theorem multiset_prod_mem {M} [CommMonoid M] [SetLike B M] [SubmonoidClass B M] (m : Multiset M) (hm : ∀ a ∈ m, a ∈ S) : m.prod ∈ S := by lift m to Multiset S using hm rw [← coe_multiset_prod] exact m.prod.coe_prop /-- Product of elements of a submonoid of a `CommMonoid` indexed by a `Finset` is in the submonoid. -/ @[to_additive "Sum of elements in an `AddSubmonoid` of an `AddCommMonoid` indexed by a `Finset` is in the `AddSubmonoid`."] theorem prod_mem {M : Type*} [CommMonoid M] [SetLike B M] [SubmonoidClass B M] {ι : Type*} {t : Finset ι} {f : ι → M} (h : ∀ c ∈ t, f c ∈ S) : (∏ c ∈ t, f c) ∈ S := multiset_prod_mem (t.1.map f) fun _x hx => let ⟨i, hi, hix⟩ := Multiset.mem_map.1 hx hix ▸ h i hi namespace Submonoid variable (s : Submonoid M) @[to_additive (attr := norm_cast)] -- Porting note (#10618): removed `simp`, `simp` can prove it theorem coe_list_prod (l : List s) : (l.prod : M) = (l.map (↑)).prod := map_list_prod s.subtype l @[to_additive (attr := norm_cast)] -- Porting note (#10618): removed `simp`, `simp` can prove it theorem coe_multiset_prod {M} [CommMonoid M] (S : Submonoid M) (m : Multiset S) : (m.prod : M) = (m.map (↑)).prod := S.subtype.map_multiset_prod m @[to_additive (attr := norm_cast, simp)] theorem coe_finset_prod {ι M} [CommMonoid M] (S : Submonoid M) (f : ι → S) (s : Finset ι) : ↑(∏ i ∈ s, f i) = (∏ i ∈ s, f i : M) := map_prod S.subtype f s /-- Product of a list of elements in a submonoid is in the submonoid. -/ @[to_additive "Sum of a list of elements in an `AddSubmonoid` is in the `AddSubmonoid`."] theorem list_prod_mem {l : List M} (hl : ∀ x ∈ l, x ∈ s) : l.prod ∈ s := by lift l to List s using hl rw [← coe_list_prod] exact l.prod.coe_prop /-- Product of a multiset of elements in a submonoid of a `CommMonoid` is in the submonoid. -/ @[to_additive "Sum of a multiset of elements in an `AddSubmonoid` of an `AddCommMonoid` is in the `AddSubmonoid`."] theorem multiset_prod_mem {M} [CommMonoid M] (S : Submonoid M) (m : Multiset M) (hm : ∀ a ∈ m, a ∈ S) : m.prod ∈ S := by lift m to Multiset S using hm rw [← coe_multiset_prod] exact m.prod.coe_prop @[to_additive] theorem multiset_noncommProd_mem (S : Submonoid M) (m : Multiset M) (comm) (h : ∀ x ∈ m, x ∈ S) : m.noncommProd comm ∈ S := by induction' m using Quotient.inductionOn with l simp only [Multiset.quot_mk_to_coe, Multiset.noncommProd_coe] exact Submonoid.list_prod_mem _ h /-- Product of elements of a submonoid of a `CommMonoid` indexed by a `Finset` is in the submonoid. -/ @[to_additive "Sum of elements in an `AddSubmonoid` of an `AddCommMonoid` indexed by a `Finset` is in the `AddSubmonoid`."] theorem prod_mem {M : Type*} [CommMonoid M] (S : Submonoid M) {ι : Type*} {t : Finset ι} {f : ι → M} (h : ∀ c ∈ t, f c ∈ S) : (∏ c ∈ t, f c) ∈ S := S.multiset_prod_mem (t.1.map f) fun _ hx => let ⟨i, hi, hix⟩ := Multiset.mem_map.1 hx hix ▸ h i hi @[to_additive] theorem noncommProd_mem (S : Submonoid M) {ι : Type*} (t : Finset ι) (f : ι → M) (comm) (h : ∀ c ∈ t, f c ∈ S) : t.noncommProd f comm ∈ S := by apply multiset_noncommProd_mem intro y rw [Multiset.mem_map] rintro ⟨x, ⟨hx, rfl⟩⟩ exact h x hx end Submonoid end Assoc section NonAssoc variable [MulOneClass M] open Set namespace Submonoid -- TODO: this section can be generalized to `[SubmonoidClass B M] [CompleteLattice B]` -- such that `CompleteLattice.LE` coincides with `SetLike.LE` @[to_additive] theorem mem_iSup_of_directed {ι} [hι : Nonempty ι] {S : ι → Submonoid M} (hS : Directed (· ≤ ·) S) {x : M} : (x ∈ ⨆ i, S i) ↔ ∃ i, x ∈ S i := by refine ⟨?_, fun ⟨i, hi⟩ ↦ le_iSup S i hi⟩ suffices x ∈ closure (⋃ i, (S i : Set M)) → ∃ i, x ∈ S i by simpa only [closure_iUnion, closure_eq (S _)] using this refine fun hx ↦ closure_induction hx (fun _ ↦ mem_iUnion.1) ?_ ?_ · exact hι.elim fun i ↦ ⟨i, (S i).one_mem⟩ · rintro x y ⟨i, hi⟩ ⟨j, hj⟩ rcases hS i j with ⟨k, hki, hkj⟩ exact ⟨k, (S k).mul_mem (hki hi) (hkj hj)⟩ @[to_additive] theorem coe_iSup_of_directed {ι} [Nonempty ι] {S : ι → Submonoid M} (hS : Directed (· ≤ ·) S) : ((⨆ i, S i : Submonoid M) : Set M) = ⋃ i, S i := Set.ext fun x ↦ by simp [mem_iSup_of_directed hS] @[to_additive] theorem mem_sSup_of_directedOn {S : Set (Submonoid M)} (Sne : S.Nonempty) (hS : DirectedOn (· ≤ ·) S) {x : M} : x ∈ sSup S ↔ ∃ s ∈ S, x ∈ s := by haveI : Nonempty S := Sne.to_subtype simp [sSup_eq_iSup', mem_iSup_of_directed hS.directed_val, SetCoe.exists, Subtype.coe_mk] @[to_additive] theorem coe_sSup_of_directedOn {S : Set (Submonoid M)} (Sne : S.Nonempty) (hS : DirectedOn (· ≤ ·) S) : (↑(sSup S) : Set M) = ⋃ s ∈ S, ↑s := Set.ext fun x => by simp [mem_sSup_of_directedOn Sne hS] @[to_additive] theorem mem_sup_left {S T : Submonoid M} : ∀ {x : M}, x ∈ S → x ∈ S ⊔ T := by rw [← SetLike.le_def] exact le_sup_left @[to_additive] theorem mem_sup_right {S T : Submonoid M} : ∀ {x : M}, x ∈ T → x ∈ S ⊔ T := by rw [← SetLike.le_def] exact le_sup_right @[to_additive] theorem mul_mem_sup {S T : Submonoid M} {x y : M} (hx : x ∈ S) (hy : y ∈ T) : x * y ∈ S ⊔ T := (S ⊔ T).mul_mem (mem_sup_left hx) (mem_sup_right hy) @[to_additive] theorem mem_iSup_of_mem {ι : Sort*} {S : ι → Submonoid M} (i : ι) : ∀ {x : M}, x ∈ S i → x ∈ iSup S := by rw [← SetLike.le_def] exact le_iSup _ _ @[to_additive] theorem mem_sSup_of_mem {S : Set (Submonoid M)} {s : Submonoid M} (hs : s ∈ S) : ∀ {x : M}, x ∈ s → x ∈ sSup S := by rw [← SetLike.le_def] exact le_sSup hs /-- An induction principle for elements of `⨆ i, S i`. If `C` holds for `1` and all elements of `S i` for all `i`, and is preserved under multiplication, then it holds for all elements of the supremum of `S`. -/ @[to_additive (attr := elab_as_elim) " An induction principle for elements of `⨆ i, S i`. If `C` holds for `0` and all elements of `S i` for all `i`, and is preserved under addition, then it holds for all elements of the supremum of `S`. "] theorem iSup_induction {ι : Sort*} (S : ι → Submonoid M) {C : M → Prop} {x : M} (hx : x ∈ ⨆ i, S i) (mem : ∀ (i), ∀ x ∈ S i, C x) (one : C 1) (mul : ∀ x y, C x → C y → C (x * y)) : C x := by rw [iSup_eq_closure] at hx refine closure_induction hx (fun x hx => ?_) one mul obtain ⟨i, hi⟩ := Set.mem_iUnion.mp hx exact mem _ _ hi /-- A dependent version of `Submonoid.iSup_induction`. -/ @[to_additive (attr := elab_as_elim) "A dependent version of `AddSubmonoid.iSup_induction`. "] theorem iSup_induction' {ι : Sort*} (S : ι → Submonoid M) {C : ∀ x, (x ∈ ⨆ i, S i) → Prop} (mem : ∀ (i), ∀ (x) (hxS : x ∈ S i), C x (mem_iSup_of_mem i hxS)) (one : C 1 (one_mem _)) (mul : ∀ x y hx hy, C x hx → C y hy → C (x * y) (mul_mem ‹_› ‹_›)) {x : M} (hx : x ∈ ⨆ i, S i) : C x hx := by refine Exists.elim (?_ : ∃ Hx, C x Hx) fun (hx : x ∈ ⨆ i, S i) (hc : C x hx) => hc refine @iSup_induction _ _ ι S (fun m => ∃ hm, C m hm) _ hx (fun i x hx => ?_) ?_ fun x y => ?_ · exact ⟨_, mem _ _ hx⟩ · exact ⟨_, one⟩ · rintro ⟨_, Cx⟩ ⟨_, Cy⟩ exact ⟨_, mul _ _ _ _ Cx Cy⟩ end Submonoid end NonAssoc namespace FreeMonoid variable {α : Type*} open Submonoid @[to_additive] theorem closure_range_of : closure (Set.range <| @of α) = ⊤ := eq_top_iff.2 fun x _ => FreeMonoid.recOn x (one_mem _) fun _x _xs hxs => mul_mem (subset_closure <| Set.mem_range_self _) hxs end FreeMonoid namespace Submonoid variable [Monoid M] {a : M} open MonoidHom theorem closure_singleton_eq (x : M) : closure ({x} : Set M) = mrange (powersHom M x) := closure_eq_of_le (Set.singleton_subset_iff.2 ⟨Multiplicative.ofAdd 1, pow_one x⟩) fun _ ⟨_, hn⟩ => hn ▸ pow_mem (subset_closure <| Set.mem_singleton _) _ /-- The submonoid generated by an element of a monoid equals the set of natural number powers of the element. -/ theorem mem_closure_singleton {x y : M} : y ∈ closure ({x} : Set M) ↔ ∃ n : ℕ, x ^ n = y := by rw [closure_singleton_eq, mem_mrange]; rfl theorem mem_closure_singleton_self {y : M} : y ∈ closure ({y} : Set M) := mem_closure_singleton.2 ⟨1, pow_one y⟩ theorem closure_singleton_one : closure ({1} : Set M) = ⊥ := by simp [eq_bot_iff_forall, mem_closure_singleton] section Submonoid variable {S : Submonoid M} [Fintype S] open Fintype /- curly brackets `{}` are used here instead of instance brackets `[]` because the instance in a goal is often not the same as the one inferred by type class inference. -/ @[to_additive] theorem card_bot {_ : Fintype (⊥ : Submonoid M)} : card (⊥ : Submonoid M) = 1 := card_eq_one_iff.2 ⟨⟨(1 : M), Set.mem_singleton 1⟩, fun ⟨_y, hy⟩ => Subtype.eq <| mem_bot.1 hy⟩ @[to_additive] theorem eq_bot_of_card_le (h : card S ≤ 1) : S = ⊥ := let _ := card_le_one_iff_subsingleton.mp h eq_bot_of_subsingleton S @[to_additive] theorem eq_bot_of_card_eq (h : card S = 1) : S = ⊥ := S.eq_bot_of_card_le (le_of_eq h) @[to_additive card_le_one_iff_eq_bot] theorem card_le_one_iff_eq_bot : card S ≤ 1 ↔ S = ⊥ := ⟨fun h => (eq_bot_iff_forall _).2 fun x hx => by simpa [Subtype.ext_iff] using card_le_one_iff.1 h ⟨x, hx⟩ 1, fun h => by simp [h]⟩ @[to_additive] lemma eq_bot_iff_card : S = ⊥ ↔ card S = 1 := ⟨by rintro rfl; exact card_bot, eq_bot_of_card_eq⟩ end Submonoid @[to_additive] theorem _root_.FreeMonoid.mrange_lift {α} (f : α → M) : mrange (FreeMonoid.lift f) = closure (Set.range f) := by rw [mrange_eq_map, ← FreeMonoid.closure_range_of, map_mclosure, ← Set.range_comp, FreeMonoid.lift_comp_of] @[to_additive] theorem closure_eq_mrange (s : Set M) : closure s = mrange (FreeMonoid.lift ((↑) : s → M)) := by rw [FreeMonoid.mrange_lift, Subtype.range_coe] @[to_additive] theorem closure_eq_image_prod (s : Set M) : (closure s : Set M) = List.prod '' { l : List M | ∀ x ∈ l, x ∈ s } := by rw [closure_eq_mrange, coe_mrange, ← Set.range_list_map_coe, ← Set.range_comp] exact congrArg _ (funext <| FreeMonoid.lift_apply _) @[to_additive] theorem exists_list_of_mem_closure {s : Set M} {x : M} (hx : x ∈ closure s) : ∃ l : List M, (∀ y ∈ l, y ∈ s) ∧ l.prod = x := by rwa [← SetLike.mem_coe, closure_eq_image_prod, Set.mem_image] at hx @[to_additive] theorem exists_multiset_of_mem_closure {M : Type*} [CommMonoid M] {s : Set M} {x : M} (hx : x ∈ closure s) : ∃ l : Multiset M, (∀ y ∈ l, y ∈ s) ∧ l.prod = x := by obtain ⟨l, h1, h2⟩ := exists_list_of_mem_closure hx exact ⟨l, h1, (Multiset.prod_coe l).trans h2⟩ @[to_additive (attr := elab_as_elim)] theorem closure_induction_left {s : Set M} {p : (m : M) → m ∈ closure s → Prop} (one : p 1 (one_mem _)) (mul_left : ∀ x (hx : x ∈ s), ∀ (y) hy, p y hy → p (x * y) (mul_mem (subset_closure hx) hy)) {x : M} (h : x ∈ closure s) : p x h := by simp_rw [closure_eq_mrange] at h obtain ⟨l, rfl⟩ := h induction' l with x y ih · exact one · simp only [map_mul, FreeMonoid.lift_eval_of] refine mul_left _ x.prop (FreeMonoid.lift Subtype.val y) _ (ih ?_) simp only [closure_eq_mrange, mem_mrange, exists_apply_eq_apply] @[to_additive (attr := elab_as_elim)] theorem induction_of_closure_eq_top_left {s : Set M} {p : M → Prop} (hs : closure s = ⊤) (x : M) (one : p 1) (mul : ∀ x ∈ s, ∀ (y), p y → p (x * y)) : p x := by have : x ∈ closure s := by simp [hs] induction this using closure_induction_left with | one => exact one | mul_left x hx y _ ih => exact mul x hx y ih @[to_additive (attr := elab_as_elim)] theorem closure_induction_right {s : Set M} {p : (m : M) → m ∈ closure s → Prop} (one : p 1 (one_mem _)) (mul_right : ∀ x hx, ∀ (y) (hy : y ∈ s), p x hx → p (x * y) (mul_mem hx (subset_closure hy))) {x : M} (h : x ∈ closure s) : p x h := closure_induction_left (s := MulOpposite.unop ⁻¹' s) (p := fun m hm => p m.unop <| by rwa [← op_closure] at hm) one (fun _x hx _y hy => mul_right _ _ _ hx) (by rwa [← op_closure]) @[to_additive (attr := elab_as_elim)] theorem induction_of_closure_eq_top_right {s : Set M} {p : M → Prop} (hs : closure s = ⊤) (x : M) (H1 : p 1) (Hmul : ∀ (x), ∀ y ∈ s, p x → p (x * y)) : p x := by have : x ∈ closure s := by simp [hs] induction this using closure_induction_right with | one => exact H1 | mul_right x _ y hy ih => exact Hmul x y hy ih /-- The submonoid generated by an element. -/ def powers (n : M) : Submonoid M := Submonoid.copy (mrange (powersHom M n)) (Set.range (n ^ · : ℕ → M)) <| Set.ext fun n => exists_congr fun i => by simp; rfl theorem mem_powers (n : M) : n ∈ powers n := ⟨1, pow_one _⟩ theorem coe_powers (x : M) : ↑(powers x) = Set.range fun n : ℕ => x ^ n := rfl theorem mem_powers_iff (x z : M) : x ∈ powers z ↔ ∃ n : ℕ, z ^ n = x := Iff.rfl noncomputable instance decidableMemPowers : DecidablePred (· ∈ Submonoid.powers a) := Classical.decPred _ -- Porting note (#11215): TODO the following instance should follow from a more general principle -- See also mathlib4#2417 noncomputable instance fintypePowers [Fintype M] : Fintype (powers a) := inferInstanceAs <| Fintype {y // y ∈ powers a} theorem powers_eq_closure (n : M) : powers n = closure {n} := by ext exact mem_closure_singleton.symm lemma powers_le {n : M} {P : Submonoid M} : powers n ≤ P ↔ n ∈ P := by simp [powers_eq_closure] lemma powers_one : powers (1 : M) = ⊥ := bot_unique <| powers_le.2 <| one_mem _ /-- The submonoid generated by an element is a group if that element has finite order. -/ abbrev groupPowers {x : M} {n : ℕ} (hpos : 0 < n) (hx : x ^ n = 1) : Group (powers x) where inv x := x ^ (n - 1) mul_left_inv y := Subtype.ext <| by obtain ⟨_, k, rfl⟩ := y simp only [coe_one, coe_mul, SubmonoidClass.coe_pow] rw [← pow_succ, Nat.sub_add_cancel hpos, ← pow_mul, mul_comm, pow_mul, hx, one_pow] zpow z x := x ^ z.natMod n zpow_zero' z := by simp only [Int.natMod, Int.zero_emod, Int.toNat_zero, pow_zero] zpow_neg' m x := Subtype.ext <| by obtain ⟨_, k, rfl⟩ := x simp only [← pow_mul, Int.natMod, SubmonoidClass.coe_pow] rw [Int.negSucc_coe, ← Int.add_mul_emod_self (b := (m + 1 : ℕ))] nth_rw 1 [← mul_one ((m + 1 : ℕ) : ℤ)] rw [← sub_eq_neg_add, ← mul_sub, ← Int.natCast_pred_of_pos hpos]; norm_cast simp only [Int.toNat_natCast] rw [mul_comm, pow_mul, ← pow_eq_pow_mod _ hx, mul_comm k, mul_assoc, pow_mul _ (_ % _), ← pow_eq_pow_mod _ hx, pow_mul, pow_mul] zpow_succ' m x := Subtype.ext <| by obtain ⟨_, k, rfl⟩ := x simp only [← pow_mul, Int.natMod, Int.ofNat_eq_coe, SubmonoidClass.coe_pow, coe_mul] norm_cast iterate 2 rw [Int.toNat_natCast, mul_comm, pow_mul, ← pow_eq_pow_mod _ hx] rw [← pow_mul _ m, mul_comm, pow_mul, ← pow_succ, ← pow_mul, mul_comm, pow_mul] /-- Exponentiation map from natural numbers to powers. -/ @[simps!] def pow (n : M) (m : ℕ) : powers n := (powersHom M n).mrangeRestrict (Multiplicative.ofAdd m) theorem pow_apply (n : M) (m : ℕ) : Submonoid.pow n m = ⟨n ^ m, m, rfl⟩ := rfl /-- Logarithms from powers to natural numbers. -/ def log [DecidableEq M] {n : M} (p : powers n) : ℕ := Nat.find <| (mem_powers_iff p.val n).mp p.prop @[simp] theorem pow_log_eq_self [DecidableEq M] {n : M} (p : powers n) : pow n (log p) = p := Subtype.ext <| Nat.find_spec p.prop theorem pow_right_injective_iff_pow_injective {n : M} : (Function.Injective fun m : ℕ => n ^ m) ↔ Function.Injective (pow n) := Subtype.coe_injective.of_comp_iff (pow n) @[simp] theorem log_pow_eq_self [DecidableEq M] {n : M} (h : Function.Injective fun m : ℕ => n ^ m) (m : ℕ) : log (pow n m) = m := pow_right_injective_iff_pow_injective.mp h <| pow_log_eq_self _ /-- The exponentiation map is an isomorphism from the additive monoid on natural numbers to powers when it is injective. The inverse is given by the logarithms. -/ @[simps] def powLogEquiv [DecidableEq M] {n : M} (h : Function.Injective fun m : ℕ => n ^ m) : Multiplicative ℕ ≃* powers n where toFun m := pow n (Multiplicative.toAdd m) invFun m := Multiplicative.ofAdd (log m) left_inv := log_pow_eq_self h right_inv := pow_log_eq_self map_mul' _ _ := by simp only [pow, map_mul, ofAdd_add, toAdd_mul] theorem log_mul [DecidableEq M] {n : M} (h : Function.Injective fun m : ℕ => n ^ m) (x y : powers (n : M)) : log (x * y) = log x + log y := (powLogEquiv h).symm.map_mul x y theorem log_pow_int_eq_self {x : ℤ} (h : 1 < x.natAbs) (m : ℕ) : log (pow x m) = m := (powLogEquiv (Int.pow_right_injective h)).symm_apply_apply _ @[simp] theorem map_powers {N : Type*} {F : Type*} [Monoid N] [FunLike F M N] [MonoidHomClass F M N] (f : F) (m : M) : (powers m).map f = powers (f m) := by simp only [powers_eq_closure, map_mclosure f, Set.image_singleton] /-- If all the elements of a set `s` commute, then `closure s` is a commutative monoid. -/ @[to_additive "If all the elements of a set `s` commute, then `closure s` forms an additive commutative monoid."] def closureCommMonoidOfComm {s : Set M} (hcomm : ∀ a ∈ s, ∀ b ∈ s, a * b = b * a) : CommMonoid (closure s) := { (closure s).toMonoid with mul_comm := fun x y => by ext simp only [Submonoid.coe_mul] exact closure_induction₂ x.prop y.prop hcomm Commute.one_left Commute.one_right (fun x y z => Commute.mul_left) fun x y z => Commute.mul_right } end Submonoid @[to_additive] theorem IsScalarTower.of_mclosure_eq_top {N α} [Monoid M] [MulAction M N] [SMul N α] [MulAction M α] {s : Set M} (htop : Submonoid.closure s = ⊤) (hs : ∀ x ∈ s, ∀ (y : N) (z : α), (x • y) • z = x • y • z) : IsScalarTower M N α := by refine ⟨fun x => Submonoid.induction_of_closure_eq_top_left htop x ?_ ?_⟩ · intro y z rw [one_smul, one_smul] · clear x intro x hx x' hx' y z rw [mul_smul, mul_smul, hs x hx, hx'] @[to_additive] theorem SMulCommClass.of_mclosure_eq_top {N α} [Monoid M] [SMul N α] [MulAction M α] {s : Set M} (htop : Submonoid.closure s = ⊤) (hs : ∀ x ∈ s, ∀ (y : N) (z : α), x • y • z = y • x • z) : SMulCommClass M N α := by refine ⟨fun x => Submonoid.induction_of_closure_eq_top_left htop x ?_ ?_⟩ · intro y z rw [one_smul, one_smul] · clear x intro x hx x' hx' y z rw [mul_smul, mul_smul, hx', hs x hx] namespace Submonoid variable {N : Type*} [CommMonoid N] open MonoidHom @[to_additive] theorem sup_eq_range (s t : Submonoid N) : s ⊔ t = mrange (s.subtype.coprod t.subtype) := by rw [mrange_eq_map, ← mrange_inl_sup_mrange_inr, map_sup, map_mrange, coprod_comp_inl, map_mrange, coprod_comp_inr, range_subtype, range_subtype] @[to_additive] theorem mem_sup {s t : Submonoid N} {x : N} : x ∈ s ⊔ t ↔ ∃ y ∈ s, ∃ z ∈ t, y * z = x := by simp only [sup_eq_range, mem_mrange, coprod_apply, coe_subtype, Prod.exists, Subtype.exists, exists_prop] end Submonoid namespace AddSubmonoid variable [AddMonoid A] open Set theorem closure_singleton_eq (x : A) : closure ({x} : Set A) = AddMonoidHom.mrange (multiplesHom A x) := closure_eq_of_le (Set.singleton_subset_iff.2 ⟨1, one_nsmul x⟩) fun _ ⟨_n, hn⟩ => hn ▸ nsmul_mem (subset_closure <| Set.mem_singleton _) _ /-- The `AddSubmonoid` generated by an element of an `AddMonoid` equals the set of natural number multiples of the element. -/ theorem mem_closure_singleton {x y : A} : y ∈ closure ({x} : Set A) ↔ ∃ n : ℕ, n • x = y := by rw [closure_singleton_eq, AddMonoidHom.mem_mrange]; rfl theorem closure_singleton_zero : closure ({0} : Set A) = ⊥ := by simp [eq_bot_iff_forall, mem_closure_singleton, nsmul_zero] /-- The additive submonoid generated by an element. -/ def multiples (x : A) : AddSubmonoid A := AddSubmonoid.copy (AddMonoidHom.mrange (multiplesHom A x)) (Set.range (fun i => i • x : ℕ → A)) <| Set.ext fun n => exists_congr fun i => by simp attribute [to_additive existing] Submonoid.powers attribute [to_additive (attr := simp)] Submonoid.mem_powers attribute [to_additive (attr := norm_cast)] Submonoid.coe_powers attribute [to_additive] Submonoid.mem_powers_iff attribute [to_additive] Submonoid.decidableMemPowers attribute [to_additive] Submonoid.fintypePowers attribute [to_additive] Submonoid.powers_eq_closure attribute [to_additive] Submonoid.powers_le attribute [to_additive (attr := simp)] Submonoid.powers_one attribute [to_additive "The additive submonoid generated by an element is an additive group if that element has finite order."] Submonoid.groupPowers end AddSubmonoid /-! Lemmas about additive closures of `Subsemigroup`. -/ namespace MulMemClass variable {R : Type*} [NonUnitalNonAssocSemiring R] [SetLike M R] [MulMemClass M R] {S : M} {a b : R} /-- The product of an element of the additive closure of a multiplicative subsemigroup `M` and an element of `M` is contained in the additive closure of `M`. -/ theorem mul_right_mem_add_closure (ha : a ∈ AddSubmonoid.closure (S : Set R)) (hb : b ∈ S) : a * b ∈ AddSubmonoid.closure (S : Set R) := by revert b apply @AddSubmonoid.closure_induction _ _ _ (fun z => ∀ (b : R), b ∈ S → z * b ∈ AddSubmonoid.closure S) _ ha <;> clear ha a · exact fun r hr b hb => AddSubmonoid.mem_closure.mpr fun y hy => hy (mul_mem hr hb) · exact fun b _ => by simp only [zero_mul, (AddSubmonoid.closure (S : Set R)).zero_mem] · simp_rw [add_mul] exact fun r s hr hs b hb => (AddSubmonoid.closure (S : Set R)).add_mem (hr _ hb) (hs _ hb) /-- The product of two elements of the additive closure of a submonoid `M` is an element of the additive closure of `M`. -/ theorem mul_mem_add_closure (ha : a ∈ AddSubmonoid.closure (S : Set R)) (hb : b ∈ AddSubmonoid.closure (S : Set R)) : a * b ∈ AddSubmonoid.closure (S : Set R) := by revert a apply @AddSubmonoid.closure_induction _ _ _ (fun z => ∀ {a : R}, a ∈ AddSubmonoid.closure ↑S → a * z ∈ AddSubmonoid.closure ↑S) _ hb <;> clear hb b · exact fun r hr b hb => MulMemClass.mul_right_mem_add_closure hb hr · exact fun _ => by simp only [mul_zero, (AddSubmonoid.closure (S : Set R)).zero_mem] · simp_rw [mul_add] exact fun r s hr hs b hb => (AddSubmonoid.closure (S : Set R)).add_mem (hr hb) (hs hb) /-- The product of an element of `S` and an element of the additive closure of a multiplicative submonoid `S` is contained in the additive closure of `S`. -/ theorem mul_left_mem_add_closure (ha : a ∈ S) (hb : b ∈ AddSubmonoid.closure (S : Set R)) : a * b ∈ AddSubmonoid.closure (S : Set R) := mul_mem_add_closure (AddSubmonoid.mem_closure.mpr fun _sT hT => hT ha) hb end MulMemClass namespace Submonoid /-- An element is in the closure of a two-element set if it is a linear combination of those two elements. -/ @[to_additive "An element is in the closure of a two-element set if it is a linear combination of those two elements."] theorem mem_closure_pair {A : Type*} [CommMonoid A] (a b c : A) : c ∈ Submonoid.closure ({a, b} : Set A) ↔ ∃ m n : ℕ, a ^ m * b ^ n = c := by rw [← Set.singleton_union, Submonoid.closure_union, mem_sup] simp_rw [mem_closure_singleton, exists_exists_eq_and] end Submonoid section mul_add theorem ofMul_image_powers_eq_multiples_ofMul [Monoid M] {x : M} : Additive.ofMul '' (Submonoid.powers x : Set M) = AddSubmonoid.multiples (Additive.ofMul x) := by ext constructor · rintro ⟨y, ⟨n, hy1⟩, hy2⟩ use n simpa [← ofMul_pow, hy1] · rintro ⟨n, hn⟩ refine ⟨x ^ n, ⟨n, rfl⟩, ?_⟩ rwa [ofMul_pow] theorem ofAdd_image_multiples_eq_powers_ofAdd [AddMonoid A] {x : A} : Multiplicative.ofAdd '' (AddSubmonoid.multiples x : Set A) = Submonoid.powers (Multiplicative.ofAdd x) := by symm rw [Equiv.eq_image_iff_symm_image_eq] exact ofMul_image_powers_eq_multiples_ofMul end mul_add /-- The submonoid of primal elements in a cancellative commutative monoid with zero. -/ def Submonoid.isPrimal (α) [CancelCommMonoidWithZero α] : Submonoid α where carrier := {a | IsPrimal a} mul_mem' := IsPrimal.mul one_mem' := isUnit_one.isPrimal
Algebra\Group\Submonoid\MulOpposite.lean
/- Copyright (c) 2023 Eric Wieser. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Eric Wieser, Jujian Zhang -/ import Mathlib.Algebra.Group.Opposite import Mathlib.Algebra.Group.Submonoid.Basic /-! # Submonoid of opposite monoids For every monoid `M`, we construct an equivalence between submonoids of `M` and that of `Mᵐᵒᵖ`. -/ assert_not_exists MonoidWithZero variable {ι : Sort*} {M : Type*} [MulOneClass M] namespace Submonoid /-- Pull a submonoid back to an opposite submonoid along `MulOpposite.unop`-/ @[to_additive (attr := simps) "Pull an additive submonoid back to an opposite submonoid along `AddOpposite.unop`"] protected def op (x : Submonoid M) : Submonoid Mᵐᵒᵖ where carrier := MulOpposite.unop ⁻¹' x mul_mem' ha hb := x.mul_mem hb ha one_mem' := Submonoid.one_mem' _ @[to_additive (attr := simp)] theorem mem_op {x : Mᵐᵒᵖ} {S : Submonoid M} : x ∈ S.op ↔ x.unop ∈ S := Iff.rfl /-- Pull an opposite submonoid back to a submonoid along `MulOpposite.op`-/ @[to_additive (attr := simps) "Pull an opposite additive submonoid back to a submonoid along `AddOpposite.op`"] protected def unop (x : Submonoid Mᵐᵒᵖ) : Submonoid M where carrier := MulOpposite.op ⁻¹' x mul_mem' ha hb := x.mul_mem hb ha one_mem' := Submonoid.one_mem' _ @[to_additive (attr := simp)] theorem mem_unop {x : M} {S : Submonoid Mᵐᵒᵖ} : x ∈ S.unop ↔ MulOpposite.op x ∈ S := Iff.rfl @[to_additive (attr := simp)] theorem unop_op (S : Submonoid M) : S.op.unop = S := rfl @[to_additive (attr := simp)] theorem op_unop (S : Submonoid Mᵐᵒᵖ) : S.unop.op = S := rfl /-! ### Lattice results -/ @[to_additive] theorem op_le_iff {S₁ : Submonoid M} {S₂ : Submonoid Mᵐᵒᵖ} : S₁.op ≤ S₂ ↔ S₁ ≤ S₂.unop := MulOpposite.op_surjective.forall @[to_additive] theorem le_op_iff {S₁ : Submonoid Mᵐᵒᵖ} {S₂ : Submonoid M} : S₁ ≤ S₂.op ↔ S₁.unop ≤ S₂ := MulOpposite.op_surjective.forall @[to_additive (attr := simp)] theorem op_le_op_iff {S₁ S₂ : Submonoid M} : S₁.op ≤ S₂.op ↔ S₁ ≤ S₂ := MulOpposite.op_surjective.forall @[to_additive (attr := simp)] theorem unop_le_unop_iff {S₁ S₂ : Submonoid Mᵐᵒᵖ} : S₁.unop ≤ S₂.unop ↔ S₁ ≤ S₂ := MulOpposite.unop_surjective.forall /-- A submonoid `H` of `G` determines a submonoid `H.op` of the opposite group `Gᵐᵒᵖ`. -/ @[to_additive (attr := simps) "A additive submonoid `H` of `G` determines an additive submonoid `H.op` of the opposite group `Gᵐᵒᵖ`."] def opEquiv : Submonoid M ≃o Submonoid Mᵐᵒᵖ where toFun := Submonoid.op invFun := Submonoid.unop left_inv := unop_op right_inv := op_unop map_rel_iff' := op_le_op_iff @[to_additive (attr := simp)] theorem op_bot : (⊥ : Submonoid M).op = ⊥ := opEquiv.map_bot @[to_additive (attr := simp)] theorem unop_bot : (⊥ : Submonoid Mᵐᵒᵖ).unop = ⊥ := opEquiv.symm.map_bot @[to_additive (attr := simp)] theorem op_top : (⊤ : Submonoid M).op = ⊤ := opEquiv.map_top @[to_additive (attr := simp)] theorem unop_top : (⊤ : Submonoid Mᵐᵒᵖ).unop = ⊤ := opEquiv.symm.map_top @[to_additive] theorem op_sup (S₁ S₂ : Submonoid M) : (S₁ ⊔ S₂).op = S₁.op ⊔ S₂.op := opEquiv.map_sup _ _ @[to_additive] theorem unop_sup (S₁ S₂ : Submonoid Mᵐᵒᵖ) : (S₁ ⊔ S₂).unop = S₁.unop ⊔ S₂.unop := opEquiv.symm.map_sup _ _ @[to_additive] theorem op_inf (S₁ S₂ : Submonoid M) : (S₁ ⊓ S₂).op = S₁.op ⊓ S₂.op := opEquiv.map_inf _ _ @[to_additive] theorem unop_inf (S₁ S₂ : Submonoid Mᵐᵒᵖ) : (S₁ ⊓ S₂).unop = S₁.unop ⊓ S₂.unop := opEquiv.symm.map_inf _ _ @[to_additive] theorem op_sSup (S : Set (Submonoid M)) : (sSup S).op = sSup (.unop ⁻¹' S) := opEquiv.map_sSup_eq_sSup_symm_preimage _ @[to_additive] theorem unop_sSup (S : Set (Submonoid Mᵐᵒᵖ)) : (sSup S).unop = sSup (.op ⁻¹' S) := opEquiv.symm.map_sSup_eq_sSup_symm_preimage _ @[to_additive] theorem op_sInf (S : Set (Submonoid M)) : (sInf S).op = sInf (.unop ⁻¹' S) := opEquiv.map_sInf_eq_sInf_symm_preimage _ @[to_additive] theorem unop_sInf (S : Set (Submonoid Mᵐᵒᵖ)) : (sInf S).unop = sInf (.op ⁻¹' S) := opEquiv.symm.map_sInf_eq_sInf_symm_preimage _ @[to_additive] theorem op_iSup (S : ι → Submonoid M) : (iSup S).op = ⨆ i, (S i).op := opEquiv.map_iSup _ @[to_additive] theorem unop_iSup (S : ι → Submonoid Mᵐᵒᵖ) : (iSup S).unop = ⨆ i, (S i).unop := opEquiv.symm.map_iSup _ @[to_additive] theorem op_iInf (S : ι → Submonoid M) : (iInf S).op = ⨅ i, (S i).op := opEquiv.map_iInf _ @[to_additive] theorem unop_iInf (S : ι → Submonoid Mᵐᵒᵖ) : (iInf S).unop = ⨅ i, (S i).unop := opEquiv.symm.map_iInf _ @[to_additive] theorem op_closure (s : Set M) : (closure s).op = closure (MulOpposite.unop ⁻¹' s) := by simp_rw [closure, op_sInf, Set.preimage_setOf_eq, Submonoid.unop_coe] congr with a exact MulOpposite.unop_surjective.forall @[to_additive] theorem unop_closure (s : Set Mᵐᵒᵖ) : (closure s).unop = closure (MulOpposite.op ⁻¹' s) := by simp_rw [closure, unop_sInf, Set.preimage_setOf_eq, Submonoid.op_coe] congr with a exact MulOpposite.op_surjective.forall /-- Bijection between a submonoid `H` and its opposite. -/ @[to_additive (attr := simps!) "Bijection between an additive submonoid `H` and its opposite."] def equivOp (H : Submonoid M) : H ≃ H.op := MulOpposite.opEquiv.subtypeEquiv fun _ => Iff.rfl end Submonoid
Algebra\Group\Submonoid\Operations.lean
/- Copyright (c) 2018 Johannes Hölzl. All rights reserved. Released under Apache 2.0 license as described in the file LICENSE. Authors: Johannes Hölzl, Kenny Lau, Johan Commelin, Mario Carneiro, Kevin Buzzard, Amelia Livingston, Yury Kudryashov -/ import Mathlib.Algebra.Group.Action.Defs import Mathlib.Algebra.Group.Nat import Mathlib.Algebra.Group.Submonoid.Basic import Mathlib.Algebra.Group.Subsemigroup.Operations /-! # Operations on `Submonoid`s In this file we define various operations on `Submonoid`s and `MonoidHom`s. ## Main definitions ### Conversion between multiplicative and additive definitions * `Submonoid.toAddSubmonoid`, `Submonoid.toAddSubmonoid'`, `AddSubmonoid.toSubmonoid`, `AddSubmonoid.toSubmonoid'`: convert between multiplicative and additive submonoids of `M`, `Multiplicative M`, and `Additive M`. These are stated as `OrderIso`s. ### (Commutative) monoid structure on a submonoid * `Submonoid.toMonoid`, `Submonoid.toCommMonoid`: a submonoid inherits a (commutative) monoid structure. ### Group actions by submonoids * `Submonoid.MulAction`, `Submonoid.DistribMulAction`: a submonoid inherits (distributive) multiplicative actions. ### Operations on submonoids * `Submonoid.comap`: preimage of a submonoid under a monoid homomorphism as a submonoid of the domain; * `Submonoid.map`: image of a submonoid under a monoid homomorphism as a submonoid of the codomain; * `Submonoid.prod`: product of two submonoids `s : Submonoid M` and `t : Submonoid N` as a submonoid of `M × N`; ### Monoid homomorphisms between submonoid * `Submonoid.subtype`: embedding of a submonoid into the ambient monoid. * `Submonoid.inclusion`: given two submonoids `S`, `T` such that `S ≤ T`, `S.inclusion T` is the inclusion of `S` into `T` as a monoid homomorphism; * `MulEquiv.submonoidCongr`: converts a proof of `S = T` into a monoid isomorphism between `S` and `T`. * `Submonoid.prodEquiv`: monoid isomorphism between `s.prod t` and `s × t`; ### Operations on `MonoidHom`s * `MonoidHom.mrange`: range of a monoid homomorphism as a submonoid of the codomain; * `MonoidHom.mker`: kernel of a monoid homomorphism as a submonoid of the domain; * `MonoidHom.restrict`: restrict a monoid homomorphism to a submonoid; * `MonoidHom.codRestrict`: restrict the codomain of a monoid homomorphism to a submonoid; * `MonoidHom.mrangeRestrict`: restrict a monoid homomorphism to its range; ## Tags submonoid, range, product, map, comap -/ assert_not_exists MonoidWithZero variable {M N P : Type*} [MulOneClass M] [MulOneClass N] [MulOneClass P] (S : Submonoid M) /-! ### Conversion to/from `Additive`/`Multiplicative` -/ section /-- Submonoids of monoid `M` are isomorphic to additive submonoids of `Additive M`. -/ @[simps] def Submonoid.toAddSubmonoid : Submonoid M ≃o AddSubmonoid (Additive M) where toFun S := { carrier := Additive.toMul ⁻¹' S zero_mem' := S.one_mem' add_mem' := fun ha hb => S.mul_mem' ha hb } invFun S := { carrier := Additive.ofMul ⁻¹' S one_mem' := S.zero_mem' mul_mem' := fun ha hb => S.add_mem' ha hb} left_inv x := by cases x; rfl right_inv x := by cases x; rfl map_rel_iff' := Iff.rfl /-- Additive submonoids of an additive monoid `Additive M` are isomorphic to submonoids of `M`. -/ abbrev AddSubmonoid.toSubmonoid' : AddSubmonoid (Additive M) ≃o Submonoid M := Submonoid.toAddSubmonoid.symm theorem Submonoid.toAddSubmonoid_closure (S : Set M) : Submonoid.toAddSubmonoid (Submonoid.closure S) = AddSubmonoid.closure (Additive.toMul ⁻¹' S) := le_antisymm (Submonoid.toAddSubmonoid.le_symm_apply.1 <| Submonoid.closure_le.2 (AddSubmonoid.subset_closure (M := Additive M))) (AddSubmonoid.closure_le.2 <| Submonoid.subset_closure (M := M)) theorem AddSubmonoid.toSubmonoid'_closure (S : Set (Additive M)) : AddSubmonoid.toSubmonoid' (AddSubmonoid.closure S) = Submonoid.closure (Multiplicative.ofAdd ⁻¹' S) := le_antisymm (AddSubmonoid.toSubmonoid'.le_symm_apply.1 <| AddSubmonoid.closure_le.2 (Submonoid.subset_closure (M := M))) (Submonoid.closure_le.2 <| AddSubmonoid.subset_closure (M := Additive M)) end section variable {A : Type*} [AddZeroClass A] /-- Additive submonoids of an additive monoid `A` are isomorphic to multiplicative submonoids of `Multiplicative A`. -/ @[simps] def AddSubmonoid.toSubmonoid : AddSubmonoid A ≃o Submonoid (Multiplicative A) where toFun S := { carrier := Multiplicative.toAdd ⁻¹' S one_mem' := S.zero_mem' mul_mem' := fun ha hb => S.add_mem' ha hb } invFun S := { carrier := Multiplicative.ofAdd ⁻¹' S zero_mem' := S.one_mem' add_mem' := fun ha hb => S.mul_mem' ha hb} left_inv x := by cases x; rfl right_inv x := by cases x; rfl map_rel_iff' := Iff.rfl /-- Submonoids of a monoid `Multiplicative A` are isomorphic to additive submonoids of `A`. -/ abbrev Submonoid.toAddSubmonoid' : Submonoid (Multiplicative A) ≃o AddSubmonoid A := AddSubmonoid.toSubmonoid.symm theorem AddSubmonoid.toSubmonoid_closure (S : Set A) : (AddSubmonoid.toSubmonoid) (AddSubmonoid.closure S) = Submonoid.closure (Multiplicative.toAdd ⁻¹' S) := le_antisymm (AddSubmonoid.toSubmonoid.to_galoisConnection.l_le <| AddSubmonoid.closure_le.2 <| Submonoid.subset_closure (M := Multiplicative A)) (Submonoid.closure_le.2 <| AddSubmonoid.subset_closure (M := A)) theorem Submonoid.toAddSubmonoid'_closure (S : Set (Multiplicative A)) : Submonoid.toAddSubmonoid' (Submonoid.closure S) = AddSubmonoid.closure (Additive.ofMul ⁻¹' S) := le_antisymm (Submonoid.toAddSubmonoid'.to_galoisConnection.l_le <| Submonoid.closure_le.2 <| AddSubmonoid.subset_closure (M := A)) (AddSubmonoid.closure_le.2 <| Submonoid.subset_closure (M := Multiplicative A)) end namespace Submonoid variable {F : Type*} [FunLike F M N] [mc : MonoidHomClass F M N] open Set /-! ### `comap` and `map` -/ /-- The preimage of a submonoid along a monoid homomorphism is a submonoid. -/ @[to_additive "The preimage of an `AddSubmonoid` along an `AddMonoid` homomorphism is an `AddSubmonoid`."] def comap (f : F) (S : Submonoid N) : Submonoid M where carrier := f ⁻¹' S one_mem' := show f 1 ∈ S by rw [map_one]; exact S.one_mem mul_mem' ha hb := show f (_ * _) ∈ S by rw [map_mul]; exact S.mul_mem ha hb @[to_additive (attr := simp)] theorem coe_comap (S : Submonoid N) (f : F) : (S.comap f : Set M) = f ⁻¹' S := rfl @[to_additive (attr := simp)] theorem mem_comap {S : Submonoid N} {f : F} {x : M} : x ∈ S.comap f ↔ f x ∈ S := Iff.rfl @[to_additive] theorem comap_comap (S : Submonoid P) (g : N →* P) (f : M →* N) : (S.comap g).comap f = S.comap (g.comp f) := rfl @[to_additive (attr := simp)] theorem comap_id (S : Submonoid P) : S.comap (MonoidHom.id P) = S := ext (by simp) /-- The image of a submonoid along a monoid homomorphism is a submonoid. -/ @[to_additive "The image of an `AddSubmonoid` along an `AddMonoid` homomorphism is an `AddSubmonoid`."] def map (f : F) (S : Submonoid M) : Submonoid N where carrier := f '' S one_mem' := ⟨1, S.one_mem, map_one f⟩ mul_mem' := by rintro _ _ ⟨x, hx, rfl⟩ ⟨y, hy, rfl⟩ exact ⟨x * y, S.mul_mem hx hy, by rw [map_mul]⟩ @[to_additive (attr := simp)] theorem coe_map (f : F) (S : Submonoid M) : (S.map f : Set N) = f '' S := rfl @[to_additive (attr := simp)] theorem mem_map {f : F} {S : Submonoid M} {y : N} : y ∈ S.map f ↔ ∃ x ∈ S, f x = y := Iff.rfl @[to_additive] theorem mem_map_of_mem (f : F) {S : Submonoid M} {x : M} (hx : x ∈ S) : f x ∈ S.map f := mem_image_of_mem f hx @[to_additive] theorem apply_coe_mem_map (f : F) (S : Submonoid M) (x : S) : f x ∈ S.map f := mem_map_of_mem f x.2 @[to_additive] theorem map_map (g : N →* P) (f : M →* N) : (S.map f).map g = S.map (g.comp f) := SetLike.coe_injective <| image_image _ _ _ -- The simpNF linter says that the LHS can be simplified via `Submonoid.mem_map`. -- However this is a higher priority lemma. -- https://github.com/leanprover/std4/issues/207 @[to_additive (attr := simp 1100, nolint simpNF)] theorem mem_map_iff_mem {f : F} (hf : Function.Injective f) {S : Submonoid M} {x : M} : f x ∈ S.map f ↔ x ∈ S := hf.mem_set_image @[to_additive] theorem map_le_iff_le_comap {f : F} {S : Submonoid M} {T : Submonoid N} : S.map f ≤ T ↔ S ≤ T.comap f := image_subset_iff @[to_additive] theorem gc_map_comap (f : F) : GaloisConnection (map f) (comap f) := fun _ _ => map_le_iff_le_comap @[to_additive] theorem map_le_of_le_comap {T : Submonoid N} {f : F} : S ≤ T.comap f → S.map f ≤ T := (gc_map_comap f).l_le @[to_additive] theorem le_comap_of_map_le {T : Submonoid N} {f : F} : S.map f ≤ T → S ≤ T.comap f := (gc_map_comap f).le_u @[to_additive] theorem le_comap_map {f : F} : S ≤ (S.map f).comap f := (gc_map_comap f).le_u_l _ @[to_additive] theorem map_comap_le {S : Submonoid N} {f : F} : (S.comap f).map f ≤ S := (gc_map_comap f).l_u_le _ @[to_additive] theorem monotone_map {f : F} : Monotone (map f) := (gc_map_comap f).monotone_l @[to_additive] theorem monotone_comap {f : F} : Monotone (comap f) := (gc_map_comap f).monotone_u @[to_additive (attr := simp)] theorem map_comap_map {f : F} : ((S.map f).comap f).map f = S.map f := (gc_map_comap f).l_u_l_eq_l _ @[to_additive (attr := simp)] theorem comap_map_comap {S : Submonoid N} {f : F} : ((S.comap f).map f).comap f = S.comap f := (gc_map_comap f).u_l_u_eq_u _ @[to_additive] theorem map_sup (S T : Submonoid M) (f : F) : (S ⊔ T).map f = S.map f ⊔ T.map f := (gc_map_comap f : GaloisConnection (map f) (comap f)).l_sup @[to_additive] theorem map_iSup {ι : Sort*} (f : F) (s : ι → Submonoid M) : (iSup s).map f = ⨆ i, (s i).map f := (gc_map_comap f : GaloisConnection (map f) (comap f)).l_iSup @[to_additive] theorem comap_inf (S T : Submonoid N) (f : F) : (S ⊓ T).comap f = S.comap f ⊓ T.comap f := (gc_map_comap f : GaloisConnection (map f) (comap f)).u_inf @[to_additive] theorem comap_iInf {ι : Sort*} (f : F) (s : ι → Submonoid N) : (iInf s).comap f = ⨅ i, (s i).comap f := (gc_map_comap f : GaloisConnection (map f) (comap f)).u_iInf @[to_additive (attr := simp)] theorem map_bot (f : F) : (⊥ : Submonoid M).map f = ⊥ := (gc_map_comap f).l_bot @[to_additive (attr := simp)] theorem comap_top (f : F) : (⊤ : Submonoid N).comap f = ⊤ := (gc_map_comap f).u_top @[to_additive (attr := simp)] theorem map_id (S : Submonoid M) : S.map (MonoidHom.id M) = S := ext fun _ => ⟨fun ⟨_, h, rfl⟩ => h, fun h => ⟨_, h, rfl⟩⟩ section GaloisCoinsertion variable {ι : Type*} {f : F} /-- `map f` and `comap f` form a `GaloisCoinsertion` when `f` is injective. -/ @[to_additive " `map f` and `comap f` form a `GaloisCoinsertion` when `f` is injective. "] def gciMapComap (hf : Function.Injective f) : GaloisCoinsertion (map f) (comap f) := (gc_map_comap f).toGaloisCoinsertion fun S x => by simp [mem_comap, mem_map, hf.eq_iff] variable (hf : Function.Injective f) @[to_additive] theorem comap_map_eq_of_injective (S : Submonoid M) : (S.map f).comap f = S := (gciMapComap hf).u_l_eq _ @[to_additive] theorem comap_surjective_of_injective : Function.Surjective (comap f) := (gciMapComap hf).u_surjective @[to_additive] theorem map_injective_of_injective : Function.Injective (map f) := (gciMapComap hf).l_injective @[to_additive] theorem comap_inf_map_of_injective (S T : Submonoid M) : (S.map f ⊓ T.map f).comap f = S ⊓ T := (gciMapComap hf).u_inf_l _ _ @[to_additive] theorem comap_iInf_map_of_injective (S : ι → Submonoid M) : (⨅ i, (S i).map f).comap f = iInf S := (gciMapComap hf).u_iInf_l _ @[to_additive] theorem comap_sup_map_of_injective (S T : Submonoid M) : (S.map f ⊔ T.map f).comap f = S ⊔ T := (gciMapComap hf).u_sup_l _ _ @[to_additive] theorem comap_iSup_map_of_injective (S : ι → Submonoid M) : (⨆ i, (S i).map f).comap f = iSup S := (gciMapComap hf).u_iSup_l _ @[to_additive] theorem map_le_map_iff_of_injective {S T : Submonoid M} : S.map f ≤ T.map f ↔ S ≤ T := (gciMapComap hf).l_le_l_iff @[to_additive] theorem map_strictMono_of_injective : StrictMono (map f) := (gciMapComap hf).strictMono_l end GaloisCoinsertion section GaloisInsertion variable {ι : Type*} {f : F} (hf : Function.Surjective f) /-- `map f` and `comap f` form a `GaloisInsertion` when `f` is surjective. -/ @[to_additive " `map f` and `comap f` form a `GaloisInsertion` when `f` is surjective. "] def giMapComap : GaloisInsertion (map f) (comap f) := (gc_map_comap f).toGaloisInsertion fun S x h => let ⟨y, hy⟩ := hf x mem_map.2 ⟨y, by simp [hy, h]⟩ @[to_additive] theorem map_comap_eq_of_surjective (S : Submonoid N) : (S.comap f).map f = S := (giMapComap hf).l_u_eq _ @[to_additive] theorem map_surjective_of_surjective : Function.Surjective (map f) := (giMapComap hf).l_surjective @[to_additive] theorem comap_injective_of_surjective : Function.Injective (comap f) := (giMapComap hf).u_injective @[to_additive] theorem map_inf_comap_of_surjective (S T : Submonoid N) : (S.comap f ⊓ T.comap f).map f = S ⊓ T := (giMapComap hf).l_inf_u _ _ @[to_additive] theorem map_iInf_comap_of_surjective (S : ι → Submonoid N) : (⨅ i, (S i).comap f).map f = iInf S := (giMapComap hf).l_iInf_u _ @[to_additive] theorem map_sup_comap_of_surjective (S T : Submonoid N) : (S.comap f ⊔ T.comap f).map f = S ⊔ T := (giMapComap hf).l_sup_u _ _ @[to_additive] theorem map_iSup_comap_of_surjective (S : ι → Submonoid N) : (⨆ i, (S i).comap f).map f = iSup S := (giMapComap hf).l_iSup_u _ @[to_additive] theorem comap_le_comap_iff_of_surjective {S T : Submonoid N} : S.comap f ≤ T.comap f ↔ S ≤ T := (giMapComap hf).u_le_u_iff @[to_additive] theorem comap_strictMono_of_surjective : StrictMono (comap f) := (giMapComap hf).strictMono_u end GaloisInsertion end Submonoid namespace OneMemClass variable {A M₁ : Type*} [SetLike A M₁] [One M₁] [hA : OneMemClass A M₁] (S' : A) /-- A submonoid of a monoid inherits a 1. -/ @[to_additive "An `AddSubmonoid` of an `AddMonoid` inherits a zero."] instance one : One S' := ⟨⟨1, OneMemClass.one_mem S'⟩⟩ @[to_additive (attr := simp, norm_cast)] theorem coe_one : ((1 : S') : M₁) = 1 := rfl variable {S'} @[to_additive (attr := simp, norm_cast)] theorem coe_eq_one {x : S'} : (↑x : M₁) = 1 ↔ x = 1 := (Subtype.ext_iff.symm : (x : M₁) = (1 : S') ↔ x = 1) variable (S') @[to_additive] theorem one_def : (1 : S') = ⟨1, OneMemClass.one_mem S'⟩ := rfl end OneMemClass variable {A : Type*} [SetLike A M] [hA : SubmonoidClass A M] (S' : A) /-- An `AddSubmonoid` of an `AddMonoid` inherits a scalar multiplication. -/ instance AddSubmonoidClass.nSMul {M} [AddMonoid M] {A : Type*} [SetLike A M] [AddSubmonoidClass A M] (S : A) : SMul ℕ S := ⟨fun n a => ⟨n • a.1, nsmul_mem a.2 n⟩⟩ namespace SubmonoidClass /-- A submonoid of a monoid inherits a power operator. -/ instance nPow {M} [Monoid M] {A : Type*} [SetLike A M] [SubmonoidClass A M] (S : A) : Pow S ℕ := ⟨fun a n => ⟨a.1 ^ n, pow_mem a.2 n⟩⟩ attribute [to_additive existing nSMul] nPow @[to_additive (attr := simp, norm_cast)] theorem coe_pow {M} [Monoid M] {A : Type*} [SetLike A M] [SubmonoidClass A M] {S : A} (x : S) (n : ℕ) : ↑(x ^ n) = (x : M) ^ n := rfl @[to_additive (attr := simp)] theorem mk_pow {M} [Monoid M] {A : Type*} [SetLike A M] [SubmonoidClass A M] {S : A} (x : M) (hx : x ∈ S) (n : ℕ) : (⟨x, hx⟩ : S) ^ n = ⟨x ^ n, pow_mem hx n⟩ := rfl -- Prefer subclasses of `Monoid` over subclasses of `SubmonoidClass`. /-- A submonoid of a unital magma inherits a unital magma structure. -/ @[to_additive "An `AddSubmonoid` of a unital additive magma inherits a unital additive magma structure."] instance (priority := 75) toMulOneClass {M : Type*} [MulOneClass M] {A : Type*} [SetLike A M] [SubmonoidClass A M] (S : A) : MulOneClass S := Subtype.coe_injective.mulOneClass (↑) rfl (fun _ _ => rfl) -- Prefer subclasses of `Monoid` over subclasses of `SubmonoidClass`. /-- A submonoid of a monoid inherits a monoid structure. -/ @[to_additive "An `AddSubmonoid` of an `AddMonoid` inherits an `AddMonoid` structure."] instance (priority := 75) toMonoid {M : Type*} [Monoid M] {A : Type*} [SetLike A M] [SubmonoidClass A M] (S : A) : Monoid S := Subtype.coe_injective.monoid (↑) rfl (fun _ _ => rfl) (fun _ _ => rfl) -- Prefer subclasses of `Monoid` over subclasses of `SubmonoidClass`. /-- A submonoid of a `CommMonoid` is a `CommMonoid`. -/ @[to_additive "An `AddSubmonoid` of an `AddCommMonoid` is an `AddCommMonoid`."] instance (priority := 75) toCommMonoid {M} [CommMonoid M] {A : Type*} [SetLike A M] [SubmonoidClass A M] (S : A) : CommMonoid S := Subtype.coe_injective.commMonoid (↑) rfl (fun _ _ => rfl) fun _ _ => rfl /-- The natural monoid hom from a submonoid of monoid `M` to `M`. -/ @[to_additive "The natural monoid hom from an `AddSubmonoid` of `AddMonoid` `M` to `M`."] def subtype : S' →* M where toFun := Subtype.val; map_one' := rfl; map_mul' _ _ := by simp @[to_additive (attr := simp)] theorem coe_subtype : (SubmonoidClass.subtype S' : S' → M) = Subtype.val := rfl end SubmonoidClass namespace Submonoid /-- A submonoid of a monoid inherits a multiplication. -/ @[to_additive "An `AddSubmonoid` of an `AddMonoid` inherits an addition."] instance mul : Mul S := ⟨fun a b => ⟨a.1 * b.1, S.mul_mem a.2 b.2⟩⟩ /-- A submonoid of a monoid inherits a 1. -/ @[to_additive "An `AddSubmonoid` of an `AddMonoid` inherits a zero."] instance one : One S := ⟨⟨_, S.one_mem⟩⟩ @[to_additive (attr := simp, norm_cast)] theorem coe_mul (x y : S) : (↑(x * y) : M) = ↑x * ↑y := rfl @[to_additive (attr := simp, norm_cast)] theorem coe_one : ((1 : S) : M) = 1 := rfl @[to_additive (attr := simp)] lemma mk_eq_one {a : M} {ha} : (⟨a, ha⟩ : S) = 1 ↔ a = 1 := by simp [← SetLike.coe_eq_coe] @[to_additive (attr := simp)] theorem mk_mul_mk (x y : M) (hx : x ∈ S) (hy : y ∈ S) : (⟨x, hx⟩ : S) * ⟨y, hy⟩ = ⟨x * y, S.mul_mem hx hy⟩ := rfl @[to_additive] theorem mul_def (x y : S) : x * y = ⟨x * y, S.mul_mem x.2 y.2⟩ := rfl @[to_additive] theorem one_def : (1 : S) = ⟨1, S.one_mem⟩ := rfl /-- A submonoid of a unital magma inherits a unital magma structure. -/ @[to_additive "An `AddSubmonoid` of a unital additive magma inherits a unital additive magma structure."] instance toMulOneClass {M : Type*} [MulOneClass M] (S : Submonoid M) : MulOneClass S := Subtype.coe_injective.mulOneClass (↑) rfl fun _ _ => rfl @[to_additive] protected theorem pow_mem {M : Type*} [Monoid M] (S : Submonoid M) {x : M} (hx : x ∈ S) (n : ℕ) : x ^ n ∈ S := pow_mem hx n -- Porting note: coe_pow removed, syntactic tautology /-- A submonoid of a monoid inherits a monoid structure. -/ @[to_additive "An `AddSubmonoid` of an `AddMonoid` inherits an `AddMonoid` structure."] instance toMonoid {M : Type*} [Monoid M] (S : Submonoid M) : Monoid S := Subtype.coe_injective.monoid (↑) rfl (fun _ _ => rfl) fun _ _ => rfl /-- A submonoid of a `CommMonoid` is a `CommMonoid`. -/ @[to_additive "An `AddSubmonoid` of an `AddCommMonoid` is an `AddCommMonoid`."] instance toCommMonoid {M} [CommMonoid M] (S : Submonoid M) : CommMonoid S := Subtype.coe_injective.commMonoid (↑) rfl (fun _ _ => rfl) fun _ _ => rfl /-- The natural monoid hom from a submonoid of monoid `M` to `M`. -/ @[to_additive "The natural monoid hom from an `AddSubmonoid` of `AddMonoid` `M` to `M`."] def subtype : S →* M where toFun := Subtype.val; map_one' := rfl; map_mul' _ _ := by simp @[to_additive (attr := simp)] theorem coe_subtype : ⇑S.subtype = Subtype.val := rfl /-- The top submonoid is isomorphic to the monoid. -/ @[to_additive (attr := simps) "The top additive submonoid is isomorphic to the additive monoid."] def topEquiv : (⊤ : Submonoid M) ≃* M where toFun x := x invFun x := ⟨x, mem_top x⟩ left_inv x := x.eta _ right_inv _ := rfl map_mul' _ _ := rfl @[to_additive (attr := simp)] theorem topEquiv_toMonoidHom : ((topEquiv : _ ≃* M) : _ →* M) = (⊤ : Submonoid M).subtype := rfl /-- A subgroup is isomorphic to its image under an injective function. If you have an isomorphism, use `MulEquiv.submonoidMap` for better definitional equalities. -/ @[to_additive "An additive subgroup is isomorphic to its image under an injective function. If you have an isomorphism, use `AddEquiv.addSubmonoidMap` for better definitional equalities."] noncomputable def equivMapOfInjective (f : M →* N) (hf : Function.Injective f) : S ≃* S.map f := { Equiv.Set.image f S hf with map_mul' := fun _ _ => Subtype.ext (f.map_mul _ _) } @[to_additive (attr := simp)] theorem coe_equivMapOfInjective_apply (f : M →* N) (hf : Function.Injective f) (x : S) : (equivMapOfInjective S f hf x : N) = f x := rfl @[to_additive (attr := simp)] theorem closure_closure_coe_preimage {s : Set M} : closure (((↑) : closure s → M) ⁻¹' s) = ⊤ := eq_top_iff.2 fun x => Subtype.recOn x fun x hx _ => by refine closure_induction' (p := fun y hy ↦ ⟨y, hy⟩ ∈ closure (((↑) : closure s → M) ⁻¹' s)) (fun g hg => subset_closure hg) ?_ (fun g₁ g₂ hg₁ hg₂ => ?_) hx · exact Submonoid.one_mem _ · exact Submonoid.mul_mem _ /-- Given submonoids `s`, `t` of monoids `M`, `N` respectively, `s × t` as a submonoid of `M × N`. -/ @[to_additive prod "Given `AddSubmonoid`s `s`, `t` of `AddMonoid`s `A`, `B` respectively, `s × t` as an `AddSubmonoid` of `A × B`."] def prod (s : Submonoid M) (t : Submonoid N) : Submonoid (M × N) where carrier := s ×ˢ t one_mem' := ⟨s.one_mem, t.one_mem⟩ mul_mem' hp hq := ⟨s.mul_mem hp.1 hq.1, t.mul_mem hp.2 hq.2⟩ @[to_additive coe_prod] theorem coe_prod (s : Submonoid M) (t : Submonoid N) : (s.prod t : Set (M × N)) = (s : Set M) ×ˢ (t : Set N) := rfl @[to_additive mem_prod] theorem mem_prod {s : Submonoid M} {t : Submonoid N} {p : M × N} : p ∈ s.prod t ↔ p.1 ∈ s ∧ p.2 ∈ t := Iff.rfl @[to_additive prod_mono] theorem prod_mono {s₁ s₂ : Submonoid M} {t₁ t₂ : Submonoid N} (hs : s₁ ≤ s₂) (ht : t₁ ≤ t₂) : s₁.prod t₁ ≤ s₂.prod t₂ := Set.prod_mono hs ht @[to_additive prod_top] theorem prod_top (s : Submonoid M) : s.prod (⊤ : Submonoid N) = s.comap (MonoidHom.fst M N) := ext fun x => by simp [mem_prod, MonoidHom.coe_fst] @[to_additive top_prod] theorem top_prod (s : Submonoid N) : (⊤ : Submonoid M).prod s = s.comap (MonoidHom.snd M N) := ext fun x => by simp [mem_prod, MonoidHom.coe_snd] @[to_additive (attr := simp) top_prod_top] theorem top_prod_top : (⊤ : Submonoid M).prod (⊤ : Submonoid N) = ⊤ := (top_prod _).trans <| comap_top _ @[to_additive bot_prod_bot] theorem bot_prod_bot : (⊥ : Submonoid M).prod (⊥ : Submonoid N) = ⊥ := SetLike.coe_injective <| by simp [coe_prod, Prod.one_eq_mk] -- Porting note: to_additive translated the name incorrectly in mathlib 3. /-- The product of submonoids is isomorphic to their product as monoids. -/ @[to_additive prodEquiv "The product of additive submonoids is isomorphic to their product as additive monoids"] def prodEquiv (s : Submonoid M) (t : Submonoid N) : s.prod t ≃* s × t := { (Equiv.Set.prod (s : Set M) (t : Set N)) with map_mul' := fun _ _ => rfl } open MonoidHom @[to_additive] theorem map_inl (s : Submonoid M) : s.map (inl M N) = s.prod ⊥ := ext fun p => ⟨fun ⟨_, hx, hp⟩ => hp ▸ ⟨hx, Set.mem_singleton 1⟩, fun ⟨hps, hp1⟩ => ⟨p.1, hps, Prod.ext rfl <| (Set.eq_of_mem_singleton hp1).symm⟩⟩ @[to_additive] theorem map_inr (s : Submonoid N) : s.map (inr M N) = prod ⊥ s := ext fun p => ⟨fun ⟨_, hx, hp⟩ => hp ▸ ⟨Set.mem_singleton 1, hx⟩, fun ⟨hp1, hps⟩ => ⟨p.2, hps, Prod.ext (Set.eq_of_mem_singleton hp1).symm rfl⟩⟩ @[to_additive (attr := simp) prod_bot_sup_bot_prod] theorem prod_bot_sup_bot_prod (s : Submonoid M) (t : Submonoid N) : (prod s ⊥) ⊔ (prod ⊥ t) = prod s t := (le_antisymm (sup_le (prod_mono (le_refl s) bot_le) (prod_mono bot_le (le_refl t)))) fun p hp => Prod.fst_mul_snd p ▸ mul_mem ((le_sup_left : prod s ⊥ ≤ prod s ⊥ ⊔ prod ⊥ t) ⟨hp.1, Set.mem_singleton 1⟩) ((le_sup_right : prod ⊥ t ≤ prod s ⊥ ⊔ prod ⊥ t) ⟨Set.mem_singleton 1, hp.2⟩) @[to_additive] theorem mem_map_equiv {f : M ≃* N} {K : Submonoid M} {x : N} : x ∈ K.map f.toMonoidHom ↔ f.symm x ∈ K := Set.mem_image_equiv @[to_additive] theorem map_equiv_eq_comap_symm (f : M ≃* N) (K : Submonoid M) : K.map f.toMonoidHom = K.comap f.symm.toMonoidHom := SetLike.coe_injective (f.toEquiv.image_eq_preimage K) @[to_additive] theorem comap_equiv_eq_map_symm (f : N ≃* M) (K : Submonoid M) : K.comap f = K.map f.symm := (map_equiv_eq_comap_symm f.symm K).symm @[to_additive (attr := simp)] theorem map_equiv_top (f : M ≃* N) : (⊤ : Submonoid M).map f = ⊤ := SetLike.coe_injective <| Set.image_univ.trans f.surjective.range_eq @[to_additive le_prod_iff] theorem le_prod_iff {s : Submonoid M} {t : Submonoid N} {u : Submonoid (M × N)} : u ≤ s.prod t ↔ u.map (fst M N) ≤ s ∧ u.map (snd M N) ≤ t := by constructor · intro h constructor · rintro x ⟨⟨y1, y2⟩, ⟨hy1, rfl⟩⟩ exact (h hy1).1 · rintro x ⟨⟨y1, y2⟩, ⟨hy1, rfl⟩⟩ exact (h hy1).2 · rintro ⟨hH, hK⟩ ⟨x1, x2⟩ h exact ⟨hH ⟨_, h, rfl⟩, hK ⟨_, h, rfl⟩⟩ @[to_additive prod_le_iff] theorem prod_le_iff {s : Submonoid M} {t : Submonoid N} {u : Submonoid (M × N)} : s.prod t ≤ u ↔ s.map (inl M N) ≤ u ∧ t.map (inr M N) ≤ u := by constructor · intro h constructor · rintro _ ⟨x, hx, rfl⟩ apply h exact ⟨hx, Submonoid.one_mem _⟩ · rintro _ ⟨x, hx, rfl⟩ apply h exact ⟨Submonoid.one_mem _, hx⟩ · rintro ⟨hH, hK⟩ ⟨x1, x2⟩ ⟨h1, h2⟩ have h1' : inl M N x1 ∈ u := by apply hH simpa using h1 have h2' : inr M N x2 ∈ u := by apply hK simpa using h2 simpa using Submonoid.mul_mem _ h1' h2' end Submonoid namespace MonoidHom variable {F : Type*} [FunLike F M N] [mc : MonoidHomClass F M N] open Submonoid library_note "range copy pattern"/-- For many categories (monoids, modules, rings, ...) the set-theoretic image of a morphism `f` is a subobject of the codomain. When this is the case, it is useful to define the range of a morphism in such a way that the underlying carrier set of the range subobject is definitionally `Set.range f`. In particular this means that the types `↥(Set.range f)` and `↥f.range` are interchangeable without proof obligations. A convenient candidate definition for range which is mathematically correct is `map ⊤ f`, just as `Set.range` could have been defined as `f '' Set.univ`. However, this lacks the desired definitional convenience, in that it both does not match `Set.range`, and that it introduces a redundant `x ∈ ⊤` term which clutters proofs. In such a case one may resort to the `copy` pattern. A `copy` function converts the definitional problem for the carrier set of a subobject into a one-off propositional proof obligation which one discharges while writing the definition of the definitionally convenient range (the parameter `hs` in the example below). A good example is the case of a morphism of monoids. A convenient definition for `MonoidHom.mrange` would be `(⊤ : Submonoid M).map f`. However since this lacks the required definitional convenience, we first define `Submonoid.copy` as follows: ```lean protected def copy (S : Submonoid M) (s : Set M) (hs : s = S) : Submonoid M := { carrier := s, one_mem' := hs.symm ▸ S.one_mem', mul_mem' := hs.symm ▸ S.mul_mem' } ``` and then finally define: ```lean def mrange (f : M →* N) : Submonoid N := ((⊤ : Submonoid M).map f).copy (Set.range f) Set.image_univ.symm ``` -/ /-- The range of a monoid homomorphism is a submonoid. See Note [range copy pattern]. -/ @[to_additive "The range of an `AddMonoidHom` is an `AddSubmonoid`."] def mrange (f : F) : Submonoid N := ((⊤ : Submonoid M).map f).copy (Set.range f) Set.image_univ.symm @[to_additive (attr := simp)] theorem coe_mrange (f : F) : (mrange f : Set N) = Set.range f := rfl @[to_additive (attr := simp)] theorem mem_mrange {f : F} {y : N} : y ∈ mrange f ↔ ∃ x, f x = y := Iff.rfl @[to_additive] theorem mrange_eq_map (f : F) : mrange f = (⊤ : Submonoid M).map f := Submonoid.copy_eq _ @[to_additive (attr := simp)] theorem mrange_id : mrange (MonoidHom.id M) = ⊤ := by simp [mrange_eq_map] @[to_additive] theorem map_mrange (g : N →* P) (f : M →* N) : f.mrange.map g = mrange (comp g f) := by simpa only [mrange_eq_map] using (⊤ : Submonoid M).map_map g f @[to_additive] theorem mrange_top_iff_surjective {f : F} : mrange f = (⊤ : Submonoid N) ↔ Function.Surjective f := SetLike.ext'_iff.trans <| Iff.trans (by rw [coe_mrange, coe_top]) Set.range_iff_surjective /-- The range of a surjective monoid hom is the whole of the codomain. -/ @[to_additive (attr := simp) "The range of a surjective `AddMonoid` hom is the whole of the codomain."] theorem mrange_top_of_surjective (f : F) (hf : Function.Surjective f) : mrange f = (⊤ : Submonoid N) := mrange_top_iff_surjective.2 hf @[to_additive] theorem mclosure_preimage_le (f : F) (s : Set N) : closure (f ⁻¹' s) ≤ (closure s).comap f := closure_le.2 fun _ hx => SetLike.mem_coe.2 <| mem_comap.2 <| subset_closure hx /-- The image under a monoid hom of the submonoid generated by a set equals the submonoid generated by the image of the set. -/ @[to_additive "The image under an `AddMonoid` hom of the `AddSubmonoid` generated by a set equals the `AddSubmonoid` generated by the image of the set."] theorem map_mclosure (f : F) (s : Set M) : (closure s).map f = closure (f '' s) := le_antisymm (map_le_iff_le_comap.2 <| le_trans (closure_mono <| Set.subset_preimage_image _ _) (mclosure_preimage_le _ _)) (closure_le.2 <| Set.image_subset _ subset_closure) @[to_additive (attr := simp)] theorem mclosure_range (f : F) : closure (Set.range f) = mrange f := by rw [← Set.image_univ, ← map_mclosure, mrange_eq_map, closure_univ] /-- Restriction of a monoid hom to a submonoid of the domain. -/ @[to_additive "Restriction of an `AddMonoid` hom to an `AddSubmonoid` of the domain."] def restrict {N S : Type*} [MulOneClass N] [SetLike S M] [SubmonoidClass S M] (f : M →* N) (s : S) : s →* N := f.comp (SubmonoidClass.subtype _) @[to_additive (attr := simp)] theorem restrict_apply {N S : Type*} [MulOneClass N] [SetLike S M] [SubmonoidClass S M] (f : M →* N) (s : S) (x : s) : f.restrict s x = f x := rfl @[to_additive (attr := simp)] theorem restrict_mrange (f : M →* N) : mrange (f.restrict S) = S.map f := by simp [SetLike.ext_iff] /-- Restriction of a monoid hom to a submonoid of the codomain. -/ @[to_additive (attr := simps apply) "Restriction of an `AddMonoid` hom to an `AddSubmonoid` of the codomain."] def codRestrict {S} [SetLike S N] [SubmonoidClass S N] (f : M →* N) (s : S) (h : ∀ x, f x ∈ s) : M →* s where toFun n := ⟨f n, h n⟩ map_one' := Subtype.eq f.map_one map_mul' x y := Subtype.eq (f.map_mul x y) /-- Restriction of a monoid hom to its range interpreted as a submonoid. -/ @[to_additive "Restriction of an `AddMonoid` hom to its range interpreted as a submonoid."] def mrangeRestrict {N} [MulOneClass N] (f : M →* N) : M →* (mrange f) := (f.codRestrict (mrange f)) fun x => ⟨x, rfl⟩ @[to_additive (attr := simp)] theorem coe_mrangeRestrict {N} [MulOneClass N] (f : M →* N) (x : M) : (f.mrangeRestrict x : N) = f x := rfl @[to_additive] theorem mrangeRestrict_surjective (f : M →* N) : Function.Surjective f.mrangeRestrict := fun ⟨_, ⟨x, rfl⟩⟩ => ⟨x, rfl⟩ /-- The multiplicative kernel of a monoid hom is the submonoid of elements `x : G` such that `f x = 1` -/ @[to_additive "The additive kernel of an `AddMonoid` hom is the `AddSubmonoid` of elements such that `f x = 0`"] def mker (f : F) : Submonoid M := (⊥ : Submonoid N).comap f @[to_additive] theorem mem_mker (f : F) {x : M} : x ∈ mker f ↔ f x = 1 := Iff.rfl @[to_additive] theorem coe_mker (f : F) : (mker f : Set M) = (f : M → N) ⁻¹' {1} := rfl @[to_additive] instance decidableMemMker [DecidableEq N] (f : F) : DecidablePred (· ∈ mker f) := fun x => decidable_of_iff (f x = 1) (mem_mker f) @[to_additive] theorem comap_mker (g : N →* P) (f : M →* N) : g.mker.comap f = mker (comp g f) := rfl @[to_additive (attr := simp)] theorem comap_bot' (f : F) : (⊥ : Submonoid N).comap f = mker f := rfl @[to_additive (attr := simp)] theorem restrict_mker (f : M →* N) : mker (f.restrict S) = f.mker.comap S.subtype := rfl @[to_additive] theorem mrangeRestrict_mker (f : M →* N) : mker (mrangeRestrict f) = mker f := by ext x change (⟨f x, _⟩ : mrange f) = ⟨1, _⟩ ↔ f x = 1 simp @[to_additive (attr := simp)] theorem mker_one : mker (1 : M →* N) = ⊤ := by ext simp [mem_mker] @[to_additive prod_map_comap_prod'] theorem prod_map_comap_prod' {M' : Type*} {N' : Type*} [MulOneClass M'] [MulOneClass N'] (f : M →* N) (g : M' →* N') (S : Submonoid N) (S' : Submonoid N') : (S.prod S').comap (prodMap f g) = (S.comap f).prod (S'.comap g) := SetLike.coe_injective <| Set.preimage_prod_map_prod f g _ _ -- Porting note: to_additive translated the name incorrectly in mathlib 3. @[to_additive mker_prod_map] theorem mker_prod_map {M' : Type*} {N' : Type*} [MulOneClass M'] [MulOneClass N'] (f : M →* N) (g : M' →* N') : mker (prodMap f g) = f.mker.prod (mker g) := by rw [← comap_bot', ← comap_bot', ← comap_bot', ← prod_map_comap_prod', bot_prod_bot] -- Porting note: to_additive translated the name incorrectly in mathlib 3. @[to_additive (attr := simp)] theorem mker_inl : mker (inl M N) = ⊥ := by ext x simp [mem_mker] @[to_additive (attr := simp)] theorem mker_inr : mker (inr M N) = ⊥ := by ext x simp [mem_mker] @[to_additive (attr := simp)] lemma mker_fst : mker (fst M N) = .prod ⊥ ⊤ := SetLike.ext fun _ => (and_true_iff _).symm @[to_additive (attr := simp)] lemma mker_snd : mker (snd M N) = .prod ⊤ ⊥ := SetLike.ext fun _ => (true_and_iff _).symm /-- The `MonoidHom` from the preimage of a submonoid to itself. -/ @[to_additive (attr := simps) "the `AddMonoidHom` from the preimage of an additive submonoid to itself."] def submonoidComap (f : M →* N) (N' : Submonoid N) : N'.comap f →* N' where toFun x := ⟨f x, x.2⟩ map_one' := Subtype.eq f.map_one map_mul' x y := Subtype.eq (f.map_mul x y) /-- The `MonoidHom` from a submonoid to its image. See `MulEquiv.SubmonoidMap` for a variant for `MulEquiv`s. -/ @[to_additive (attr := simps) "the `AddMonoidHom` from an additive submonoid to its image. See `AddEquiv.AddSubmonoidMap` for a variant for `AddEquiv`s."] def submonoidMap (f : M →* N) (M' : Submonoid M) : M' →* M'.map f where toFun x := ⟨f x, ⟨x, x.2, rfl⟩⟩ map_one' := Subtype.eq <| f.map_one map_mul' x y := Subtype.eq <| f.map_mul x y @[to_additive] theorem submonoidMap_surjective (f : M →* N) (M' : Submonoid M) : Function.Surjective (f.submonoidMap M') := by rintro ⟨_, x, hx, rfl⟩ exact ⟨⟨x, hx⟩, rfl⟩ end MonoidHom namespace Submonoid open MonoidHom @[to_additive] theorem mrange_inl : mrange (inl M N) = prod ⊤ ⊥ := by simpa only [mrange_eq_map] using map_inl ⊤ @[to_additive] theorem mrange_inr : mrange (inr M N) = prod ⊥ ⊤ := by simpa only [mrange_eq_map] using map_inr ⊤ @[to_additive] theorem mrange_inl' : mrange (inl M N) = comap (snd M N) ⊥ := mrange_inl.trans (top_prod _) @[to_additive] theorem mrange_inr' : mrange (inr M N) = comap (fst M N) ⊥ := mrange_inr.trans (prod_top _) @[to_additive (attr := simp)] theorem mrange_fst : mrange (fst M N) = ⊤ := mrange_top_of_surjective (fst M N) <| @Prod.fst_surjective _ _ ⟨1⟩ @[to_additive (attr := simp)] theorem mrange_snd : mrange (snd M N) = ⊤ := mrange_top_of_surjective (snd M N) <| @Prod.snd_surjective _ _ ⟨1⟩ @[to_additive prod_eq_bot_iff] theorem prod_eq_bot_iff {s : Submonoid M} {t : Submonoid N} : s.prod t = ⊥ ↔ s = ⊥ ∧ t = ⊥ := by simp only [eq_bot_iff, prod_le_iff, (gc_map_comap _).le_iff_le, comap_bot', mker_inl, mker_inr] -- Porting note: to_additive translated the name incorrectly in mathlib 3. @[to_additive prod_eq_top_iff] theorem prod_eq_top_iff {s : Submonoid M} {t : Submonoid N} : s.prod t = ⊤ ↔ s = ⊤ ∧ t = ⊤ := by simp only [eq_top_iff, le_prod_iff, ← (gc_map_comap _).le_iff_le, ← mrange_eq_map, mrange_fst, mrange_snd] -- Porting note: to_additive translated the name incorrectly in mathlib 3. @[to_additive (attr := simp)] theorem mrange_inl_sup_mrange_inr : mrange (inl M N) ⊔ mrange (inr M N) = ⊤ := by simp only [mrange_inl, mrange_inr, prod_bot_sup_bot_prod, top_prod_top] /-- The monoid hom associated to an inclusion of submonoids. -/ @[to_additive "The `AddMonoid` hom associated to an inclusion of submonoids."] def inclusion {S T : Submonoid M} (h : S ≤ T) : S →* T := S.subtype.codRestrict _ fun x => h x.2 @[to_additive (attr := simp)] theorem range_subtype (s : Submonoid M) : mrange s.subtype = s := SetLike.coe_injective <| (coe_mrange _).trans <| Subtype.range_coe @[to_additive] theorem eq_top_iff' : S = ⊤ ↔ ∀ x : M, x ∈ S := eq_top_iff.trans ⟨fun h m => h <| mem_top m, fun h m _ => h m⟩ @[to_additive] theorem eq_bot_iff_forall : S = ⊥ ↔ ∀ x ∈ S, x = (1 : M) := SetLike.ext_iff.trans <| by simp (config := { contextual := true }) [iff_def, S.one_mem] @[to_additive] theorem eq_bot_of_subsingleton [Subsingleton S] : S = ⊥ := by rw [eq_bot_iff_forall] intro y hy simpa using congr_arg ((↑) : S → M) <| Subsingleton.elim (⟨y, hy⟩ : S) 1 @[to_additive] theorem nontrivial_iff_exists_ne_one (S : Submonoid M) : Nontrivial S ↔ ∃ x ∈ S, x ≠ (1 : M) := calc Nontrivial S ↔ ∃ x : S, x ≠ 1 := nontrivial_iff_exists_ne 1 _ ↔ ∃ (x : _) (hx : x ∈ S), (⟨x, hx⟩ : S) ≠ ⟨1, S.one_mem⟩ := Subtype.exists _ ↔ ∃ x ∈ S, x ≠ (1 : M) := by simp [Ne] /-- A submonoid is either the trivial submonoid or nontrivial. -/ @[to_additive "An additive submonoid is either the trivial additive submonoid or nontrivial."] theorem bot_or_nontrivial (S : Submonoid M) : S = ⊥ ∨ Nontrivial S := by simp only [eq_bot_iff_forall, nontrivial_iff_exists_ne_one, ← not_forall, ← Classical.not_imp, Classical.em] /-- A submonoid is either the trivial submonoid or contains a nonzero element. -/ @[to_additive "An additive submonoid is either the trivial additive submonoid or contains a nonzero element."] theorem bot_or_exists_ne_one (S : Submonoid M) : S = ⊥ ∨ ∃ x ∈ S, x ≠ (1 : M) := S.bot_or_nontrivial.imp_right S.nontrivial_iff_exists_ne_one.mp end Submonoid namespace MulEquiv variable {S} {T : Submonoid M} /-- Makes the identity isomorphism from a proof that two submonoids of a multiplicative monoid are equal. -/ @[to_additive "Makes the identity additive isomorphism from a proof two submonoids of an additive monoid are equal."] def submonoidCongr (h : S = T) : S ≃* T := { Equiv.setCongr <| congr_arg _ h with map_mul' := fun _ _ => rfl } -- this name is primed so that the version to `f.range` instead of `f.mrange` can be unprimed. /-- A monoid homomorphism `f : M →* N` with a left-inverse `g : N → M` defines a multiplicative equivalence between `M` and `f.mrange`. This is a bidirectional version of `MonoidHom.mrange_restrict`. -/ @[to_additive (attr := simps (config := { simpRhs := true })) "An additive monoid homomorphism `f : M →+ N` with a left-inverse `g : N → M` defines an additive equivalence between `M` and `f.mrange`. This is a bidirectional version of `AddMonoidHom.mrange_restrict`. "] def ofLeftInverse' (f : M →* N) {g : N → M} (h : Function.LeftInverse g f) : M ≃* MonoidHom.mrange f := { f.mrangeRestrict with toFun := f.mrangeRestrict invFun := g ∘ f.mrange.subtype left_inv := h right_inv := fun x => Subtype.ext <| let ⟨x', hx'⟩ := MonoidHom.mem_mrange.mp x.2 show f (g x) = x by rw [← hx', h x'] } /-- A `MulEquiv` `φ` between two monoids `M` and `N` induces a `MulEquiv` between a submonoid `S ≤ M` and the submonoid `φ(S) ≤ N`. See `MonoidHom.submonoidMap` for a variant for `MonoidHom`s. -/ @[to_additive "An `AddEquiv` `φ` between two additive monoids `M` and `N` induces an `AddEquiv` between a submonoid `S ≤ M` and the submonoid `φ(S) ≤ N`. See `AddMonoidHom.addSubmonoidMap` for a variant for `AddMonoidHom`s."] def submonoidMap (e : M ≃* N) (S : Submonoid M) : S ≃* S.map e := { (e : M ≃ N).image S with map_mul' := fun _ _ => Subtype.ext (map_mul e _ _) } @[to_additive (attr := simp)] theorem coe_submonoidMap_apply (e : M ≃* N) (S : Submonoid M) (g : S) : ((submonoidMap e S g : S.map (e : M →* N)) : N) = e g := rfl @[to_additive (attr := simp) AddEquiv.add_submonoid_map_symm_apply] theorem submonoidMap_symm_apply (e : M ≃* N) (S : Submonoid M) (g : S.map (e : M →* N)) : (e.submonoidMap S).symm g = ⟨e.symm g, SetLike.mem_coe.1 <| Set.mem_image_equiv.1 g.2⟩ := rfl end MulEquiv @[to_additive (attr := simp)] theorem Submonoid.equivMapOfInjective_coe_mulEquiv (e : M ≃* N) : S.equivMapOfInjective (e : M →* N) (EquivLike.injective e) = e.submonoidMap S := by ext rfl section Actions /-! ### Actions by `Submonoid`s These instances transfer the action by an element `m : M` of a monoid `M` written as `m • a` onto the action by an element `s : S` of a submonoid `S : Submonoid M` such that `s • a = (s : M) • a`. These instances work particularly well in conjunction with `Monoid.toMulAction`, enabling `s • m` as an alias for `↑s * m`. -/ namespace Submonoid variable {M' : Type*} {α β : Type*} section MulOneClass variable [MulOneClass M'] @[to_additive] instance smul [SMul M' α] (S : Submonoid M') : SMul S α := SMul.comp _ S.subtype @[to_additive] instance smulCommClass_left [SMul M' β] [SMul α β] [SMulCommClass M' α β] (S : Submonoid M') : SMulCommClass S α β := ⟨fun a _ _ => (smul_comm (a : M') _ _ : _)⟩ @[to_additive] instance smulCommClass_right [SMul α β] [SMul M' β] [SMulCommClass α M' β] (S : Submonoid M') : SMulCommClass α S β := ⟨fun a s => (smul_comm a (s : M') : _)⟩ /-- Note that this provides `IsScalarTower S M' M'` which is needed by `SMulMulAssoc`. -/ instance isScalarTower [SMul α β] [SMul M' α] [SMul M' β] [IsScalarTower M' α β] (S : Submonoid M') : IsScalarTower S α β := ⟨fun a => (smul_assoc (a : M') : _)⟩ section SMul variable [SMul M' α] {S : Submonoid M'} @[to_additive] lemma smul_def (g : S) (a : α) : g • a = (g : M') • a := rfl @[to_additive (attr := simp)] lemma mk_smul (g : M') (hg : g ∈ S) (a : α) : (⟨g, hg⟩ : S) • a = g • a := rfl instance faithfulSMul [FaithfulSMul M' α] : FaithfulSMul S α := ⟨fun h => Subtype.ext <| eq_of_smul_eq_smul h⟩ end SMul end MulOneClass variable [Monoid M'] /-- The action by a submonoid is the action by the underlying monoid. -/ @[to_additive "The additive action by an `AddSubmonoid` is the action by the underlying `AddMonoid`. "] instance mulAction [MulAction M' α] (S : Submonoid M') : MulAction S α := MulAction.compHom _ S.subtype example {S : Submonoid M'} : IsScalarTower S M' M' := by infer_instance end Submonoid end Actions section Units namespace Submonoid /-- The multiplicative equivalence between the type of units of `M` and the submonoid of unit elements of `M`. -/ @[to_additive (attr := simps!) " The additive equivalence between the type of additive units of `M` and the additive submonoid whose elements are the additive units of `M`. "] noncomputable def unitsTypeEquivIsUnitSubmonoid [Monoid M] : Mˣ ≃* IsUnit.submonoid M where toFun x := ⟨x, Units.isUnit x⟩ invFun x := x.prop.unit left_inv x := IsUnit.unit_of_val_units _ right_inv x := by simp_rw [IsUnit.unit_spec] map_mul' x y := by simp_rw [Units.val_mul]; rfl end Submonoid end Units open AddSubmonoid Set namespace Nat @[simp] lemma addSubmonoid_closure_one : closure ({1} : Set ℕ) = ⊤ := by refine (eq_top_iff' _).2 <| Nat.rec (zero_mem _) ?_ simp_rw [Nat.succ_eq_add_one] exact fun n hn ↦ AddSubmonoid.add_mem _ hn <| subset_closure <| Set.mem_singleton _ end Nat namespace Submonoid variable {F : Type*} [FunLike F M N] [mc : MonoidHomClass F M N] @[to_additive] theorem map_comap_eq (f : F) (S : Submonoid N) : (S.comap f).map f = S ⊓ MonoidHom.mrange f := SetLike.coe_injective Set.image_preimage_eq_inter_range @[to_additive] theorem map_comap_eq_self {f : F} {S : Submonoid N} (h : S ≤ MonoidHom.mrange f) : (S.comap f).map f = S := by simpa only [inf_of_le_left h] using map_comap_eq f S end Submonoid