Skip to content

Commit

Permalink
Document how to simplify proofs when requiring MC >= 1.16.0
Browse files Browse the repository at this point in the history
  • Loading branch information
Julien Puydt committed Sep 14, 2022
1 parent c84a549 commit f7181aa
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 0 deletions.
3 changes: 3 additions & 0 deletions theories/abel.v
Original file line number Diff line number Diff line change
Expand Up @@ -417,6 +417,7 @@ rewrite [LHS](@all_roots_prod_XsubC _ _ ws).
- by rewrite (monicP _) ?monic_XnsubC// scale1r big_map big_enum.
- by rewrite size_XnsubC// size_map size_enum_ord.
- rewrite all_map; apply/allP => i _ /=; rewrite /root !hornerE ?hornerXn.
(* FIXME: remove ?hornerXn when requiring MC >= 1.16.0 *)
by rewrite exprMn exprAC [w ^+ _]prim_expr_order// expr1n mulr1 subrr.
- by rewrite uniq_rootsE uniq_roots_Xn_sub_xn.
Qed.
Expand All @@ -434,6 +435,7 @@ Lemma dvdp_minpoly_Xn_subn E :
Proof using.
move=> xpE; have [->|p_gt0] := posnP p; first by rewrite !expr0 subrr dvdp0.
by rewrite minPoly_dvdp /root ?poly_XnsubC_over// !hornerE ?hornerXn subrr.
(* FIXME: remove ?hornerXn when requiring MC >= 1.16.0 *)
Qed.

Lemma galois_cyclo_radical E : (p > 0)%N -> x ^+ p \in E ->
Expand Down Expand Up @@ -1506,6 +1508,7 @@ have Cchar := Cchar => p_neq0; split.
pose v := i.+1.-root (iota (u ^+ i.+1)).
have : ('X ^+ i.+1 - (v ^+ i.+1)%:P).[iota u] == 0.
by rewrite !hornerE ?hornerXn rootCK// rmorphX subrr.
(* FIXME: remove ?hornerXn when requiring MC >= 1.16.0 *)
have /Xn_sub_xnE->// := prim1rootP (isT : 0 < i.+1)%N.
rewrite horner_prod prodf_seq_eq0/= => /hasP[/= l _].
rewrite hornerXsubC subr_eq0 => /eqP u_eq.
Expand Down
1 change: 1 addition & 0 deletions theories/xmathcomp/various.v
Original file line number Diff line number Diff line change
Expand Up @@ -433,6 +433,7 @@ apply/eqP; rewrite eqn_leq mup_leq ?mup_geq//.
have [->|Nxy] := eqVneq x y.
by rewrite /= dvdpp ?dvdp_Pexp2l ?size_XsubC ?ltnn.
by rewrite dvd1p dvdp_XsubCl /root !hornerE ?horner_exp ?hornerE expf_neq0// subr_eq0.
(* FIXME: remove ?horner_exp ?hornerE when requiring MC >= 1.16.0 *)
Qed.

Lemma mupNroot (x : L) q : ~~ root q x -> mup x q = 0%N.
Expand Down

0 comments on commit f7181aa

Please sign in to comment.