aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Wf.v
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-02-19 09:35:01 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-02-19 09:35:01 +0000
commitd66a2e9671f9a4d0c0de92b5f2520e69e2747fd4 (patch)
treeb0154520af51e6b89d1f4a0ad13775dc82761120 /theories/Init/Wf.v
parentfd561b8d22aa7b04904d6fcd85036fdd6b255ca3 (diff)
Uniformisation des theoremes dans Set et Type (def. de Acc_rect et
well_founded_induction_type) git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2485 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init/Wf.v')
-rwxr-xr-xtheories/Init/Wf.v30
1 files changed, 19 insertions, 11 deletions
diff --git a/theories/Init/Wf.v b/theories/Init/Wf.v
index 58c159b78..78432dcf4 100755
--- a/theories/Init/Wf.v
+++ b/theories/Init/Wf.v
@@ -36,14 +36,16 @@ Chapter Well_founded.
(** the informative elimination :
[let Acc_rec F = let rec wf x = F x wf in wf] *)
- Section AccRec.
- Variable P : A -> Set.
+ Section AccRecType.
+ Variable P : A -> Type.
Variable F : (x:A)((y:A)(R y x)->(Acc y))->((y:A)(R y x)->(P y))->(P x).
- Fixpoint Acc_rec [x:A;a:(Acc x)] : (P x)
- := (F x (Acc_inv x a) ([y:A][h:(R y x)](Acc_rec y (Acc_inv x a y h)))).
+ Fixpoint Acc_rect [x:A;a:(Acc x)] : (P x)
+ := (F x (Acc_inv x a) ([y:A][h:(R y x)](Acc_rect y (Acc_inv x a y h)))).
- End AccRec.
+ End AccRecType.
+
+ Definition Acc_rec [P:A->Set] := (Acc_rect P).
(** A relation is well-founded if every element is accessible *)
@@ -53,17 +55,23 @@ Chapter Well_founded.
Hypothesis Rwf : well_founded.
- Theorem well_founded_induction :
+ Theorem well_founded_induction_type :
+ (P:A->Type)((x:A)((y:A)(R y x)->(P y))->(P x))->(a:A)(P a).
+ Proof.
+ Intros; Apply (Acc_rect P); Auto.
+ Save.
+
+ Theorem well_founded_induction :
(P:A->Set)((x:A)((y:A)(R y x)->(P y))->(P x))->(a:A)(P a).
Proof.
- Intros; Apply (Acc_rec P); Auto.
+ Exact [P:A->Set](well_founded_induction_type P).
Save.
- Theorem well_founded_ind :
+ Theorem well_founded_ind :
(P:A->Prop)((x:A)((y:A)(R y x)->(P y))->(P x))->(a:A)(P a).
- Proof.
- Intros; Apply (Acc_ind P); Auto.
- Qed.
+ Proof.
+ Exact [P:A->Prop](well_founded_induction_type P).
+ Qed.
(** Building fixpoints *)