File: bug_19047.out

package info (click to toggle)
coq 8.20.1%2Bdfsg-1
  • links: PTS, VCS
  • area: main
  • in suites: forky, sid, trixie
  • size: 44,116 kB
  • sloc: ml: 234,160; sh: 4,301; python: 3,270; ansic: 2,644; makefile: 882; lisp: 172; javascript: 63; xml: 24; sed: 2
file content (25 lines) | stat: -rw-r--r-- 758 bytes parent folder | download | duplicates (2)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
File "./output/bug_19047.v", line 11, characters 2-135:
The command has indeed failed with message:
Recursive definition of F is ill-formed.
In environment
coacc_rect :
  forall (A : Type) (R : A -> A -> Prop) (P : A -> Type),
  (forall x : A,
   (forall y : A, R x y -> coAcc R y) -> (forall y : A, R x y -> P y) -> P x) ->
  forall x : A, coAcc R x -> P x
A : Type
R : A -> A -> Prop
P : A -> Type
f :
  forall x : A,
  (forall y : A, R x y -> coAcc R y) -> (forall y : A, R x y -> P y) -> P x
F : forall x : A, coAcc R x -> P x
x : R
a : coAcc P x
The codomain is "f x"
which should be a coinductive type.
Recursive definition is:
"fun (x : A) (a : coAcc R x) =>
 match a with
 | coAcc_intro _ _ g => f x g (fun (y : A) (r : R x y) => F y (g y r))
 end".