aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Classes/CMorphisms.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Classes/CMorphisms.v')
-rw-r--r--theories/Classes/CMorphisms.v9
1 files changed, 4 insertions, 5 deletions
diff --git a/theories/Classes/CMorphisms.v b/theories/Classes/CMorphisms.v
index d36833c71..a644654bc 100644
--- a/theories/Classes/CMorphisms.v
+++ b/theories/Classes/CMorphisms.v
@@ -73,7 +73,6 @@ Section Proper.
Definition respectful (R : crelation A) (R' : crelation B) : crelation (A -> B) :=
Eval compute in @respectful_hetero A A (fun _ => B) (fun _ => B) R (fun _ _ => R').
-
End Proper.
(** We favor the use of Leibniz equality or a declared reflexive crelation
@@ -396,14 +395,14 @@ Section GenericInstances.
Reflexive (@Logic.eq A ==> R').
Proof. simpl_crelation. Qed.
- (** [respectful] is a morphism for crelation equivalence. *)
-
+ (** [respectful] is a morphism for crelation equivalence . *)
+ Set Printing All. Set Printing Universes.
Global Instance respectful_morphism :
Proper (relation_equivalence ++> relation_equivalence ++> relation_equivalence)
(@respectful A B).
Proof.
- intros R R' HRR' S S' HSS' f g.
- unfold respectful, relation_equivalence in * ; simpl in *.
+ intros R R' HRR' S S' HSS' f g.
+ unfold respectful , relation_equivalence in *; simpl in *.
split ; intros H x y Hxy.
apply (fst (HSS' _ _)). apply H. now apply (snd (HRR' _ _)).
apply (snd (HSS' _ _)). apply H. now apply (fst (HRR' _ _)).