aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/ssreflect/choice.v
diff options
context:
space:
mode:
authorJasper Hugunin2018-02-21 22:41:00 -0800
committerJasper Hugunin2018-02-21 22:41:00 -0800
commit19f9b3e774db1dedca149675f022d65cdeab7e6c (patch)
treec7ef14c60588c4595fc7d0b1740383d4429f5fcb /mathcomp/ssreflect/choice.v
parent13f26ccc09f87b222f9601892f085276a6ddb8c0 (diff)
Change Implicit Arguments to Arguments in ssreflect
Diffstat (limited to 'mathcomp/ssreflect/choice.v')
-rw-r--r--mathcomp/ssreflect/choice.v4
1 files changed, 2 insertions, 2 deletions
diff --git a/mathcomp/ssreflect/choice.v b/mathcomp/ssreflect/choice.v
index a696bbd..b5c2391 100644
--- a/mathcomp/ssreflect/choice.v
+++ b/mathcomp/ssreflect/choice.v
@@ -193,7 +193,7 @@ Qed.
End Def.
End GenTree.
-Implicit Arguments GenTree.codeK [].
+Arguments GenTree.codeK : clear implicits.
Definition tree_eqMixin (T : eqType) := PcanEqMixin (GenTree.codeK T).
Canonical tree_eqType (T : eqType) := EqType (GenTree.tree T) (tree_eqMixin T).
@@ -558,7 +558,7 @@ Export Countable.Exports.
Definition unpickle T := Countable.unpickle (Countable.class T).
Definition pickle T := Countable.pickle (Countable.class T).
-Implicit Arguments unpickle [T].
+Arguments unpickle [T].
Prenex Implicits pickle unpickle.
Section CountableTheory.