summaryrefslogtreecommitdiff
path: root/backend/Lineartyping.v
diff options
context:
space:
mode:
Diffstat (limited to 'backend/Lineartyping.v')
-rw-r--r--backend/Lineartyping.v1
1 files changed, 0 insertions, 1 deletions
diff --git a/backend/Lineartyping.v b/backend/Lineartyping.v
index 3a0ee13..cbe1831 100644
--- a/backend/Lineartyping.v
+++ b/backend/Lineartyping.v
@@ -254,7 +254,6 @@ Definition wt_function (f: function) : Prop :=
Inductive wt_fundef: fundef -> Prop :=
| wt_fundef_external: forall ef,
- Conventions.sig_external_ok ef.(ef_sig) ->
wt_fundef (External ef)
| wt_function_internal: forall f,
wt_function f ->