aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success
diff options
context:
space:
mode:
authorGravatar corbinea <corbinea@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-21 13:54:00 +0000
committerGravatar corbinea <corbinea@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-02-21 13:54:00 +0000
commit2e67ff1b33d05b9efc020de664f3200f9ff0d479 (patch)
tree15ee065d3e0ab19d0e46eea62be18333aeff8083 /test-suite/success
parente1a5d40aeb341c382aec7bcce977c3979c6b8ef2 (diff)
congruence now knows about _ -> _
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10579 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success')
-rw-r--r--test-suite/success/cc.v9
1 files changed, 9 insertions, 0 deletions
diff --git a/test-suite/success/cc.v b/test-suite/success/cc.v
index fecc89772..94d827fd5 100644
--- a/test-suite/success/cc.v
+++ b/test-suite/success/cc.v
@@ -78,6 +78,14 @@ intros.
congruence.
Qed.
+(* example with implications *)
+
+Theorem arrow : forall (A B: Prop) (C D:Set) , A=B -> C=D ->
+(A -> C) = (B -> D).
+congruence.
+Qed.
+
+
Set Implicit Arguments.
Parameter elt: Set.
@@ -94,5 +102,6 @@ Proof.
auto.
Qed.
+
\ No newline at end of file