aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Bool
diff options
context:
space:
mode:
authorGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-19 12:25:05 +0000
committerGravatar mohring <mohring@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-04-19 12:25:05 +0000
commitbdbbb1bea47909ad5d0daffd77e090ef9b59d826 (patch)
tree4d1265dfb29299fb395a554a3b32eb550b4662a2 /theories/Bool
parent45aa164112c77d61f726d5db32041c9518ed378a (diff)
Mise de (*i autour CVS info
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1619 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Bool')
-rwxr-xr-xtheories/Bool/Bool.v8
-rwxr-xr-xtheories/Bool/DecBool.v6
-rwxr-xr-xtheories/Bool/IfProp.v2
-rw-r--r--theories/Bool/Sumbool.v2
-rwxr-xr-xtheories/Bool/Zerob.v2
5 files changed, 10 insertions, 10 deletions
diff --git a/theories/Bool/Bool.v b/theories/Bool/Bool.v
index 459c145e1..4f7df44fd 100755
--- a/theories/Bool/Bool.v
+++ b/theories/Bool/Bool.v
@@ -6,14 +6,14 @@
(* * GNU Lesser General Public License Version 2.1 *)
(***********************************************************************)
-(* $Id$ *)
+(*i $Id$ i*)
(*************)
-(*s Booleans *)
+(* Booleans *)
(* The type [bool] is defined in the prelude as \\
- [Inductive bool : Set := true : bool | false : bool (from Prelude)] *)
+ [Inductive bool : Set := true : bool | false : bool] *)
-(*s Interpretation of booleans as Propopsition *)
+(* Interpretation of booleans as Proposition *)
Definition Is_true := [b:bool](Cases b of
true => True
| false => False
diff --git a/theories/Bool/DecBool.v b/theories/Bool/DecBool.v
index 59278ec11..8daabd479 100755
--- a/theories/Bool/DecBool.v
+++ b/theories/Bool/DecBool.v
@@ -6,9 +6,9 @@
(* * GNU Lesser General Public License Version 2.1 *)
(***********************************************************************)
-(* $Id$ *)
+(*i $Id$ i*)
-Implicit Arguments On.
+Set Implicit Arguments.
Definition ifdec : (A,B:Prop)(C:Set)({A}+{B})->C->C->C
:= [A,B,C,H,x,y]if H then [_]x else [_]y.
@@ -24,4 +24,4 @@ Intros; Case H; Auto.
Intro; Absurd A; Trivial.
Save.
-Implicit Arguments Off.
+Unset Implicit Arguments.
diff --git a/theories/Bool/IfProp.v b/theories/Bool/IfProp.v
index f4c4d4cb4..bcbe0f714 100755
--- a/theories/Bool/IfProp.v
+++ b/theories/Bool/IfProp.v
@@ -6,7 +6,7 @@
(* * GNU Lesser General Public License Version 2.1 *)
(***********************************************************************)
-(* $Id$ *)
+(*i $Id$ i*)
Require Bool.
diff --git a/theories/Bool/Sumbool.v b/theories/Bool/Sumbool.v
index 749accdd4..e91b3fb1a 100644
--- a/theories/Bool/Sumbool.v
+++ b/theories/Bool/Sumbool.v
@@ -6,7 +6,7 @@
(* * GNU Lesser General Public License Version 2.1 *)
(***********************************************************************)
-(* $Id$ *)
+(*i $Id$ i*)
(* Here are collected some results about the type sumbool (see INIT/Specif.v)
*
diff --git a/theories/Bool/Zerob.v b/theories/Bool/Zerob.v
index b36fc94d5..8a8d09621 100755
--- a/theories/Bool/Zerob.v
+++ b/theories/Bool/Zerob.v
@@ -6,7 +6,7 @@
(* * GNU Lesser General Public License Version 2.1 *)
(***********************************************************************)
-(* $Id$ *)
+(*i $Id$ i*)
Require Arith.
Require Bool.