Skip to content

Commit d419332

Browse files
committed
Fix warnings
1 parent 08f826d commit d419332

File tree

6 files changed

+25
-15
lines changed

6 files changed

+25
-15
lines changed

_CoqProject

Lines changed: 5 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1 +1,6 @@
1+
-arg -w -arg -ambiguous-paths
2+
-arg -w -arg -notation-overridden
3+
-arg -w -arg -redundant-canonical-projection
4+
-arg -w -arg -projection-no-head-constant
5+
16
-R _build/default/src SsrMultinomials

src/dune

Lines changed: 1 addition & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -4,6 +4,4 @@
44
(flags -w -ambiguous-paths
55
-w -notation-overridden
66
-w -redundant-canonical-projection
7-
-w -projection-no-head-constant
8-
-w -duplicate-clear
9-
-w -undeclared-scope))
7+
-w -projection-no-head-constant))

src/freeg.v

Lines changed: 5 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -44,9 +44,11 @@ Local Notation simpm := Monoid.simpm.
4444
Reserved Notation "{ 'freeg' K / G }" (at level 0, K, G at level 2, format "{ 'freeg' K / G }").
4545
Reserved Notation "{ 'freeg' K }" (at level 0, K at level 2, format "{ 'freeg' K }").
4646
Reserved Notation "[ 'freeg' S ]" (at level 0, S at level 2, format "[ 'freeg' S ]").
47+
Reserved Notation "<< z *p k >>" (at level 0, format "<< z *p k >>").
48+
Reserved Notation "<< k >>" (at level 0, format "<< k >>").
4749

4850
(* -------------------------------------------------------------------- *)
49-
Let perm_eq_map (T U : eqType) (f : T -> U) (xs ys : seq T):
51+
Lemma perm_eq_map (T U : eqType) (f : T -> U) (xs ys : seq T):
5052
perm_eq xs ys -> (perm_eq (map f xs) (map f ys)).
5153
Proof. by move/permP=> h; apply/permP=> p; rewrite !count_map. Qed.
5254

@@ -207,7 +209,7 @@ Section FreegTheory.
207209
Definition dom D := [seq zx.2 | zx <- (repr D)].
208210

209211
Lemma uniq_dom D: uniq (dom D).
210-
Proof. by rewrite /dom; case: (repr D)=> /= {D} D; case/andP. Qed.
212+
Proof. by rewrite /dom; case: (repr D)=> /= {}D; case/andP. Qed.
211213

212214
Lemma reduced_cons zx s:
213215
reduced (zx :: s) = [&& zx.1 != 0, zx.2 \notin predom s & reduced s].
@@ -516,7 +518,7 @@ Section FreegTheory.
516518
Proof.
517519
apply/esym/eqP/freeg_eqP=> k.
518520
rewrite -{1 2}[D]freeg_repr !coeff_Freeg /dom.
519-
case: (repr D)=> {D} D rD /=; rewrite -map_comp map_id_in //.
521+
case: (repr D)=> {}D rD /=; rewrite -map_comp map_id_in //.
520522
move=> [z x]; rewrite reduced_mem // => /andP [/eqP <- _].
521523
by rewrite /= coeff_Freeg.
522524
Qed.

src/monalg.v

Lines changed: 4 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -25,6 +25,7 @@ Local Open Scope fset.
2525
Local Open Scope fmap.
2626
Local Open Scope ring_scope.
2727

28+
Declare Scope malg_scope.
2829
Delimit Scope malg_scope with MP.
2930

3031
Local Notation simpm := Monoid.simpm.
@@ -33,6 +34,7 @@ Local Notation ilift := fintype.lift.
3334
Local Notation efst := (@fst _ _) (only parsing).
3435
Local Notation esnd := (@snd _ _) (only parsing).
3536

37+
Declare Scope m_scope.
3638
Delimit Scope m_scope with M.
3739

3840
(* -------------------------------------------------------------------- *)
@@ -53,9 +55,9 @@ Reserved Notation "[ 'malg' x => E ]"
5355
Reserved Notation "{ 'mpoly' T [ n ] }"
5456
(at level 0, T, n at level 2, format "{ 'mpoly' T [ n ] }").
5557
Reserved Notation "<< z *p k >>"
56-
(at level 0).
58+
(at level 0, format "<< z *p k >>").
5759
Reserved Notation "<< k >>"
58-
(at level 0).
60+
(at level 0, format "<< k >>").
5961
Reserved Notation "g @_ k"
6062
(at level 3, k at level 2, left associativity, format "g @_ k").
6163
Reserved Notation "c %:MP"

src/mpoly.v

Lines changed: 9 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -93,6 +93,9 @@ Import Monoid GRing.Theory BigEnough Order.Theory.
9393

9494
Local Open Scope ring_scope.
9595

96+
Declare Scope mpoly_scope.
97+
Declare Scope multi_scope.
98+
9699
Delimit Scope mpoly_scope with MP.
97100
Delimit Scope multi_scope with MM.
98101

@@ -159,10 +162,10 @@ Hypothesis ih: forall t1, (forall t2, t2 < t1 -> P t2) -> P t1.
159162

160163
Lemma ltxwf t : P t.
161164
Proof.
162-
elim: n P ih t => [|k wih] Pn kih t; last case: (tupleP t) => a {t}t.
165+
elim: n P ih t => [|k wih] Pn kih t; last case: (tupleP t) => a {}t.
163166
by rewrite tuple0; apply/kih=> t2; rewrite tuple0.
164167
elim/wf: a t => a iha t; elim/wih: t => t iht.
165-
apply/kih => t'; case: (tupleP t') => a' {t'}t'; rewrite [_ < _]ltxi_cons.
168+
apply/kih => t'; case: (tupleP t') => a' {}t'; rewrite [_ < _]ltxi_cons.
166169
by case: (comparableP a a') => //= [/iha/(_ t')|<- /iht].
167170
Qed.
168171

@@ -761,7 +764,7 @@ elim/(@ltxwf _ [porderType of nat]): t m=> //=; last first.
761764
move=> t wih m Em; apply/ih=> m' lt_m'm.
762765
apply/(wih (tof m'))=> //; rewrite -Em.
763766
by rewrite /tof ltEsub/= -ltEmnm.
764-
move=> Q {ih} ih x; elim: x {-2}x (leqnn x).
767+
move=> Q {}ih x; elim: x {-2}x (leqnn x).
765768
move=> x; rewrite leqn0=> /eqP->; apply/ih.
766769
by move=> y; rewrite ltEnat/= ltn0.
767770
move=> k wih l le_l_Sk; apply/ih=> y; rewrite ltEnat => lt_yl.
@@ -2420,7 +2423,7 @@ have: sorted <=%O%O s by apply/sort_sorted/le_total.
24202423
case: s => /= [_|m' s srt_s]; first rewrite perm_sym.
24212424
by move/perm_small_eq=> -> //.
24222425
move/perm_mem => <-; rewrite in_cons => /orP[/eqP->//|].
2423-
elim: s m' srt_s => //= m'' s ih m' /andP[le_mm' /ih {ih}ih].
2426+
elim: s m' srt_s => //= m'' s ih m' /andP[le_mm' /ih {}ih].
24242427
by rewrite in_cons => /orP[/eqP->//|] /ih /(le_trans le_mm').
24252428
Qed.
24262429

@@ -4112,7 +4115,7 @@ apply/(irr_sorted_eq (leT := ltn))=> //.
41124115
by apply/ltn_trans.
41134116
by move=> ?; rewrite /ltn /= ltnn.
41144117
move=> m; apply/mapP/mapP; case=> /= x;
4115-
by rewrite (h, =^~ h)=> {h} h ->; exists x.
4118+
by rewrite (h, =^~ h)=> {}h ->; exists x.
41164119
Qed.
41174120

41184121
Lemma mesym_tupleE (k : nat) : 's_k =
@@ -4975,7 +4978,7 @@ Lemma homog_prod (s : seq {mpoly R[n]}) :
49754978
Proof.
49764979
move=> homs; apply/homogP; elim: s homs => [_ | p s ihs] /=.
49774980
by exists 0%N; rewrite big_nil; apply/dhomog1.
4978-
case/andP=> /homogP [dp p_hdp] {ihs}/ihs [d ih].
4981+
case/andP=> /homogP [dp p_hdp] {}/ihs [d ih].
49794982
by exists (dp + d)%N; rewrite big_cons; apply/dhomogM.
49804983
Qed.
49814984

src/ssrcomplements.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -139,7 +139,7 @@ Section BigMkSub.
139139
try rewrite filter_uniq // (map_inj_uniq val_inj).
140140
by rewrite /index_enum -enumT enum_uniq.
141141
move=> x; rewrite !mem_filter {}/Q; apply/andb_idr.
142-
rewrite andbC; case/andP=> /h {h}h /h sT_x.
142+
rewrite andbC; case/andP=> /h {}h /h sT_x.
143143
apply/mapP; exists (Sub x sT_x).
144144
by rewrite /index_enum -enumT mem_enum.
145145
by rewrite SubK.

0 commit comments

Comments
 (0)