aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Bool
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-05 21:10:29 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-05 21:10:29 +0000
commit9fa2e7e48f3259758a462d8de30cfd66af78c627 (patch)
treec9a7b28ad183f3b44910ded5b6fdd807874e2a44 /theories/Bool
parenteb196f1e86b446bffc9a2fff672be2f3fd589182 (diff)
Plus besoin de débrancher la preuve qui ne passait pas
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@804 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Bool')
-rwxr-xr-xtheories/Bool/Bool.v2
1 files changed, 0 insertions, 2 deletions
diff --git a/theories/Bool/Bool.v b/theories/Bool/Bool.v
index 7737c4837..c49c4bf8e 100755
--- a/theories/Bool/Bool.v
+++ b/theories/Bool/Bool.v
@@ -106,7 +106,6 @@ 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 .
@@ -122,7 +121,6 @@ Intros H.
Inversion_clear H.
Trivial with bool.
Save.
-*****)
Lemma eqb_reflx : (b:bool)(eqb b b)=true.
Intro b.