leanprover-community / mathlib4

The math library of Lean 4

Home Page:https://leanprover-community.github.io/mathlib4_docs

Geek Repo:Geek Repo

Github PK Tool:Github PK Tool

Porting note: `rfl` required

pitmonticone opened this issue · comments

Classifies porting notes claiming:

rfl required

Examples

@[to_additive]
instance mulAction [Monoid M] [MulAction M β] : MulAction M (Germ l β) where
-- Porting note: `rfl` required.
one_smul f :=
inductionOn f fun f => by
norm_cast
simp only [one_smul]
rfl
mul_smul c₁ c₂ f :=
inductionOn f fun f => by
norm_cast
simp only [mul_smul]
rfl
@[to_additive]
instance mulAction' [Monoid M] [MulAction M β] : MulAction (Germ l M) (Germ l β) where
-- Porting note: `rfl` required.
one_smul f := inductionOn f fun f => by simp only [← coe_one, ← coe_smul', one_smul]
mul_smul c₁ c₂ f :=
inductionOn₃ c₁ c₂ f fun c₁ c₂ f => by
norm_cast
simp only [mul_smul]
rfl
#align filter.germ.mul_action' Filter.Germ.mulAction'
#align filter.germ.add_action' Filter.Germ.addAction'
instance distribMulAction [Monoid M] [AddMonoid N] [DistribMulAction M N] :
DistribMulAction M (Germ l N) where
-- Porting note: `rfl` required.
smul_add c f g :=
inductionOn₂ f g fun f g => by
norm_cast
simp only [smul_add]
rfl
smul_zero c := by simp only [← coe_zero, ← coe_smul, smul_zero]
instance distribMulAction' [Monoid M] [AddMonoid N] [DistribMulAction M N] :
DistribMulAction (Germ l M) (Germ l N) where
-- Porting note: `rfl` required.
smul_add c f g :=
inductionOn₃ c f g fun c f g => by
norm_cast
simp only [smul_add]
rfl
smul_zero c := inductionOn c fun c => by simp only [← coe_zero, ← coe_smul', smul_zero]
#align filter.germ.distrib_mul_action' Filter.Germ.distribMulAction'
instance module [Semiring R] [AddCommMonoid M] [Module R M] : Module R (Germ l M) where
-- Porting note: `rfl` required.
add_smul c₁ c₂ f :=
inductionOn f fun f => by
norm_cast
simp only [add_smul]
rfl
zero_smul f :=
inductionOn f fun f => by
norm_cast
simp only [zero_smul, coe_zero]
rfl
instance module' [Semiring R] [AddCommMonoid M] [Module R M] : Module (Germ l R) (Germ l M) where
-- Porting note: `rfl` required.
add_smul c₁ c₂ f :=
inductionOn₃ c₁ c₂ f fun c₁ c₂ f => by
norm_cast
simp only [add_smul]
rfl
zero_smul f := inductionOn f fun f => by simp only [← coe_zero, ← coe_smul', zero_smul]
#align filter.germ.module' Filter.Germ.module'