summaryrefslogtreecommitdiff
path: root/cfrontend/Csyntax.v
diff options
context:
space:
mode:
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 5155689..6c333aa 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.