blob: cf035edf7918996b6da97debfacf9296b20e2589 (
plain)
1
2
3
4
5
|
(* Check that the nested inductive types positivity check avoids recursively
non uniform parameters (at least if these parameters break positivity) *)
Inductive t (A:Type) : Type := c : t (A -> A) -> t A.
Inductive u : Type := d : u | e : t u -> u.
|