aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/algebra/poly.v
diff options
context:
space:
mode:
authorCyril Cohen2018-11-24 17:58:35 +0100
committerGitHub2018-11-24 17:58:35 +0100
commitadd6e85884691faef1bf8742e803374815672cc2 (patch)
tree2ffb41f5afa11a147989c8efcc1dcb295ae2ed2b /mathcomp/algebra/poly.v
parent967088a6f87405a93ce21971392c58996df8c99f (diff)
parentf049e51c39077a025907ea87c08178dad1841801 (diff)
Merge pull request #249 from anton-trunov/prenex-implicits
Merge Arguments and Prenex Implicits
Diffstat (limited to 'mathcomp/algebra/poly.v')
-rw-r--r--mathcomp/algebra/poly.v12
1 files changed, 6 insertions, 6 deletions
diff --git a/mathcomp/algebra/poly.v b/mathcomp/algebra/poly.v
index 040b3a8..34174bf 100644
--- a/mathcomp/algebra/poly.v
+++ b/mathcomp/algebra/poly.v
@@ -1688,11 +1688,11 @@ Notation "a ^` ()" := (deriv a) : ring_scope.
Notation "a ^` ( n )" := (derivn n a) : ring_scope.
Notation "a ^`N ( n )" := (nderivn n a) : ring_scope.
-Arguments monicP [R p].
-Arguments rootP [R p x].
-Arguments rootPf [R p x].
-Arguments rootPt [R p x].
-Arguments unity_rootP [R n z].
+Arguments monicP {R p}.
+Arguments rootP {R p x}.
+Arguments rootPf {R p x}.
+Arguments rootPt {R p x}.
+Arguments unity_rootP {R n z}.
Arguments polyOverP {R S0 addS kS p}.
Canonical polynomial_countZmodType (R : countRingType) :=
@@ -2611,7 +2611,7 @@ Open Scope unity_root_scope.
Definition unity_rootE := unity_rootE.
Definition unity_rootP := @unity_rootP.
-Arguments unity_rootP [R n z].
+Arguments unity_rootP {R n z}.
Definition prim_order_exists := prim_order_exists.
Notation prim_order_gt0 := prim_order_gt0.