aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/Case8.v
blob: b512b5f820482e395390ec9add191af5424cd86e (plain)
1
2
3
4
5
6
7
(* Check dependencies in the matching predicate (was failing in V8.0pl1) *)

Inductive t : (x:O=O) x=x -> Prop := 
  c : (x:0=0) (t x (refl_equal ? x)).

Definition a [x:(t ? (refl_equal ? (refl_equal ? O)))] :=
  <[_;_;x]Cases x of (c y) => Prop end>Cases x of (c y) => y=y end.