From ed06a90f16fcf7d45672bbddf42efe4cc0efd4d4 Mon Sep 17 00:00:00 2001 From: gareuselesinge Date: Mon, 21 Nov 2011 17:03:52 +0000 Subject: theories/, plugins/ and test-suite/ ported to the Arguments vernacular git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14718 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Program/Basics.v | 6 +++--- 1 file changed, 3 insertions(+), 3 deletions(-) (limited to 'theories/Program/Basics.v') diff --git a/theories/Program/Basics.v b/theories/Program/Basics.v index 5293a66cbe..7cef5c5ad8 100644 --- a/theories/Program/Basics.v +++ b/theories/Program/Basics.v @@ -17,7 +17,7 @@ (** The polymorphic identity function is defined in [Datatypes]. *) -Implicit Arguments id [[A]]. +Arguments id {A} x. (** Function composition. *) @@ -53,5 +53,5 @@ Definition apply {A B} (f : A -> B) (x : A) := f x. (** Curryfication of [prod] is defined in [Logic.Datatypes]. *) -Implicit Arguments prod_curry [[A] [B] [C]]. -Implicit Arguments prod_uncurry [[A] [B] [C]]. +Arguments prod_curry {A B C} f p. +Arguments prod_uncurry {A B C} f x y. -- cgit v1.2.3