diff options
Diffstat (limited to 'theories/Logic')
-rw-r--r-- | theories/Logic/EqdepFacts.v | 8 | ||||
-rw-r--r-- | theories/Logic/ExtensionalityFacts.v | 4 | ||||
-rw-r--r-- | theories/Logic/JMeq.v | 2 |
3 files changed, 7 insertions, 7 deletions
diff --git a/theories/Logic/EqdepFacts.v b/theories/Logic/EqdepFacts.v index a341a7a5a..d84cd8240 100644 --- a/theories/Logic/EqdepFacts.v +++ b/theories/Logic/EqdepFacts.v @@ -107,8 +107,8 @@ Section Dependent_Equality. End Dependent_Equality. -Implicit Arguments eq_dep [U P]. -Implicit Arguments eq_dep1 [U P]. +Arguments eq_dep [U P] p x q _. +Arguments eq_dep1 [U P] p x q y. (** Dependent equality is equivalent to equality on dependent pairs *) @@ -412,5 +412,5 @@ Notation inj_pairT2 := inj_pair2. End EqdepTheory. -Implicit Arguments eq_dep []. -Implicit Arguments eq_dep1 []. +Arguments eq_dep U P p x q _ : clear implicits. +Arguments eq_dep1 U P p x q y : clear implicits. diff --git a/theories/Logic/ExtensionalityFacts.v b/theories/Logic/ExtensionalityFacts.v index 421bbebcf..f5e71ef49 100644 --- a/theories/Logic/ExtensionalityFacts.v +++ b/theories/Logic/ExtensionalityFacts.v @@ -42,8 +42,8 @@ Record Delta A := { pi1:A; pi2:A; eq:pi1=pi2 }. Definition delta {A} (a:A) := {|pi1 := a; pi2 := a; eq := eq_refl a |}. -Implicit Arguments pi1 [[A]]. -Implicit Arguments pi2 [[A]]. +Arguments pi1 {A} _. +Arguments pi2 {A} _. Lemma diagonal_projs_same_behavior : forall A (x:Delta A), pi1 x = pi2 x. Proof. diff --git a/theories/Logic/JMeq.v b/theories/Logic/JMeq.v index 583d348a2..753009e68 100644 --- a/theories/Logic/JMeq.v +++ b/theories/Logic/JMeq.v @@ -24,7 +24,7 @@ Inductive JMeq (A:Type) (x:A) : forall B:Type, B -> Prop := Set Elimination Schemes. -Implicit Arguments JMeq_refl [[A] [x]] [A]. +Arguments JMeq_refl {A x} , [A] x. Hint Resolve JMeq_refl. |