aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Classes/Morphisms_Prop.v
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-05-11 22:04:26 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-05-11 22:04:26 +0000
commit30443ddaba7a0cc996216b3d692b97e0b05907fe (patch)
tree1a1bdadcdf69582262bd6bddc21e9e03215d2871 /theories/Classes/Morphisms_Prop.v
parentb6c6e36afa8da16a62bf16191baa2531894c54fc (diff)
- Cleanup parsing of binders, reducing to a single production for all
binders. - Change syntax of type class instances to better match the usual syntax of lemmas/definitions with name first, then arguments ":" instance. Update theories/Classes accordingly. - Correct globalization of tactic references when doing Ltac :=/::=, update documentation. - Remove the not so useful "(x &)" and "{{x}}" syntaxes from Program.Utils, and subset_scope as well. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10919 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Classes/Morphisms_Prop.v')
-rw-r--r--theories/Classes/Morphisms_Prop.v12
1 files changed, 6 insertions, 6 deletions
diff --git a/theories/Classes/Morphisms_Prop.v b/theories/Classes/Morphisms_Prop.v
index 301fba534..7dc1f95ef 100644
--- a/theories/Classes/Morphisms_Prop.v
+++ b/theories/Classes/Morphisms_Prop.v
@@ -73,7 +73,7 @@ Program Instance iff_iff_iff_impl_morphism : Morphism (iff ==> iff ==> iff) impl
(** Morphisms for quantifiers *)
-Program Instance {A : Type} => ex_iff_morphism : Morphism (pointwise_relation iff ==> iff) (@ex A).
+Program Instance ex_iff_morphism {A : Type} : Morphism (pointwise_relation iff ==> iff) (@ex A).
Next Obligation.
Proof.
@@ -86,7 +86,7 @@ Program Instance {A : Type} => ex_iff_morphism : Morphism (pointwise_relation if
exists x₁. rewrite H. assumption.
Qed.
-Program Instance {A : Type} => ex_impl_morphism :
+Program Instance ex_impl_morphism {A : Type} :
Morphism (pointwise_relation impl ==> impl) (@ex A).
Next Obligation.
@@ -95,7 +95,7 @@ Program Instance {A : Type} => ex_impl_morphism :
exists H0. apply H. assumption.
Qed.
-Program Instance {A : Type} => ex_inverse_impl_morphism :
+Program Instance ex_inverse_impl_morphism {A : Type} :
Morphism (pointwise_relation (inverse impl) ==> inverse impl) (@ex A).
Next Obligation.
@@ -104,7 +104,7 @@ Program Instance {A : Type} => ex_inverse_impl_morphism :
exists H0. apply H. assumption.
Qed.
-Program Instance {A : Type} => all_iff_morphism :
+Program Instance all_iff_morphism {A : Type} :
Morphism (pointwise_relation iff ==> iff) (@all A).
Next Obligation.
@@ -113,7 +113,7 @@ Program Instance {A : Type} => all_iff_morphism :
intuition ; specialize (H x0) ; intuition.
Qed.
-Program Instance {A : Type} => all_impl_morphism :
+Program Instance all_impl_morphism {A : Type} :
Morphism (pointwise_relation impl ==> impl) (@all A).
Next Obligation.
@@ -122,7 +122,7 @@ Program Instance {A : Type} => all_impl_morphism :
intuition ; specialize (H x0) ; intuition.
Qed.
-Program Instance {A : Type} => all_inverse_impl_morphism :
+Program Instance all_inverse_impl_morphism {A : Type} :
Morphism (pointwise_relation (inverse impl) ==> inverse impl) (@all A).
Next Obligation.