@@ -59,8 +59,7 @@ def coeff (A : HVertexOperator Γ R V W) (n : Γ) : V →ₗ[R] W where
59
59
toFun v := ((of R).symm (A v)).coeff n
60
60
map_add' _ _ := by simp
61
61
map_smul' _ _ := by
62
- simp only [map_smul, RingHom.id_apply]
63
- exact rfl
62
+ simp only [map_smul, RingHom.id_apply, of_symm_smul, HahnSeries.smul_coeff]
64
63
65
64
@[deprecated (since := "2024-06-18")] alias _root_.VertexAlg.coeff := coeff
66
65
@@ -85,12 +84,8 @@ condition, we produce a heterogeneous vertex operator. -/
85
84
def of_coeff (f : Γ → V →ₗ[R] W)
86
85
(hf : ∀(x : V), (Function.support (f · x)).IsPWO) : HVertexOperator Γ R V W where
87
86
toFun x := (of R) { coeff := fun g => f g x, isPWO_support' := hf x }
88
- map_add' _ _ := by
89
- ext
90
- simp
91
- map_smul' _ _ := by
92
- simp only [map_smul, RingHom.id_apply]
93
- exact rfl
87
+ map_add' _ _ := by ext; simp
88
+ map_smul' _ _ := by ext; simp
94
89
95
90
@[deprecated (since := "2024-06-18")] alias _root_.VertexAlg.HetVertexOperator.of_coeff := of_coeff
96
91
@@ -122,14 +117,14 @@ theorem compHahnSeries_add (u v : U) :
122
117
compHahnSeries A B (u + v) = compHahnSeries A B u + compHahnSeries A B v := by
123
118
ext
124
119
simp only [compHahnSeries_coeff, map_add, coeff_apply, HahnSeries.add_coeff', Pi.add_apply]
125
- rw [← @ HahnSeries.add_coeff]
120
+ rw [← HahnSeries.add_coeff]
126
121
127
122
@[simp]
128
123
theorem compHahnSeries_smul (r : R) (u : U) :
129
124
compHahnSeries A B (r • u) = r • compHahnSeries A B u := by
130
125
ext
131
126
simp only [compHahnSeries_coeff, LinearMapClass.map_smul, coeff_apply, HahnSeries.smul_coeff]
132
- exact rfl
127
+ rw [← HahnSeries.smul_coeff]
133
128
134
129
/-- The composite of two heterogeneous vertex operators, as a heterogeneous vertex operator. -/
135
130
@[simps]
@@ -143,9 +138,8 @@ def comp : HVertexOperator (Γ' ×ₗ Γ) R U W where
143
138
map_smul' := by
144
139
intro r x
145
140
ext g
146
- simp only [HahnSeries.ofIterate, compHahnSeries_smul, Equiv.symm_apply_apply, RingHom.id_apply,
147
- HahnSeries.smul_coeff, compHahnSeries_coeff, coeff_apply]
148
- exact rfl
141
+ simp only [HahnSeries.ofIterate, compHahnSeries_smul, HahnSeries.smul_coeff,
142
+ compHahnSeries_coeff, coeff_apply, Equiv.symm_apply_apply, RingHom.id_apply, of_symm_smul]
149
143
150
144
@[simp]
151
145
theorem comp_coeff (g : Γ' ×ₗ Γ) :
0 commit comments