aboutsummaryrefslogtreecommitdiffstats
path: root/cfrontend/Csharpminor.v
diff options
context:
space:
mode:
authorxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2010-08-18 09:58:24 +0000
committerxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2010-08-18 09:58:24 +0000
commit6f9b68c8de22fe540bfe85c2fabec4b967c6a80d (patch)
treebcdc970a7cd51c9edc74cfe2d428b7d2f7205b61 /cfrontend/Csharpminor.v
parentdcaf93a7432304b3479ed191607aa4cd2966baf3 (diff)
downloadcompcert-kvx-6f9b68c8de22fe540bfe85c2fabec4b967c6a80d.tar.gz
compcert-kvx-6f9b68c8de22fe540bfe85c2fabec4b967c6a80d.zip
Removed useless constraints on return type at Sreturn instructions
git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@1470 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'cfrontend/Csharpminor.v')
-rw-r--r--cfrontend/Csharpminor.v2
1 files changed, 0 insertions, 2 deletions
diff --git a/cfrontend/Csharpminor.v b/cfrontend/Csharpminor.v
index 1a362e32..2f05678e 100644
--- a/cfrontend/Csharpminor.v
+++ b/cfrontend/Csharpminor.v
@@ -512,12 +512,10 @@ Inductive step: state -> trace -> state -> Prop :=
E0 (State f (seq_of_lbl_stmt (select_switch n cases)) k e le m)
| step_return_0: forall f k e le m m',
- f.(fn_return) = None ->
Mem.free_list m (blocks_of_env e) = Some m' ->
step (State f (Sreturn None) k e le m)
E0 (Returnstate Vundef (call_cont k) m')
| step_return_1: forall f a k e le m v m',
- f.(fn_return) <> None ->
eval_expr e le m a v ->
Mem.free_list m (blocks_of_env e) = Some m' ->
step (State f (Sreturn (Some a)) k e le m)