aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--theories/Init/DatatypesSyntax.v10
-rw-r--r--theories/Init/PeanoSyntax.v12
-rwxr-xr-xtheories/Init/Prelude.v2
3 files changed, 0 insertions, 24 deletions
diff --git a/theories/Init/DatatypesSyntax.v b/theories/Init/DatatypesSyntax.v
deleted file mode 100644
index a4b6a57aa..000000000
--- a/theories/Init/DatatypesSyntax.v
+++ /dev/null
@@ -1,10 +0,0 @@
-(***********************************************************************)
-(* v * The Coq Proof Assistant / The Coq Development Team *)
-(* <O___,, * INRIA-Rocquencourt & LRI-CNRS-Orsay *)
-(* \VV/ *************************************************************)
-(* // * This file is distributed under the terms of the *)
-(* * GNU Lesser General Public License Version 2.1 *)
-(***********************************************************************)
-
-(*i $Id$ i*)
-
diff --git a/theories/Init/PeanoSyntax.v b/theories/Init/PeanoSyntax.v
deleted file mode 100644
index 3b7b91454..000000000
--- a/theories/Init/PeanoSyntax.v
+++ /dev/null
@@ -1,12 +0,0 @@
-(***********************************************************************)
-(* v * The Coq Proof Assistant / The Coq Development Team *)
-(* <O___,, * INRIA-Rocquencourt & LRI-CNRS-Orsay *)
-(* \VV/ *************************************************************)
-(* // * This file is distributed under the terms of the *)
-(* * GNU Lesser General Public License Version 2.1 *)
-(***********************************************************************)
-(*i $Id$ *)
-
-Require Datatypes.
-Require Peano.
-
diff --git a/theories/Init/Prelude.v b/theories/Init/Prelude.v
index 51a62db8e..972a80986 100755
--- a/theories/Init/Prelude.v
+++ b/theories/Init/Prelude.v
@@ -10,11 +10,9 @@
Require Export Notations.
Require Export Datatypes.
-Require Export DatatypesSyntax.
Require Export Logic.
Require Export LogicSyntax.
Require Export Specif.
Require Export SpecifSyntax.
Require Export Peano.
-Require Export PeanoSyntax.
Require Export Wf.