Skip to content

Commit

Permalink
Remove spurious injections
Browse files Browse the repository at this point in the history
  • Loading branch information
Georges Gonthier committed Dec 4, 2015
1 parent 03363b8 commit 19ac062
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 4 deletions.
4 changes: 1 addition & 3 deletions mathcomp/odd_order/BGsection15.v
Original file line number Diff line number Diff line change
Expand Up @@ -1248,7 +1248,7 @@ Lemma nonTI_Fitting_facts M :
[/\ M \in 'M_'F :|: 'M_'P1, M`_\F = M`_\sigma & M^`(1) \subset 'F(M)].
Proof.
move=> maxM nonTI; suff: [exists (y | y \notin M), 'F(M) :&: 'F(M) :^ y != 1].
by case/exists_inP=> y notMy /nonTI_Fitting_structure[] // [[-> ?] _ []].
by case/exists_inP=> y notMy /nonTI_Fitting_structure[] // [-> dMF] _ [].
rewrite -negb_forall_in; apply: contra nonTI => /forall_inP tiF.
apply/normedTI_P; rewrite normD1 setTI gFnorm setD_eq0 subG1.
split=> // [|g _]; first by rewrite (trivg_Fitting (mmax_sol maxM)) mmax_neq1.
Expand Down Expand Up @@ -1509,5 +1509,3 @@ by rewrite (subG1_contra _ ntCMsx) ?setIS //= -cent_cycle centS.
Qed.

End Section15.


2 changes: 1 addition & 1 deletion mathcomp/odd_order/BGsection16.v
Original file line number Diff line number Diff line change
Expand Up @@ -786,7 +786,7 @@ split; first by have [_ _ _ _ []] := Ptype_structure PmaxM hallK.
have [<- | neqMF_Ms] := eqVneq M`_\F M`_\sigma; first exact: Fcore_sub_Fitting.
have solMs: solvable M`_\sigma := solvableS (pcore_sub _ _) (mmax_sol maxM).
have [D hallD] := Hall_exists #|Kstar|^' solMs.
by case: (Fcore_structure maxM) notP1maxM => _ /(_ K D)[] // [[->]].
by case: (Fcore_structure maxM) notP1maxM => _ /(_ K D)[] // [->].
Qed.

End SingleGroupSummaries.
Expand Down

0 comments on commit 19ac062

Please sign in to comment.