aboutsummaryrefslogtreecommitdiffstats
path: root/cfrontend/Csyntax.v
diff options
context:
space:
mode:
authorxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2012-12-30 17:47:53 +0000
committerxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2012-12-30 17:47:53 +0000
commit5bf13140754a55599ae27942b17cdbb4b7ed74e9 (patch)
tree57d4ef372149baf47291ad21e65ec77bf9ae15cb /cfrontend/Csyntax.v
parent71dfc9f28a1bf4b62c586b3ebee8e2c78088fd84 (diff)
downloadcompcert-kvx-5bf13140754a55599ae27942b17cdbb4b7ed74e9.tar.gz
compcert-kvx-5bf13140754a55599ae27942b17cdbb4b7ed74e9.zip
Remove some useless "Require".
Update ARM port. git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@2085 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'cfrontend/Csyntax.v')
-rw-r--r--cfrontend/Csyntax.v1
1 files changed, 0 insertions, 1 deletions
diff --git a/cfrontend/Csyntax.v b/cfrontend/Csyntax.v
index 51556897..6c333aac 100644
--- a/cfrontend/Csyntax.v
+++ b/cfrontend/Csyntax.v
@@ -16,7 +16,6 @@
(** Abstract syntax for the Compcert C language *)
Require Import Coqlib.
-Require Import Errors.
Require Import Integers.
Require Import Floats.
Require Import Values.