aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/setoid_ring/Field_theory.v
diff options
context:
space:
mode:
authorGravatar Emilio Jesus Gallego Arias <e+git@x80.org>2017-10-15 19:11:48 +0200
committerGravatar Emilio Jesus Gallego Arias <e+git@x80.org>2017-10-15 19:11:48 +0200
commitcc03c37b48af466e6673fa4cb034e6ef19f709c0 (patch)
treeca2d65fd304bddfcd896db64a8856e32fff9207a /plugins/setoid_ring/Field_theory.v
parentf8975f9fce08c7d43e6e57be980cfa36635969a9 (diff)
[stdlib] Fix warnings on deprecated `Add Setoid`
The test suite cases are preserved until the feature is actually removed.
Diffstat (limited to 'plugins/setoid_ring/Field_theory.v')
-rw-r--r--plugins/setoid_ring/Field_theory.v6
1 files changed, 5 insertions, 1 deletions
diff --git a/plugins/setoid_ring/Field_theory.v b/plugins/setoid_ring/Field_theory.v
index 88e2cb1da..462ffde31 100644
--- a/plugins/setoid_ring/Field_theory.v
+++ b/plugins/setoid_ring/Field_theory.v
@@ -1612,7 +1612,11 @@ Section Complete.
Notation "x / y " := (rdiv x y). Notation "/ x" := (rinv x).
Notation "x == y" := (req x y) (at level 70, no associativity).
Variable Rsth : Setoid_Theory R req.
- Add Setoid R req Rsth as R_setoid3.
+ Add Parametric Relation : R req
+ reflexivity proved by Rsth.(@Equivalence_Reflexive _ _)
+ symmetry proved by Rsth.(@Equivalence_Symmetric _ _)
+ transitivity proved by Rsth.(@Equivalence_Transitive _ _)
+ as R_setoid3.
Variable Reqe : ring_eq_ext radd rmul ropp req.
Add Morphism radd with signature (req ==> req ==> req) as radd_ext3.
Proof. exact (Radd_ext Reqe). Qed.