aboutsummaryrefslogtreecommitdiffstats
path: root/cfrontend/SimplExprproof.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/SimplExprproof.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/SimplExprproof.v')
-rw-r--r--cfrontend/SimplExprproof.v2
1 files changed, 0 insertions, 2 deletions
diff --git a/cfrontend/SimplExprproof.v b/cfrontend/SimplExprproof.v
index 7fc0a46e..59fc9bc7 100644
--- a/cfrontend/SimplExprproof.v
+++ b/cfrontend/SimplExprproof.v
@@ -12,8 +12,6 @@
(** Correctness proof for expression simplification. *)
-Require Import Coq.Program.Equality.
-Require Import Axioms.
Require Import Coqlib.
Require Import Maps.
Require Import AST.