X-Git-Url: http://git.megacz.com/?a=blobdiff_plain;ds=sidebyside;f=src%2FHaskProofToLatex.v;h=61a0bdb5e56a6d9f98c1303deb6771ca8fffe9c6;hb=a9a60dc234f76a4740b32c0f62aa0fe3a89fea83;hp=0d33b0aebfe6986efb3c9a0bc4b0ef8eaad5f4e5;hpb=b4857a6f575dffd5c9c9d5decbc21ff63a338270;p=coq-hetmet.git diff --git a/src/HaskProofToLatex.v b/src/HaskProofToLatex.v index 0d33b0a..61a0bdb 100644 --- a/src/HaskProofToLatex.v +++ b/src/HaskProofToLatex.v @@ -11,7 +11,8 @@ Require Import Coq.Lists.List. Require Import HaskKinds. Require Import HaskWeakVars. Require Import HaskWeakTypes. -Require Import HaskLiteralsAndTyCons. +Require Import HaskLiterals. +Require Import HaskTyCons. Require Import HaskStrongTypes. Require Import HaskStrong. Require Import HaskProof. @@ -160,6 +161,7 @@ Fixpoint nd_uruleToRawLatexMath {T}{h}{c}(r:@Arrange T h c) : string := match r with | RLeft _ _ _ r => nd_uruleToRawLatexMath r | RRight _ _ _ r => nd_uruleToRawLatexMath r + | RId _ => "Id" | RCanL _ => "CanL" | RCanR _ => "CanR" | RuCanL _ => "uCanL" @@ -187,12 +189,13 @@ Fixpoint nd_ruleToRawLatexMath {h}{c}(r:Rule h c) : string := | RAbsCo _ _ _ _ _ _ _ _ => "AbsCo" | RApp _ _ _ _ _ _ _ => "App" | RLet _ _ _ _ _ _ _ => "Let" - | RJoin _ _ _ _ _ _ => "RJoin" + | RWhere _ _ _ _ _ _ _ _ => "Where" + | RJoin _ _ _ _ _ _ => "RJoin" | RLetRec _ _ _ _ _ _ => "LetRec" | RCase _ _ _ _ _ _ _ _ => "Case" | RBrak _ _ _ _ _ _ => "Brak" | REsc _ _ _ _ _ _ => "Esc" - | RVoid _ _ => "RVoid" + | RVoid _ _ => "RVoid" end. Fixpoint nd_hideURule {T}{h}{c}(r:@Arrange T h c) : bool :=