aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Sets/Relations_1_facts.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-10-06 16:06:34 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-10-06 16:06:34 +0000
commit44eb01365e01c41e632b3f601195d82ca07419ac (patch)
treefba8cc37627fc6f75a239abf71ee55defbae57ce /theories/Sets/Relations_1_facts.v
parent209738abe5f77ea8f04f7cff6bccb133c4cccb33 (diff)
Parenthèses pour les tactiques
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@671 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Sets/Relations_1_facts.v')
-rwxr-xr-xtheories/Sets/Relations_1_facts.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Sets/Relations_1_facts.v b/theories/Sets/Relations_1_facts.v
index 1b27a4a9d..c86e57318 100755
--- a/theories/Sets/Relations_1_facts.v
+++ b/theories/Sets/Relations_1_facts.v
@@ -28,7 +28,7 @@ Theorem Rsym_imp_notRsym: (U: Type) (R: (Relation U)) (Symmetric U R) ->
(Symmetric U (Complement U R)).
Proof.
Unfold Symmetric Complement.
-(Intros U R H' x y H'0; Red; Intro H'1; Apply H'0); Auto with sets.
+Intros U R H' x y H'0; Red; Intro H'1; Apply H'0; Auto with sets.
Qed.
Theorem Equiv_from_preorder :