X-Git-Url: http://git.megacz.com/?p=coq-hetmet.git;a=blobdiff_plain;f=src%2FExtraction.v;fp=src%2FExtraction.v;h=3371ed5199e7305e44fad21ecad2c818a476f726;hp=e2e380086947baafec36071820027f86ce6bd699;hb=5c493a75fbaf8454d8a21e55edc5b193e2c5879c;hpb=6232ffa2805211654c6ff40a9852d7fc312382d2 diff --git a/src/Extraction.v b/src/Extraction.v index e2e3800..3371ed5 100644 --- a/src/Extraction.v +++ b/src/Extraction.v @@ -77,10 +77,14 @@ Section core2proof. (* We need to be able to resolve unbound exprvars, but we can be sure their types will have no * free tyvars in them *) - Definition ξ (wev:WeakExprVar) : LeveledHaskType Γ ★ := - match weakTypeToType' φ wev ★ with - | Error s => fail ("Error in top-level xi: " +++ s) - | OK t => t @@ nil + Definition ξ (cv:CoreVar) : LeveledHaskType Γ ★ := + match coreVarToWeakVar cv with + | WExprVar wev => match weakTypeToType' φ wev ★ with + | Error s => fail ("Error in top-level xi: " +++ s) + | OK t => t @@ nil + end + | WTypeVar _ => fail "top-level xi got a type variable" + | WCoerVar _ => fail "top-level xi got a coercion variable" end. Definition header : string :=