summaryrefslogtreecommitdiff
path: root/test-suite/success/Case22.v
blob: 4eb2dbe9f52a6e26d02a7aa5a98fa2eeeeb087da (plain)
1
2
3
4
5
6
7
(* Check typing in the presence of let-in in inductive arity *)

Inductive I : let a := 1 in a=a -> let b := 2 in Type := C : I (eq_refl).
Lemma a : forall x:I eq_refl, match x in I a b c return b = b with C => eq_refl end = eq_refl.
intro.
match goal with |- ?c => let x := eval cbv in c in change x end.
Abort.