aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Sets/Partial_Order.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-07-05 16:56:37 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2012-07-05 16:56:37 +0000
commitffb64d16132dd80f72ecb619ef87e3eee1fa8bda (patch)
tree5368562b42af1aeef7e19b4bd897c9fc5655769b /theories/Sets/Partial_Order.v
parenta46ccd71539257bb55dcddd9ae8510856a5c9a16 (diff)
Kills the useless tactic annotations "in |- *"
Most of these heavyweight annotations were introduced a long time ago by the automatic 7.x -> 8.0 translator git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@15518 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Sets/Partial_Order.v')
-rw-r--r--theories/Sets/Partial_Order.v18
1 files changed, 9 insertions, 9 deletions
diff --git a/theories/Sets/Partial_Order.v b/theories/Sets/Partial_Order.v
index a319b9832..bb1cf7083 100644
--- a/theories/Sets/Partial_Order.v
+++ b/theories/Sets/Partial_Order.v
@@ -63,13 +63,13 @@ Section Partial_order_facts.
forall x y z:U,
Strict_Rel_of U D x y -> Rel_of U D y z -> Strict_Rel_of U D x z.
Proof.
- unfold Strict_Rel_of at 1 in |- *.
- red in |- *.
- elim D; simpl in |- *.
+ unfold Strict_Rel_of at 1.
+ red.
+ elim D; simpl.
intros C R H' H'0; elim H'0.
intros H'1 H'2 H'3 x y z H'4 H'5; split.
apply H'2 with (y := y); tauto.
- red in |- *; intro H'6.
+ red; intro H'6.
elim H'4; intros H'7 H'8; apply H'8; clear H'4.
apply H'3; auto.
rewrite H'6; tauto.
@@ -79,20 +79,20 @@ Section Partial_order_facts.
forall x y z:U,
Rel_of U D x y -> Strict_Rel_of U D y z -> Strict_Rel_of U D x z.
Proof.
- unfold Strict_Rel_of at 1 in |- *.
- red in |- *.
- elim D; simpl in |- *.
+ unfold Strict_Rel_of at 1.
+ red.
+ elim D; simpl.
intros C R H' H'0; elim H'0.
intros H'1 H'2 H'3 x y z H'4 H'5; split.
apply H'2 with (y := y); tauto.
- red in |- *; intro H'6.
+ red; intro H'6.
elim H'5; intros H'7 H'8; apply H'8; clear H'5.
apply H'3; auto.
rewrite <- H'6; auto.
Qed.
Lemma Strict_Rel_Transitive : Transitive U (Strict_Rel_of U D).
- red in |- *.
+ red.
intros x y z H' H'0.
apply Strict_Rel_Transitive_with_Rel with (y := y);
[ intuition | unfold Strict_Rel_of in H', H'0; intuition ].