aboutsummaryrefslogtreecommitdiffstats
path: root/cfrontend/Csharpminor.v
diff options
context:
space:
mode:
authorxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2011-08-19 09:13:09 +0000
committerxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2011-08-19 09:13:09 +0000
commit7ea8a55692e2a2d32efa0c84e19c37a3b56a0fd1 (patch)
treee324aff1a958e0a5d83f805ff3ca1d9eb07939f4 /cfrontend/Csharpminor.v
parent5b73a4f223a0cadb7df3f1320fed86cde0d67d6e (diff)
downloadcompcert-kvx-7ea8a55692e2a2d32efa0c84e19c37a3b56a0fd1.tar.gz
compcert-kvx-7ea8a55692e2a2d32efa0c84e19c37a3b56a0fd1.zip
Cleaned up old commented-out parts
git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@1719 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'cfrontend/Csharpminor.v')
-rw-r--r--cfrontend/Csharpminor.v9
1 files changed, 0 insertions, 9 deletions
diff --git a/cfrontend/Csharpminor.v b/cfrontend/Csharpminor.v
index c192e463..a1ed8b33 100644
--- a/cfrontend/Csharpminor.v
+++ b/cfrontend/Csharpminor.v
@@ -416,15 +416,6 @@ Inductive exec_assign: env -> mem -> ident -> val -> mem -> Prop :=
Mem.store chunk m b 0 v = Some m' ->
exec_assign e m id v m'.
-(*
-Inductive exec_opt_assign: env -> mem -> option ident -> val -> mem -> Prop :=
- | exec_assign_none: forall e m v,
- exec_opt_assign e m None v m
- | exec_assign_some: forall e m id v m',
- exec_assign e m id v m' ->
- exec_opt_assign e m (Some id) v m'.
-*)
-
(** One step of execution *)
Inductive step: state -> trace -> state -> Prop :=