aboutsummaryrefslogtreecommitdiffstats
path: root/common/Errors.v
diff options
context:
space:
mode:
authorxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2012-03-09 09:52:04 +0000
committerxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2012-03-09 09:52:04 +0000
commit8a64451e6f474d20a469b939a938577bbe6d3d66 (patch)
treee49a52973b9fbf726ba2ceff3e7af0ee2b84e617 /common/Errors.v
parent8a26cc219f8c8211301f021bd0ee4a27153528f8 (diff)
downloadcompcert-kvx-8a64451e6f474d20a469b939a938577bbe6d3d66.tar.gz
compcert-kvx-8a64451e6f474d20a469b939a938577bbe6d3d66.zip
Merge of Andrew Tolmach's HASP-related changes
git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@1838 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'common/Errors.v')
-rw-r--r--common/Errors.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/common/Errors.v b/common/Errors.v
index 36e70c5d..a70ea6ea 100644
--- a/common/Errors.v
+++ b/common/Errors.v
@@ -30,7 +30,8 @@ Set Implicit Arguments.
Inductive errcode: Type :=
| MSG: string -> errcode
- | CTX: positive -> errcode.
+ | CTX: positive -> errcode (* a top-level identifier *)
+ | CTXL: positive -> errcode. (* an encoded local identifier *)
Definition errmsg: Type := list errcode.