X-Git-Url: http://git.megacz.com/?a=blobdiff_plain;f=src%2FExtractionMain.v;h=2f0856fc199537a40117c4f548f473867cc4a812;hb=be2a24c17877b3401c3c46bee1436b8ec0bbdaf5;hp=61993a1515802b1d9f14e812de3ad19a864f4450;hpb=992203bb4a221ea2f415c0d14bb34d35af2ee637;p=coq-hetmet.git diff --git a/src/ExtractionMain.v b/src/ExtractionMain.v index 61993a1..2f0856f 100644 --- a/src/ExtractionMain.v +++ b/src/ExtractionMain.v @@ -40,7 +40,7 @@ Require Import HaskProofCategory. (* Require Import HaskStrongCategory. *) -Require Import ReificationsEquivalentToGeneralizedArrows. +Require Import ReificationsIsomorphicToGeneralizedArrows. Open Scope string_scope. Extraction Language Haskell. @@ -62,7 +62,7 @@ Extract Inlined Constant string_dec => "(==)". Extract Inlined Constant ascii_dec => "(==)". (* adapted from ExtrOcamlString.v *) -Extract Inductive ascii => "Char" [ "bin2ascii" ] "bin2ascii'". +Extract Inductive ascii => "Char" [ "you_forgot_to_patch_coq" ] "you_forgot_to_patch_coq". Extract Constant zero => "'\000'". Extract Constant one => "'\001'". Extract Constant shift => "shiftAscii". @@ -100,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"