X-Git-Url: http://git.megacz.com/?p=coq-hetmet.git;a=blobdiff_plain;f=src%2FHaskKinds.v;h=3539e953ab946166f39e094c64d0157a5a4281d8;hp=54a1f64459375759e49cbf6d13edd7719ed05f2d;hb=ec8ee5cde986e5b38bcae38cda9e63eba94f1d9f;hpb=3d56944e3882ec751fa99b4476a013c4d86fd0f8 diff --git a/src/HaskKinds.v b/src/HaskKinds.v index 54a1f64..3539e95 100644 --- a/src/HaskKinds.v +++ b/src/HaskKinds.v @@ -12,7 +12,6 @@ Variable Note : Type. Extract Inlined Con Variable natToString : nat -> string. Extract Inlined Constant natToString => "natToString". Instance NatToStringInstance : ToString nat := { toString := natToString }. -(* Figure 7: production κ, ι *) Inductive Kind : Type := | KindStar : Kind (* ★ - the kind of coercions and the kind of types inhabited by [boxed] values *) | KindArrow : Kind -> Kind -> Kind (* ⇛ - type-function-space; things of kind X⇛Y are NOT inhabited by expressions*) @@ -38,6 +37,18 @@ Instance KindToString : ToString Kind := { toString := kindToString }. Notation "'★'" := KindStar. Notation "a ⇛ b" := (KindArrow a b). +Fixpoint kindToLatexMath (k:Kind) : LatexMath := + match k with + | ★ => rawLatexMath "\star" + | ★ ⇛ k2 => (rawLatexMath "\star\Rightarrow ")+++kindToLatexMath k2 + | k1 ⇛ k2 => (rawLatexMath "(")+++kindToLatexMath k1+++(rawLatexMath ")\Rightarrow ")+++kindToLatexMath k2 + | KindUnliftedType => rawLatexMath "\text{\tt{\#}}" + | KindUnboxedTuple => rawLatexMath "\text{\tt{(\#)}}" + | KindArgType => rawLatexMath "\text{\tt{??}}" + | KindOpenType => rawLatexMath "\text{\tt{?}}" + end. +Instance KindToLatexMath : ToLatexMath Kind := { toLatexMath := kindToLatexMath }. + Instance KindEqDecidable : EqDecidable Kind. apply Build_EqDecidable. induction v1.