summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/7068.v
blob: 9fadb195bf2e8f04e4c7aee871d75130402eed15 (plain)
1
2
3
4
5
6
(* These tests are only about a subset of #7068 *)
(* The original issue is still open *)

Inductive foo : let T := Type in T := .
Definition bob1 := Eval vm_compute in foo_rect.
Definition bob2 := Eval native_compute in foo_rect.