blob: b586cba50f179c9358689c0bf69f4491ffece2ff (
plain)
1
2
3
4
5
6
7
8
9
|
(* [Unset Bracketing Last Introduction Pattern] was not working *)
Unset Bracketing Last Introduction Pattern.
Goal forall T (x y : T * T), fst x = fst y /\ snd x = snd y -> x = y.
do 10 ((intros [] || intro); simpl); reflexivity.
Qed.
|