aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/character/mxabelem.v
diff options
context:
space:
mode:
authorJasper Hugunin2018-03-04 16:57:06 -0800
committerJasper Hugunin2018-03-04 16:57:06 -0800
commit2525c33691e25f837b7dca31d4c702199b3dbc5d (patch)
tree7937f252a0818909c715ccc20f3611a4f5c482d5 /mathcomp/character/mxabelem.v
parent6f075b64b936de9ee4fa79ea4dc1d2fb9b9cf2c8 (diff)
Change deprecated Arguments Scope to Arguments
Diffstat (limited to 'mathcomp/character/mxabelem.v')
-rw-r--r--mathcomp/character/mxabelem.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/mathcomp/character/mxabelem.v b/mathcomp/character/mxabelem.v
index 92fdb0e..b121f4c 100644
--- a/mathcomp/character/mxabelem.v
+++ b/mathcomp/character/mxabelem.v
@@ -341,7 +341,7 @@ Proof. by move=> sHG; rewrite gacentE // setTI afix_repr. Qed.
End FinFieldRepr.
-Arguments Scope rowg_mx [_ _ group_scope].
+Arguments rowg_mx _ _ _%g.
Notation "''Zm'" := (scale_action _ _ _) (at level 8) : action_scope.
Notation "''Zm'" := (scale_groupAction _ _ _) : groupAction_scope.
@@ -406,7 +406,7 @@ Open Scope abelem_scope.
Definition abelem_dim' (gT : finGroupType) (E : {set gT}) :=
(logn (pdiv #|E|) #|E|).-1.
-Arguments Scope abelem_dim' [_ group_scope].
+Arguments abelem_dim' _ _%g.
Notation "''dim' E" := (abelem_dim' E).+1
(at level 10, E at level 8, format "''dim' E") : abelem_scope.