aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/algebra/poly.v
diff options
context:
space:
mode:
authorCyril Cohen2018-07-14 01:26:16 +0100
committerCyril Cohen2018-07-14 01:26:16 +0100
commitededc3786a779f26303e9545dc68bd6006b4aae4 (patch)
treecebe4ef3365d341b2289aefd977bb717988ef27d /mathcomp/algebra/poly.v
parent618c9229fecbf6f1e85035aa0033943dcd4f3464 (diff)
Laurent's simplifications
Diffstat (limited to 'mathcomp/algebra/poly.v')
-rw-r--r--mathcomp/algebra/poly.v7
1 files changed, 2 insertions, 5 deletions
diff --git a/mathcomp/algebra/poly.v b/mathcomp/algebra/poly.v
index 1c5de11..5019eda 100644
--- a/mathcomp/algebra/poly.v
+++ b/mathcomp/algebra/poly.v
@@ -1950,10 +1950,7 @@ Qed.
Lemma coef_comp_poly p q n :
(p \Po q)`_n = \sum_(i < size p) p`_i * (q ^+ i)`_n.
-Proof.
-rewrite comp_polyE coef_sum.
-by elim/big_ind2: _ => [//|? ? ? ? -> -> //|i]; rewrite coefZ.
-Qed.
+Proof. by rewrite comp_polyE coef_sum; apply: eq_bigr => i; rewrite coefZ. Qed.
Lemma polyOver_comp S (ringS : semiringPred S) (kS : keyed_pred ringS) :
{in polyOver kS &, forall p q, p \Po q \in polyOver kS}.
@@ -2255,7 +2252,7 @@ rewrite big_split /= addnK -big_andE /=.
by elim/big_ind2: _ => // [[] [|n] [] [|m]|i Pi]; rewrite -?polySpred ?F_neq0.
Qed.
-Lemma size_prod_seq_eq1 (I : choiceType) (s : seq I) (F : I -> {poly R}) :
+Lemma size_prod_seq_eq1 (I : eqType) (s : seq I) (F : I -> {poly R}) :
reflect (forall i, i \in s -> size (F i) = 1%N)
(size (\prod_(i <- s) F i) == 1%N).
Proof.