aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/micromega/ZCoeff.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-08-01 14:39:51 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-08-05 19:52:20 +0200
commit99be46eb50213d1f35dfc4d30f35760ad5e75621 (patch)
tree9893c47cf1778fdeede3c2f6e1ec13539ca9ca14 /plugins/micromega/ZCoeff.v
parent69aff8116b4878671daf73cc7ccf713aac0c0e6d (diff)
More proofs independent of the names generated by induction/elim over
a dependent elimination principle for Prop arguments.
Diffstat (limited to 'plugins/micromega/ZCoeff.v')
-rw-r--r--plugins/micromega/ZCoeff.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/plugins/micromega/ZCoeff.v b/plugins/micromega/ZCoeff.v
index e30295e6a..d65c60167 100644
--- a/plugins/micromega/ZCoeff.v
+++ b/plugins/micromega/ZCoeff.v
@@ -41,19 +41,19 @@ Notation "x < y" := (rlt x y).
Lemma req_refl : forall x, req x x.
Proof.
- destruct sor.(SORsetoid).
+ destruct sor.(SORsetoid) as (Equivalence_Reflexive,_,_).
apply Equivalence_Reflexive.
Qed.
Lemma req_sym : forall x y, req x y -> req y x.
Proof.
- destruct sor.(SORsetoid).
+ destruct sor.(SORsetoid) as (_,Equivalence_Symmetric,_).
apply Equivalence_Symmetric.
Qed.
Lemma req_trans : forall x y z, req x y -> req y z -> req x z.
Proof.
- destruct sor.(SORsetoid).
+ destruct sor.(SORsetoid) as (_,_,Equivalence_Transitive).
apply Equivalence_Transitive.
Qed.