This repository was archived by the owner on Jul 24, 2024. It is now read-only.
File tree Expand file tree Collapse file tree 3 files changed +5
-5
lines changed
group_theory/subsemigroup Expand file tree Collapse file tree 3 files changed +5
-5
lines changed Original file line number Diff line number Diff line change @@ -309,10 +309,10 @@ fun_like.ext _ _ e.apply_symm_apply
309
309
theorem self_trans_symm (e : M ≃* N) : e.trans e.symm = refl M :=
310
310
fun_like.ext _ _ e.symm_apply_apply
311
311
312
- @[to_additive, simp ] lemma coe_monoid_hom_refl {M} [mul_one_class M] :
312
+ @[simp, to_additive ] lemma coe_monoid_hom_refl {M} [mul_one_class M] :
313
313
(refl M : M →* M) = monoid_hom.id M := rfl
314
314
315
- @[to_additive, simp ] lemma coe_monoid_hom_trans {M N P}
315
+ @[simp, to_additive ] lemma coe_monoid_hom_trans {M N P}
316
316
[mul_one_class M] [mul_one_class N] [mul_one_class P] (e₁ : M ≃* N) (e₂ : N ≃* P) :
317
317
(e₁.trans e₂ : M →* P) = (e₂ : N →* P).comp ↑e₁ :=
318
318
rfl
Original file line number Diff line number Diff line change 151
151
section
152
152
variables (M) [comm_semigroup M]
153
153
154
- @[to_additive, simp ] lemma center_eq_top : center M = ⊤ :=
154
+ @[simp, to_additive ] lemma center_eq_top : center M = ⊤ :=
155
155
set_like.coe_injective (set.center_eq_univ M)
156
156
157
157
end
Original file line number Diff line number Diff line change @@ -698,14 +698,14 @@ variables [has_mul X] [has_continuous_mul X]
698
698
@[to_additive " The continuous map `λ y, y + x" ]
699
699
protected def mul_right (x : X) : C(X, X) := mk _ (continuous_mul_right x)
700
700
701
- @[to_additive, simp ]
701
+ @[simp, to_additive ]
702
702
lemma coe_mul_right (x : X) : ⇑(continuous_map.mul_right x) = λ y, y * x := rfl
703
703
704
704
/-- The continuous map `λ y, x * y` -/
705
705
@[to_additive " The continuous map `λ y, x + y" ]
706
706
protected def mul_left (x : X) : C(X, X) := mk _ (continuous_mul_left x)
707
707
708
- @[to_additive, simp ]
708
+ @[simp, to_additive ]
709
709
lemma coe_mul_left (x : X) : ⇑(continuous_map.mul_left x) = λ y, x * y := rfl
710
710
711
711
end continuous_map
You can’t perform that action at this time.
0 commit comments