aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/cc.v
diff options
context:
space:
mode:
authorGravatar corbinea <corbinea@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-26 14:33:04 +0000
committerGravatar corbinea <corbinea@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-26 14:33:04 +0000
commitcdb1422b199d1966fb2276c197a3d2ed516a735f (patch)
treefbded1c9006c68b2bba57202b16d722ccc5c5adc /test-suite/success/cc.v
parent4cc4a78c44a2d156fe55acec58195d89e08df9ac (diff)
removal of CC.v lemata in cc (deprecated)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4994 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/cc.v')
-rw-r--r--test-suite/success/cc.v22
1 files changed, 16 insertions, 6 deletions
diff --git a/test-suite/success/cc.v b/test-suite/success/cc.v
index 18a99056b..4c0287dc3 100644
--- a/test-suite/success/cc.v
+++ b/test-suite/success/cc.v
@@ -1,4 +1,3 @@
-Require CC.
Theorem t1: (A:Set)(a:A)(f:A->A)
(f a)=a->(f (f a))=a.
@@ -40,14 +39,16 @@ Theorem dep2:(A,B:Set)(f:(A:Set)(b:bool)if b then unit else A->unit)(e:A==B)
Intros;Rewrite e;Reflexivity.
Save.
-(* example with CCSolve *)
-Theorem t4 : (A:Set; P:(A->Prop); u,v:A)u=v->(P u)->(P v).
-Intros.
-CCsolve.
+(* example that CC can solve
+ (dependent function applied to the same argument)*)
+
+Theorem dep3:(A:Set)(P:(A->Set))(f,g:(x:A)(P x))f=g->(x:A)(f x)=(g x).
+Intros.
+CC.
Save.
-(* Exambles with injection rule *)
+(* Examples with injection rule *)
Theorem t5 : (A:Set;a,b,c,d:A)(a,c)=(b,d)->a=b/\c=d.
Intros.
@@ -59,3 +60,12 @@ Intros.
CC.
Save.
+(* example with CCSolve (requires CC)*)
+
+Require CC.
+
+Theorem t4 : (A:Set; P:(A->Prop); a,b,c,d:A)a=b->c=d->
+ (P a)->((P b)->(P c))->(P d).
+Intros.
+CCsolve.
+Save.