aboutsummaryrefslogtreecommitdiffstats
path: root/cfrontend/Clight.v
diff options
context:
space:
mode:
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 4cc97ab2..4f4123e0 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')