index
:
coq
master
the Coq proof assistant
about
summary
refs
log
tree
commit
diff
homepage
log msg
author
committer
range
path:
root
/
test-suite
/
output
/
Inductive.v
blob: 8db8956e32f84bf539d0261d0bdf533a90308e63 (
plain
)
1
2
3
Fail Inductive list' (A:Set) : Set := | nil' : list' A | cons' : A -> list' A -> list' (A*A).