summaryrefslogtreecommitdiff
path: root/test-suite/failure/Case2.v
blob: 183f612b0491654f14564d0491d9c3026fcf3e1b (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
Inductive IFExpr : Set := 
          Var  : nat -> IFExpr
        | Tr   : IFExpr
        | Fa   : IFExpr
        | IfE   : IFExpr -> IFExpr -> IFExpr -> IFExpr.

Type [F:IFExpr]
    <Prop>Cases F of
       (IfE (Var _) H I) => True
     | (IfE _ _ _)   => False
     |  _          => True
     end.