summaryrefslogtreecommitdiff
path: root/cfrontend/Clight.v
diff options
context:
space:
mode:
authorGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2010-08-18 09:58:24 +0000
committerGravatar xleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2010-08-18 09:58:24 +0000
commit6f9b68c8de22fe540bfe85c2fabec4b967c6a80d (patch)
treebcdc970a7cd51c9edc74cfe2d428b7d2f7205b61 /cfrontend/Clight.v
parentdcaf93a7432304b3479ed191607aa4cd2966baf3 (diff)
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/Clight.v')
-rw-r--r--cfrontend/Clight.v1
1 files changed, 0 insertions, 1 deletions
diff --git a/cfrontend/Clight.v b/cfrontend/Clight.v
index 4cc97ab..4f4123e 100644
--- a/cfrontend/Clight.v
+++ b/cfrontend/Clight.v
@@ -533,7 +533,6 @@ Inductive step: state -> trace -> state -> Prop :=
E0 (State f Sskip k e le m)
| step_return_0: forall f k e le m m',
- f.(fn_return) = Tvoid ->
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')