X-Git-Url: http://git.megacz.com/?p=coq-hetmet.git;a=blobdiff_plain;f=src%2FExtractionMain.v;h=dbeb3ccec21ea55152b6015ccd2fa9d0f529cd70;hp=2b65a182ac5efc36942cbd4f67d4449fd03c3b83;hb=42d914b9626cdacdc2e4ff3a4ea5f2ce0e39071d;hpb=97552c1a6dfb32098d4491951929ab1d4aca96a0 diff --git a/src/ExtractionMain.v b/src/ExtractionMain.v index 2b65a18..dbeb3cc 100644 --- a/src/ExtractionMain.v +++ b/src/ExtractionMain.v @@ -34,12 +34,13 @@ Require Import HaskStrongToWeak. Require Import HaskWeakToCore. Require Import HaskProofToStrong. +Require Import ProgrammingLanguage. + Require Import HaskProofCategory. (* Require Import HaskStrongCategory. -Require Import ReificationsEquivalentToGeneralizedArrows. -Require Import ProgrammingLanguage. *) +Require Import ReificationsIsomorphicToGeneralizedArrows. Open Scope string_scope. Extraction Language Haskell. @@ -99,7 +100,8 @@ Section core2proof. Definition ξ (cv:CoreVar) : LeveledHaskType Γ ★ := match coreVarToWeakVar cv with | WExprVar wev => match weakTypeToTypeOfKind φ wev ★ with - | Error s => Prelude_error ("Error in top-level xi: " +++ s) + | Error s => Prelude_error ("Error converting weakType of top-level variable "+++ + toString cv+++": " +++ s) | OK t => t @@ nil end | WTypeVar _ => Prelude_error "top-level xi got a type variable"