X-Git-Url: http://git.megacz.com/?p=coq-hetmet.git;a=blobdiff_plain;f=src%2FHaskStrong.v;h=c5f46dc5bf216017125b123131c766d639b20843;hp=d688c2f66cf8a1fd5eda4f5b53fa372af45160dd;hb=ec8ee5cde986e5b38bcae38cda9e63eba94f1d9f;hpb=97552c1a6dfb32098d4491951929ab1d4aca96a0 diff --git a/src/HaskStrong.v b/src/HaskStrong.v index d688c2f..c5f46dc 100644 --- a/src/HaskStrong.v +++ b/src/HaskStrong.v @@ -20,7 +20,6 @@ Section HaskStrong. Context `{EQD_VV:EqDecidable VV}. (* a StrongCaseBranchWithVVs contains all the data found in a case branch except the expression itself *) - Record StrongCaseBranchWithVVs {tc:TyCon}{Γ}{atypes:IList _ (HaskType Γ) (tyConKind tc)}{sac:@StrongAltCon tc} := { scbwv_exprvars : vec VV (sac_numExprVars sac) ; scbwv_exprvars_distinct : distinct (vec2list scbwv_exprvars) @@ -28,7 +27,6 @@ Section HaskStrong. ; scbwv_ξ := fun ξ lev => update_ξ (weakLT'○ξ) (weakL' lev) (vec2list scbwv_varstypes) }. Implicit Arguments StrongCaseBranchWithVVs [[Γ]]. - (*Coercion scbwv_sac : StrongCaseBranchWithVVs >-> StrongAltCon.*) Inductive Expr : forall Γ (Δ:CoercionEnv Γ), (VV -> LeveledHaskType Γ ★) -> LeveledHaskType Γ ★ -> Type :=