summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/shouldsucceed/1582.v
blob: 47953a66f99b05b7b48d2fb26530061a3cd4494d (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
Require Import Peano_dec.

Definition fact_F : 
  forall (n:nat),
  (forall m, m<n -> nat) ->
  nat.
refine 
  (fun n fact_rec =>
     if eq_nat_dec n 0 then 
        1
     else
        let fn := fact_rec (n-1) _ in
        n * fn).
Admitted.