summaryrefslogtreecommitdiff
path: root/cfrontend/ClightBigstep.v
diff options
context:
space:
mode:
authorGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2012-12-30 17:47:53 +0000
committerGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2012-12-30 17:47:53 +0000
commit5bf13140754a55599ae27942b17cdbb4b7ed74e9 (patch)
tree57d4ef372149baf47291ad21e65ec77bf9ae15cb /cfrontend/ClightBigstep.v
parent71dfc9f28a1bf4b62c586b3ebee8e2c78088fd84 (diff)
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/ClightBigstep.v')
-rw-r--r--cfrontend/ClightBigstep.v1
1 files changed, 0 insertions, 1 deletions
diff --git a/cfrontend/ClightBigstep.v b/cfrontend/ClightBigstep.v
index 293ea5d..4d10c62 100644
--- a/cfrontend/ClightBigstep.v
+++ b/cfrontend/ClightBigstep.v
@@ -16,7 +16,6 @@
(** A big-step semantics for the Clight language. *)
Require Import Coqlib.
-Require Import Errors.
Require Import Maps.
Require Import Integers.
Require Import Floats.