Skip to content

Commit

Permalink
remove duplicate in map_gal; remove temp
Browse files Browse the repository at this point in the history
  • Loading branch information
qvermande committed Jul 25, 2023
1 parent 49fd41e commit 7dff68d
Show file tree
Hide file tree
Showing 4 changed files with 5 additions and 51 deletions.
1 change: 0 additions & 1 deletion _CoqProject
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,6 @@ theories/xmathcomp/char0.v
theories/xmathcomp/cyclotomic_ext.v
theories/xmathcomp/real_closed_ext.v
theories/xmathcomp/artin_scheier.v
theories/xmathcomp/temp.v

-R theories Abel
-arg -w -arg -projection-no-head-constant
Expand Down
2 changes: 0 additions & 2 deletions theories/xmathcomp/map_gal.v
Original file line number Diff line number Diff line change
Expand Up @@ -19,8 +19,6 @@ Import AEnd_FinGroup.
Variables (F0 : fieldType) (L : splittingFieldType F0).
Implicit Types (K E F : {subfield L}).

Lemma galois_subW E F : galois E F -> (E <= F)%VS. Proof. by case/andP. Qed.

Lemma galois_normalW E F : galois E F -> (normalField E F)%VS.
Proof. by case/and3P. Qed.

Expand Down
38 changes: 0 additions & 38 deletions theories/xmathcomp/temp.v

This file was deleted.

15 changes: 5 additions & 10 deletions theories/xmathcomp/various.v
Original file line number Diff line number Diff line change
Expand Up @@ -175,18 +175,13 @@ apply/dvdn_partP => // p /[!(inE, mem_primes)]/and3P[p_prime _ pm].
by rewrite p_part pfactor_dvdn// vp_le.
Qed.

Lemma logn_prod [I : eqType] (r : seq I) (P : pred I) (F : I -> nat) (p : nat) :
{in r, forall n, P n -> (0 < F n)%N} ->
Lemma logn_prod [I : Type] (r : seq I) (P : pred I) (F : I -> nat) (p : nat) :
(forall n, P n -> (0 < F n)%N) ->
(logn p (\prod_(n <- r | P n) F n) = \sum_(n <- r | P n) logn p (F n))%N.
Proof.
elim: r => [|n r IHn Fnr0]; first by rewrite 2!big_nil logn1.
have Fr0: {in r, forall n : I, P n -> (0 < F n)%N}.
by move=> i ir; apply/Fnr0; rewrite in_cons ir orbT.
rewrite 2!big_cons; case /boolP: (P n) => Pn; last by apply/IHn.
move: (Fnr0 n); rewrite mem_head Pn => /= /(_ is_true_true is_true_true) Fn0.
rewrite lognM// ?IHn//.
rewrite big_seq_cond big_mkcond prodn_gt0// => i.
by case /boolP: ((i \in r) && P i) => // /andP[/Fr0].
move=> F_gt0; elim/(big_load (fun n => (n > 0)%N)): _.
elim/big_rec2: _; first by rewrite logn1.
by move=> i m n Pi [n_gt0 <-]; rewrite muln_gt0 lognM ?F_gt0.
Qed.

Lemma logn_partn (p n : nat) (pi : nat_pred) :
Expand Down

0 comments on commit 7dff68d

Please sign in to comment.