aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/fingroup/perm.v
diff options
context:
space:
mode:
authorReynald Affeldt2020-04-08 00:47:30 +0900
committerReynald Affeldt2020-04-09 20:58:12 +0900
commit691e0c20a8934343a6840f2a19735acea6e79d05 (patch)
tree0ab5012172dc0e4135a47afc15200a5fa1c85853 /mathcomp/fingroup/perm.v
parent504a34ba48a29a252c40cfc0467f6b192243b6bc (diff)
- switching long suffixes to short suffixes
+ `odd_add` -> `oddD` + `odd_sub` -> `oddB` + `take_addn` -> `takeD` + `rot_addn` -> `rotD` + `nseq_addn` -> `nseqD` fixes #359
Diffstat (limited to 'mathcomp/fingroup/perm.v')
-rw-r--r--mathcomp/fingroup/perm.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/mathcomp/fingroup/perm.v b/mathcomp/fingroup/perm.v
index eb5e028..aff97b0 100644
--- a/mathcomp/fingroup/perm.v
+++ b/mathcomp/fingroup/perm.v
@@ -452,8 +452,8 @@ Qed.
Lemma odd_mul_tperm x y s : odd_perm (tperm x y * s) = (x != y) (+) odd_perm s.
Proof.
-rewrite addbC -addbA -[~~ _]oddb -odd_add -ncycles_mul_tperm.
-by rewrite odd_add odd_double addbF.
+rewrite addbC -addbA -[~~ _]oddb -oddD -ncycles_mul_tperm.
+by rewrite oddD odd_double addbF.
Qed.
Lemma odd_tperm x y : odd_perm (tperm x y) = (x != y).
@@ -490,7 +490,7 @@ Lemma odd_permM : {morph odd_perm : s1 s2 / s1 * s2 >-> s1 (+) s2}.
Proof.
move=> s1 s2; case: (prod_tpermP s1) => ts1 ->{s1} dts1.
case: (prod_tpermP s2) => ts2 ->{s2} dts2.
-by rewrite -big_cat !odd_perm_prod ?all_cat ?dts1 // size_cat odd_add.
+by rewrite -big_cat !odd_perm_prod ?all_cat ?dts1 // size_cat oddD.
Qed.
Lemma odd_permV s : odd_perm s^-1 = odd_perm s.