aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Wf.v
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-07-08 13:43:16 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-07-08 13:43:16 +0000
commit4844bf0fa24d049b28a7aa1788c5d85e8b98753d (patch)
treee8d9003ad3e0e6cf6d95b9b2e7550d5fe0ae0110 /theories/Init/Wf.v
parent0f07e18c269c2c5db3c557cfa83e6d88a1cb7bd4 (diff)
recursion bien fondee sur des pairs
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4224 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init/Wf.v')
-rwxr-xr-xtheories/Init/Wf.v25
1 files changed, 25 insertions, 0 deletions
diff --git a/theories/Init/Wf.v b/theories/Init/Wf.v
index dff48c953..93111571f 100755
--- a/theories/Init/Wf.v
+++ b/theories/Init/Wf.v
@@ -19,6 +19,7 @@ V7only [Unset Implicit Arguments.].
Require Logic.
Require LogicSyntax.
+Require Datatypes.
(** Well-founded induction principle on Prop *)
@@ -131,3 +132,27 @@ Qed.
End FixPoint.
End Well_founded.
+
+(** A recursor over pairs *)
+
+Chapter Well_founded_2.
+
+ Variable A,B : Set.
+ Variable R : A * B -> A * B -> Prop.
+
+ Variable P : A -> B -> Type.
+ Variable F : (x:A)(x':B)((y:A)(y':B)(R (y,y') (x,x'))-> (P y y'))->(P x x').
+
+ Fixpoint Acc_iter_2 [x:A;x':B;a:(Acc ? R (x,x'))] : (P x x')
+ := (F x x' ([y:A][y':B][h:(R (y,y') (x,x'))](Acc_iter_2 y y' (Acc_inv ? ? (x,x') a (y,y') h)))).
+
+ Hypothesis Rwf : (well_founded ? R).
+
+ Theorem well_founded_induction_type_2 :
+ ((x:A)(x':B)((y:A)(y':B)(R (y,y') (x,x'))->(P y y'))->(P x x'))->(a:A)(b:B)(P a b).
+ Proof.
+ Intros; Apply Acc_iter_2; Auto.
+ Qed.
+
+End Well_founded_2.
+