diff options
author | msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2008-11-05 22:03:08 +0000 |
---|---|---|
committer | msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2008-11-05 22:03:08 +0000 |
commit | 792c7e078754f440ab16b0420a4ea045d7daccef (patch) | |
tree | 563a5b7e55d7d33498a0a8cd4ecfb1955bcb4b77 /theories | |
parent | 215bbe5cddc7fae276fe50131dcff70bc1b7f6d9 (diff) |
Minor fixes:
- Rework definition of the type of respecful functions in Morphisms.v
- Unfold [flip] in "Add Morphism" tactic (suggested by N. Tabareau)
- Add a "coqvariableref" command in coqdoc.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11545 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rw-r--r-- | theories/Classes/Equivalence.v | 6 | ||||
-rw-r--r-- | theories/Classes/SetoidTactics.v | 2 |
2 files changed, 4 insertions, 4 deletions
diff --git a/theories/Classes/Equivalence.v b/theories/Classes/Equivalence.v index ef85c14aa..469147cf4 100644 --- a/theories/Classes/Equivalence.v +++ b/theories/Classes/Equivalence.v @@ -103,12 +103,12 @@ Section Respecting. (** Here we build an equivalence instance for functions which relates respectful ones only, we do not export it. *) - Definition respecting [ Equivalence A (R : relation A), Equivalence B (R' : relation B) ] : Type := + Definition respecting {( eqa : Equivalence A (R : relation A), eqb : Equivalence B (R' : relation B) )} : Type := { morph : A -> B | respectful R R' morph morph }. Program Instance respecting_equiv [ eqa : Equivalence A R, eqb : Equivalence B R' ] : - Equivalence (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 eqa eqb) => 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. Next Obligation. diff --git a/theories/Classes/SetoidTactics.v b/theories/Classes/SetoidTactics.v index f8b7f62e9..024b400ae 100644 --- a/theories/Classes/SetoidTactics.v +++ b/theories/Classes/SetoidTactics.v @@ -178,7 +178,7 @@ Ltac reverse_arrows x := end. Ltac default_add_morphism_tactic := - intros ; + unfold flip ; intros ; (try destruct_morphism) ; match goal with | [ |- (?x ==> ?y) _ _ ] => red_subst_eq_morphism (x ==> y) ; reverse_arrows (x ==> y) |