aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Bool
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-05-02 20:49:25 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-05-02 20:49:25 +0000
commit5b0f516e7e1f6d2ea8ca0485ffe347a613b01a5c (patch)
treebf106a29e38172fcbd0ee48bc4531c07d46ff5aa /theories/Bool
parent1555e5a4cf7c2662d31d7875f7cc217150b49f4c (diff)
portage Omega (mais toujours pas Zpower et Zlogarithm)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@400 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Bool')
-rwxr-xr-xtheories/Bool/Bool.v4
1 files changed, 3 insertions, 1 deletions
diff --git a/theories/Bool/Bool.v b/theories/Bool/Bool.v
index 7f8f52c4f..ab1a4b9e0 100755
--- a/theories/Bool/Bool.v
+++ b/theories/Bool/Bool.v
@@ -106,6 +106,7 @@ Lemma Is_true_eq_true2 : (x:bool) x=true -> (Is_true x).
Destruct x; Simpl; Auto with bool.
Save.
+(***** TODO
Lemma eqb_subst :
(P:bool->Prop)(b1,b2:bool)(eqb b1 b2)=true->(P b1)->(P b2).
Unfold eqb .
@@ -121,7 +122,8 @@ Intros H.
Inversion_clear H.
Trivial with bool.
Save.
-
+*****)
+
Lemma eqb_reflx : (b:bool)(eqb b b)=true.
Intro b.
Case b.