summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/shouldsucceed/1618.v
blob: a90290bfb21eac400fc72ccd3350116bc2bbb019 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
Inductive A: Set :=
| A1: nat -> A.

Definition A_size (a: A) : nat :=
  match a with
    | A1 n => 0
  end.

Require Import Recdef. 

Function n3 (P: A -> Prop) (f: forall n, P (A1 n)) (a: A) {struct a} : P a :=
  match a  return (P a) with
    | A1 n => f n
  end.


Function n1 (P: A -> Prop) (f: forall n, P (A1 n)) (a: A) {measure A_size a} :
P
a :=
  match a return (P a) with
    | A1 n => f n
  end.