aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-04-09 12:35:39 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-04-09 12:35:39 +0000
commit7ca14f9aba7a619853704e75efc2454f6a7406bf (patch)
tree4aa8cb8e11689b6ff8399940dea39cc83cd61d6d /theories/Init
parent974b4298df814d84304c76925310e2d19b3aca57 (diff)
Activation des implicites pour la v8
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3886 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init')
-rwxr-xr-xtheories/Init/Datatypes.v3
-rwxr-xr-xtheories/Init/Logic.v3
-rwxr-xr-xtheories/Init/Logic_Type.v3
-rwxr-xr-xtheories/Init/Specif.v3
-rwxr-xr-xtheories/Init/Wf.v3
5 files changed, 15 insertions, 0 deletions
diff --git a/theories/Init/Datatypes.v b/theories/Init/Datatypes.v
index 26608a294..aed8c53f5 100755
--- a/theories/Init/Datatypes.v
+++ b/theories/Init/Datatypes.v
@@ -8,6 +8,9 @@
(*i $Id$ i*)
+Set Implicit Arguments.
+V7only [Unset Implicit Arguments.].
+
(** [unit] is a singleton datatype with sole inhabitant [tt] *)
Inductive unit : Set := tt : unit.
diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v
index ab78af469..aace0f804 100755
--- a/theories/Init/Logic.v
+++ b/theories/Init/Logic.v
@@ -8,6 +8,9 @@
(*i $Id$ i*)
+Set Implicit Arguments.
+V7only [Unset Implicit Arguments.].
+
Require Datatypes.
(** [True] is the always true proposition *)
diff --git a/theories/Init/Logic_Type.v b/theories/Init/Logic_Type.v
index b5a6e6038..5ad3716ed 100755
--- a/theories/Init/Logic_Type.v
+++ b/theories/Init/Logic_Type.v
@@ -8,6 +8,9 @@
(*i $Id$ i*)
+Set Implicit Arguments.
+V7only [Unset Implicit Arguments.].
+
(** This module defines quantification on the world [Type]
([Logic.v] was defining it on the world [Set]) *)
diff --git a/theories/Init/Specif.v b/theories/Init/Specif.v
index daf7e5d85..77b9980f9 100755
--- a/theories/Init/Specif.v
+++ b/theories/Init/Specif.v
@@ -8,6 +8,9 @@
(*i $Id$ i*)
+Set Implicit Arguments.
+V7only [Unset Implicit Arguments.].
+
(** Basic specifications : Sets containing logical information *)
Require Datatypes.
diff --git a/theories/Init/Wf.v b/theories/Init/Wf.v
index 4fb640827..01509fa12 100755
--- a/theories/Init/Wf.v
+++ b/theories/Init/Wf.v
@@ -6,6 +6,9 @@
(* * GNU Lesser General Public License Version 2.1 *)
(***********************************************************************)
+Set Implicit Arguments.
+V7only [Unset Implicit Arguments.].
+
(*i $Id$ i*)
(** This module proves the validity of