aboutsummaryrefslogtreecommitdiffstats
path: root/backend/LTLin.v
diff options
context:
space:
mode:
Diffstat (limited to 'backend/LTLin.v')
-rw-r--r--backend/LTLin.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/backend/LTLin.v b/backend/LTLin.v
index 64017c30..806a7aa9 100644
--- a/backend/LTLin.v
+++ b/backend/LTLin.v
@@ -225,7 +225,7 @@ Inductive step: state -> trace -> state -> Prop :=
E0 (State s f (Vptr stk Int.zero) f.(fn_code) (init_locs args f.(fn_params)) m')
| exec_function_external:
forall s ef args t res m m',
- external_call ef (Genv.find_symbol ge) args m t res m' ->
+ external_call ef ge args m t res m' ->
step (Callstate s (External ef) args m)
t (Returnstate s res m')
| exec_return: