aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Bool/DecBool.v
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-03-16 22:45:07 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-03-16 22:45:07 +0000
commit93da0ad0e56bf54f1be8913d0a5832868fc6be7c (patch)
tree966b7f847b5c8ffef75723fa6f44f8c9e574d56f /theories/Bool/DecBool.v
parent629ac006253938d252529edb56dd2442e8e6b76f (diff)
mise sous CVS
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@318 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Bool/DecBool.v')
-rwxr-xr-xtheories/Bool/DecBool.v20
1 files changed, 20 insertions, 0 deletions
diff --git a/theories/Bool/DecBool.v b/theories/Bool/DecBool.v
new file mode 100755
index 000000000..a713c0409
--- /dev/null
+++ b/theories/Bool/DecBool.v
@@ -0,0 +1,20 @@
+
+(* $Id$ *)
+
+Implicit Arguments On.
+
+Definition ifdec : (A,B:Prop)(C:Set)({A}+{B})->C->C->C
+ := [A,B,C,H,x,y]if H then [_]x else [_]y.
+
+
+Theorem ifdec_left : (A,B:Prop)(C:Set)(H:{A}+{B})~B->(x,y:C)(ifdec H x y)=x.
+Intros; Case H; Auto.
+Intro; Absurd B; Trivial.
+Save.
+
+Theorem ifdec_right : (A,B:Prop)(C:Set)(H:{A}+{B})~A->(x,y:C)(ifdec H x y)=y.
+Intros; Case H; Auto.
+Intro; Absurd A; Trivial.
+Save.
+
+Implicit Arguments Off.