aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic/ClassicalFacts.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-07 22:43:31 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-11-07 22:43:31 +0000
commit568366ceb8437efa002aaf5ca66a86b5c0c30020 (patch)
tree5a947a97f9ff900e92e336779d6d08b4cd1d345a /theories/Logic/ClassicalFacts.v
parentd35cb0f46fff92db0c44243f31beef4e29e2209f (diff)
Biblio standard sans mention de la possibilite d'etre impredicatif
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4823 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Logic/ClassicalFacts.v')
-rw-r--r--theories/Logic/ClassicalFacts.v22
1 files changed, 11 insertions, 11 deletions
diff --git a/theories/Logic/ClassicalFacts.v b/theories/Logic/ClassicalFacts.v
index bedbc4cbd..622e6959d 100644
--- a/theories/Logic/ClassicalFacts.v
+++ b/theories/Logic/ClassicalFacts.v
@@ -163,22 +163,22 @@ End Proof_irrelevance_gen.
Section Proof_irrelevance_CC.
-Definition Bool := (C:Prop)C->C->C.
-Definition True := [C][c1,c2]c1 : Bool.
-Definition False := [C][c1,c2]c2 : Bool.
-Definition Bool_elim := [C][c1,c2][b:Bool](b C c1 c2).
-Definition Bool_elim_redl : (C:Prop)(c1,c2:C)c1==(Bool_elim C c1 c2 True)
+Definition BoolP := (C:Prop)C->C->C.
+Definition TrueP := [C][c1,c2]c1 : BoolP.
+Definition FalseP := [C][c1,c2]c2 : BoolP.
+Definition BoolP_elim := [C][c1,c2][b:BoolP](b C c1 c2).
+Definition BoolP_elim_redl : (C:Prop)(c1,c2:C)c1==(BoolP_elim C c1 c2 TrueP)
:= [C;c1,c2](refl_eqT C c1).
-Definition Bool_elim_redr : (C:Prop)(c1,c2:C)c2==(Bool_elim C c1 c2 False)
+Definition BoolP_elim_redr : (C:Prop)(c1,c2:C)c2==(BoolP_elim C c1 c2 FalseP)
:= [C;c1,c2](refl_eqT C c2).
-Definition Bool_dep_induction :=
- (P:Bool->Prop)(P True)->(P False)->(b:Bool)(P b).
+Definition BoolP_dep_induction :=
+ (P:BoolP->Prop)(P TrueP)->(P FalseP)->(b:BoolP)(P b).
Lemma ext_prop_dep_proof_irrel_cc :
- prop_extensionality -> Bool_dep_induction -> proof_irrelevance.
-Proof (ext_prop_dep_proof_irrel_gen Bool True False Bool_elim
- Bool_elim_redl Bool_elim_redr).
+ prop_extensionality -> BoolP_dep_induction -> proof_irrelevance.
+Proof (ext_prop_dep_proof_irrel_gen BoolP TrueP FalseP BoolP_elim
+ BoolP_elim_redl BoolP_elim_redr).
End Proof_irrelevance_CC.