@@ -1041,7 +1041,8 @@ mapPTermFC f g (PDoBlock dos) = PDoBlock (map mapPDoFC dos)
10411041 mapPDoFC (DoBindP fc t1 t2 alts) =
10421042 DoBindP (f fc) (mapPTermFC f g t1) (mapPTermFC f g t2) (map (\ (l,r)-> (mapPTermFC f g l, mapPTermFC f g r)) alts)
10431043 mapPDoFC (DoLet fc rc n nfc t1 t2) = DoLet (f fc) rc n (g nfc) (mapPTermFC f g t1) (mapPTermFC f g t2)
1044- mapPDoFC (DoLetP fc t1 t2) = DoLetP (f fc) (mapPTermFC f g t1) (mapPTermFC f g t2)
1044+ mapPDoFC (DoLetP fc t1 t2 alts) =
1045+ DoLetP (f fc) (mapPTermFC f g t1) (mapPTermFC f g t2) (map (\ (l,r) -> (mapPTermFC f g l, mapPTermFC f g r)) alts)
10451046 mapPDoFC (DoRewrite fc h) = DoRewrite (f fc) (mapPTermFC f g h)
10461047mapPTermFC f g (PIdiom fc t) = PIdiom (f fc) (mapPTermFC f g t)
10471048mapPTermFC f g (PMetavar fc n) = PMetavar (g fc) n
@@ -1166,7 +1167,7 @@ data PDo' t = DoExp FC t
11661167 | DoBind FC Name FC t -- ^ second FC is precise name location
11671168 | DoBindP FC t t [(t ,t )]
11681169 | DoLet FC RigCount Name FC t t -- ^ second FC is precise name location
1169- | DoLetP FC t t
1170+ | DoLetP FC t t [( t , t )]
11701171 | DoRewrite FC t -- rewrite in do block
11711172 deriving (Eq , Ord , Functor , Data , Generic , Typeable )
11721173{- !
@@ -1178,7 +1179,7 @@ instance Sized a => Sized (PDo' a) where
11781179 size (DoBind fc nm nfc t) = 1 + size fc + size nm + size nfc + size t
11791180 size (DoBindP fc l r alts) = 1 + size fc + size l + size r + size alts
11801181 size (DoLet fc rc nm nfc l r) = 1 + size fc + size nm + size l + size r
1181- size (DoLetP fc l r) = 1 + size fc + size l + size r
1182+ size (DoLetP fc l r alts ) = 1 + size fc + size l + size r + size alts
11821183 size (DoRewrite fc h) = 1 + size fc + size h
11831184
11841185type PDo = PDo' PTerm
@@ -1274,7 +1275,7 @@ highestFC (PDoBlock lines) =
12741275 getDoFC (DoBind fc nm nfc t) = fc
12751276 getDoFC (DoBindP fc l r alts) = fc
12761277 getDoFC (DoLet fc rc nm nfc l r) = fc
1277- getDoFC (DoLetP fc l r) = fc
1278+ getDoFC (DoLetP fc l r alts) = fc
12781279 getDoFC (DoRewrite fc h) = fc
12791280
12801281highestFC (PIdiom fc _) = Just fc
@@ -1955,7 +1956,7 @@ pprintPTerm ppo bnd docArgs infixes = prettySe (ppopt_depth ppo) startPrec bnd
19551956 else text " =" ) <+>
19561957 group (align (hang 2 (prettySe (decD d) startPrec bnd v)))) :
19571958 ppdo ((ln, False ): bnd) dos
1958- ppdo bnd (DoLetP _ _ _ : dos) = -- ok because never made by delab
1959+ ppdo bnd (DoLetP _ _ _ _ : dos) = -- ok because never made by delab
19591960 text " no pretty printer for pattern-matching do binding" :
19601961 ppdo bnd dos
19611962 ppdo bnd (DoRewrite _ _ : dos) = -- ok because never made by delab
0 commit comments