blob: ee2918c6e9b8b9e77e08d58802da64c997659f3d (
plain)
1
2
3
4
5
6
7
8
9
|
(* Test some uses of ? in introduction patterns *)
Inductive J : nat -> Prop :=
| K : forall p, J p -> (True /\ True) -> J (S p).
Lemma bug : forall n, J n -> J (S n).
Proof.
intros ? H.
induction H as [? ? [? ?]].
|