Built with
doc-gen4 , running Lean4.
Bubbles (
) indicate interactive fragments: hover for details, tap to reveal contents.
Use
Ctrl+β Ctrl+β to navigate,
Ctrl+π±οΈ to focus.
On Mac, use
Cmd instead of
Ctrl .
/-
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
Ported by: FrΓ©dΓ©ric Dupuis
! This file was ported from Lean 3 source module algebra.hom.commute
! leanprover-community/mathlib commit 6eb334bd8f3433d5b08ba156b8ec3e6af47e1904
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
import Mathlib.Algebra.Hom.Group
import Mathlib.Algebra.Group.Commute
/-!
# Multiplicative homomorphisms respect semiconjugation and commutation.
-/
section Commute
variable { F M N : Type _ } [ Mul M ] [ Mul N ] { a x y : M }
@[ to_additive ( attr := simp )]
protected theorem SemiconjBy.map [ MulHomClass F M N ] ( h : SemiconjBy : {M : Type ?u.63} β [inst : Mul M ] β M β M β M β Prop SemiconjBy a x y ) ( f : F ) :
SemiconjBy : {M : Type ?u.85} β [inst : Mul M ] β M β M β M β Prop SemiconjBy ( f a ) ( f x ) ( f y ) := by simpa only [ SemiconjBy : {M : Type ?u.385} β [inst : Mul M ] β M β M β M β Prop SemiconjBy, map_mul : β {M : Type ?u.388} {N : Type ?u.389} {F : Type ?u.387} [inst : Mul M ] [inst_1 : Mul N ] [inst_2 : MulHomClass F M N ]
(f : F ) (x y : M ), βf (x * y ) = βf x * βf y map_mul] using congr_arg : β {Ξ± : Sort ?u.523} {Ξ² : Sort ?u.522} {aβ aβ : Ξ± } (f : Ξ± β Ξ² ), aβ = aβ β f aβ = f aβ congr_arg f h
#align semiconj_by.map SemiconjBy.map
#align add_semiconj_by.map AddSemiconjBy.map
@[ to_additive ( attr := simp )]
protected theorem Commute.map [ MulHomClass F M N ] ( h : Commute : {S : Type ?u.993} β [inst : Mul S ] β S β S β Prop Commute x y ) ( f : F ) : Commute : {S : Type ?u.1015} β [inst : Mul S ] β S β S β Prop Commute ( f x ) ( f y ) :=
SemiconjBy.map h f
#align commute.map Commute.map
#align add_commute.map AddCommute.map
end Commute