aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/solvable
diff options
context:
space:
mode:
authorCyril Cohen2018-02-06 14:04:50 +0100
committerCyril Cohen2018-02-06 14:14:36 +0100
commitf3ce9ace4b55654d6240db9eb41a6de3c488f0d9 (patch)
treed44ad1d84bb57b368f6e65fe871ec0c6e5a558eb /mathcomp/solvable
parentfafd4dac5315e1d4e071b0044a50a16360b31964 (diff)
fixing things that @ggonthier and @ybertot spotted and some I spotted
Diffstat (limited to 'mathcomp/solvable')
-rw-r--r--mathcomp/solvable/burnside_app.v6
-rw-r--r--mathcomp/solvable/gfunctor.v2
-rw-r--r--mathcomp/solvable/jordanholder.v2
3 files changed, 5 insertions, 5 deletions
diff --git a/mathcomp/solvable/burnside_app.v b/mathcomp/solvable/burnside_app.v
index d602d0a..d9010d5 100644
--- a/mathcomp/solvable/burnside_app.v
+++ b/mathcomp/solvable/burnside_app.v
@@ -75,7 +75,7 @@ Ltac inj_tac :=
move: (erefl rot_inv); unfold rot_inv;
match goal with |- ?X = _ -> injective ?Y =>
move=> _; let x := get_inv Y X in
- apply: (can_inj (g:=x)); move => [val H1]
+ apply: (can_inj (g:=x)); move=> [val H1]
end.
Lemma R1_inj : injective R1.
@@ -1137,10 +1137,10 @@ Qed.
Lemma uniq4_uniq6 : forall x y z t : cube,
uniq [:: x; y; z; t] -> exists u, exists v, uniq [:: x; y; z; t; u; v].
Proof.
-move=> x y z t Uxt; move: ( cardC (mem [:: x; y; z; t])).
+move=> x y z t Uxt; move: (cardC (mem [:: x; y; z; t])).
rewrite card_ord (card_uniq_tuple Uxt) => hcard.
have hcard2: #|predC (mem [:: x; y; z; t])| = 2.
- by apply: ( @addnI 4); rewrite /injective hcard.
+ by apply: (@addnI 4); rewrite /injective hcard.
have: #|predC (mem [:: x; y; z; t])| != 0 by rewrite hcard2.
case/existsP=> u Hu; exists u.
move: (cardC (mem [:: x; y; z; t; u])); rewrite card_ord => hcard5.
diff --git a/mathcomp/solvable/gfunctor.v b/mathcomp/solvable/gfunctor.v
index 7fbee8c..fc8385d 100644
--- a/mathcomp/solvable/gfunctor.v
+++ b/mathcomp/solvable/gfunctor.v
@@ -158,7 +158,7 @@ End Definitions.
Section ClassDefinitions.
Structure iso_map := IsoMap {
- apply: object_map;
+ apply : object_map;
_ : group_valued apply;
_ : closed apply;
_ : iso_continuous apply
diff --git a/mathcomp/solvable/jordanholder.v b/mathcomp/solvable/jordanholder.v
index 66f6156..7f60bed 100644
--- a/mathcomp/solvable/jordanholder.v
+++ b/mathcomp/solvable/jordanholder.v
@@ -531,7 +531,7 @@ have: K' :=: 1%G \/ K' :=: (G / H).
case; last first.
move/quotient_injG; rewrite !inE /=; move/(_ nKH nHG)=> c; move: nsGK.
by rewrite c subxx.
-rewrite /= -trivg_quotient => - tK'; apply: (congr1 (@gval _)); move: tK'.
+rewrite /= -trivg_quotient => tK'; apply: (congr1 (@gval _)); move: tK'.
by apply: (@quotient_injG _ H); rewrite ?inE /= ?normal_refl.
Qed.