aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Sets/Relations_1_facts.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Sets/Relations_1_facts.v')
-rwxr-xr-xtheories/Sets/Relations_1_facts.v7
1 files changed, 5 insertions, 2 deletions
diff --git a/theories/Sets/Relations_1_facts.v b/theories/Sets/Relations_1_facts.v
index c86e57318..ad6b55c0c 100755
--- a/theories/Sets/Relations_1_facts.v
+++ b/theories/Sets/Relations_1_facts.v
@@ -79,13 +79,16 @@ Theorem cong_symmetric_same_relation:
(U:Type) (R, R':(Relation U)) (same_relation U R R') -> (Symmetric U R) ->
(Symmetric U R').
Proof.
-Intuition.
+ Compute;Intros;Elim H;Intros;Clear H;Apply (H3 y x (H0 x y (H2 x y H1))).
+(*Intuition.*)
Qed.
Theorem cong_antisymmetric_same_relation:
(U:Type) (R, R':(Relation U)) (same_relation U R R') ->
(Antisymmetric U R) -> (Antisymmetric U R').
-Intuition.
+Proof.
+ Compute;Intros;Elim H;Intros;Clear H;Apply (H0 x y (H3 x y H1) (H3 y x H2)).
+(*Intuition.*)
Qed.
Theorem cong_transitive_same_relation: