aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Classes/Equivalence.v
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-09-14 12:45:57 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-09-14 12:45:57 +0000
commit3c8057d3c28b9243328ecb1f0a8197b11cf9fd77 (patch)
treedc673d3999f77765fd81bc2a0b6c65694a496d7a /theories/Classes/Equivalence.v
parent32b759737d89205340714979505eae22c5e3c4c3 (diff)
Use manual implicts in Classes and rationalize class parameter names.
Now it's [A] and [R] for carriers and relations and [eqA] when the relation is supposed to be an equivalence. The types are always implicit except for [pointwise_relation] which now takes the domain type as an explicit argument. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11408 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Classes/Equivalence.v')
-rw-r--r--theories/Classes/Equivalence.v7
1 files changed, 3 insertions, 4 deletions
diff --git a/theories/Classes/Equivalence.v b/theories/Classes/Equivalence.v
index 197786c8b..9909f18ad 100644
--- a/theories/Classes/Equivalence.v
+++ b/theories/Classes/Equivalence.v
@@ -111,8 +111,7 @@ Section Respecting.
{ morph : A -> B | respectful R R' morph morph }.
Program Instance respecting_equiv [ eqa : Equivalence A R, eqb : Equivalence B R' ] :
- Equivalence respecting
- (fun (f g : respecting) => forall (x y : A), R x y -> R' (proj1_sig f x) (proj1_sig g y)).
+ Equivalence (fun (f g : respecting) => forall (x y : A), R x y -> R' (proj1_sig f x) (proj1_sig g y)).
Solve Obligations using unfold respecting in * ; simpl_relation ; program_simpl.
@@ -125,8 +124,8 @@ End Respecting.
(** The default equivalence on function spaces, with higher-priority than [eq]. *)
-Program Instance pointwise_equivalence [ eqb : Equivalence B eqB ] :
- Equivalence (A -> B) (pointwise_relation eqB) | 9.
+Program Instance pointwise_equivalence A ((eqb : Equivalence B eqB)) :
+ Equivalence (pointwise_relation A eqB) | 9.
Next Obligation.
Proof.