@@ -3,7 +3,6 @@ Copyright (c) 2018 Kenny Lau. All rights reserved.
3
3
Released under Apache 2.0 license as described in the file LICENSE.
4
4
Authors: Kenny Lau, Yury Kudryashov
5
5
-/
6
- import Mathlib.Algebra.BigOperators.Group.Finset
7
6
import Mathlib.Algebra.Module.LinearMap.Defs
8
7
9
8
/-!
@@ -82,6 +81,7 @@ the second approach only when you need to weaken a condition on either `R` or `A
82
81
-/
83
82
84
83
assert_not_exists Field
84
+ assert_not_exists Finset
85
85
assert_not_exists Module.End
86
86
87
87
universe u v w u₁ v₁
@@ -165,26 +165,6 @@ theorem coe_sub (a b : R) :
165
165
166
166
end CommRingRing
167
167
168
- section CommSemiringCommSemiring
169
-
170
- variable {R A : Type *} [CommSemiring R] [CommSemiring A] [Algebra R A]
171
-
172
- -- direct to_additive fails because of some mix-up with polynomials
173
- @[norm_cast]
174
- theorem coe_prod {ι : Type *} {s : Finset ι} (a : ι → R) :
175
- (↑(∏ i ∈ s, a i : R) : A) = ∏ i ∈ s, (↑(a i) : A) :=
176
- map_prod (algebraMap R A) a s
177
-
178
- -- to_additive fails for some reason
179
- @[norm_cast]
180
- theorem coe_sum {ι : Type *} {s : Finset ι} (a : ι → R) :
181
- ↑(∑ i ∈ s, a i) = ∑ i ∈ s, (↑(a i) : A) :=
182
- map_sum (algebraMap R A) a s
183
-
184
- -- Porting note: removed attribute [ to_additive ] coe_prod; why should this be a `to_additive`?
185
-
186
- end CommSemiringCommSemiring
187
-
188
168
end algebraMap
189
169
190
170
/-- Creating an algebra from a morphism to the center of a semiring. -/
0 commit comments