aboutsummaryrefslogtreecommitdiff
path: root/src/Algebra/Field_test.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Algebra/Field_test.v')
-rw-r--r--src/Algebra/Field_test.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/Algebra/Field_test.v b/src/Algebra/Field_test.v
index 0743729c2..59ca72c6b 100644
--- a/src/Algebra/Field_test.v
+++ b/src/Algebra/Field_test.v
@@ -4,7 +4,7 @@ Require Import Crypto.Algebra.Ring Crypto.Algebra.Field.
Module _fsatz_test.
Section _test.
Context {F eq zero one opp add sub mul inv div}
- {fld:@Algebra.field F eq zero one opp add sub mul inv div}
+ {fld:@Hierarchy.field F eq zero one opp add sub mul inv div}
{eq_dec:DecidableRel eq}.
Local Infix "=" := eq. Local Notation "a <> b" := (not (a = b)).
Local Infix "=" := eq : type_scope. Local Notation "a <> b" := (not (a = b)) : type_scope.