summaryrefslogtreecommitdiff
path: root/cfrontend/Cexec.v
diff options
context:
space:
mode:
Diffstat (limited to 'cfrontend/Cexec.v')
-rw-r--r--cfrontend/Cexec.v16
1 files changed, 14 insertions, 2 deletions
diff --git a/cfrontend/Cexec.v b/cfrontend/Cexec.v
index 3dd34c1..383eeb8 100644
--- a/cfrontend/Cexec.v
+++ b/cfrontend/Cexec.v
@@ -1,3 +1,17 @@
+(* *********************************************************************)
+(* *)
+(* The Compcert verified compiler *)
+(* *)
+(* Xavier Leroy, INRIA Paris-Rocquencourt *)
+(* *)
+(* Copyright Institut National de Recherche en Informatique et en *)
+(* Automatique. All rights reserved. This file is distributed *)
+(* under the terms of the INRIA Non-Commercial License Agreement. *)
+(* *)
+(* *********************************************************************)
+
+(** Animating the CompCert C semantics *)
+
Require Import Axioms.
Require Import Coqlib.
Require Import Errors.
@@ -14,8 +28,6 @@ Require Import Csyntax.
Require Import Csem.
Require Cstrategy.
-(** Animating the CompCert C semantics *)
-
Lemma type_eq: forall (ty1 ty2: type), {ty1=ty2} + {ty1<>ty2}
with typelist_eq: forall (tyl1 tyl2: typelist), {tyl1=tyl2} + {tyl1<>tyl2}
with fieldlist_eq: forall (fld1 fld2: fieldlist), {fld1=fld2} + {fld1<>fld2}.