aboutsummaryrefslogtreecommitdiff
path: root/src/Util/Tuple.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jagro@google.com>2016-09-08 11:22:45 -0700
committerGravatar Jason Gross <jagro@google.com>2016-09-08 11:22:45 -0700
commit3eab786d92b348c1dec33640eec3a02a5a86606b (patch)
tree91adbd9562c3a952b1714245cc4e64dcccda2f16 /src/Util/Tuple.v
parent054752ccf0b80bc413e70202a823fd034db6ea6b (diff)
Fully qualify [Require]s
This way they won't become ambiguous if we add new files
Diffstat (limited to 'src/Util/Tuple.v')
-rw-r--r--src/Util/Tuple.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/src/Util/Tuple.v b/src/Util/Tuple.v
index 568c3ce21..76064e7b4 100644
--- a/src/Util/Tuple.v
+++ b/src/Util/Tuple.v
@@ -1,5 +1,5 @@
Require Import Coq.Classes.Morphisms.
-Require Import Relation_Definitions.
+Require Import Coq.Relations.Relation_Definitions.
Require Import Crypto.Util.Decidable.
Require Export Crypto.Util.FixCoqMistakes.
@@ -162,7 +162,7 @@ Arguments fieldwiseb {A B n} _ _ _.
Lemma fieldwiseb'_fieldwise' :forall {A B} n R Rb
(a:tuple' A n) (b:tuple' B n),
- (forall a b, Rb a b = true <-> R a b) ->
+ (forall a b, Rb a b = true <-> R a b) ->
(fieldwiseb' Rb a b = true <-> fieldwise' R a b).
Proof.
intros.
@@ -176,7 +176,7 @@ Qed.
Lemma fieldwiseb_fieldwise :forall {A B} n R Rb
(a:tuple A n) (b:tuple B n),
- (forall a b, Rb a b = true <-> R a b) ->
+ (forall a b, Rb a b = true <-> R a b) ->
(fieldwiseb Rb a b = true <-> fieldwise R a b).
Proof.
intros; destruct n; simpl @tuple in *;