aboutsummaryrefslogtreecommitdiff
path: root/test-suite/stm/arg_filter_1.v
blob: ed87d674055eed59216f56bcd7c023746668414c (plain)
1
2
3
4
(* coq-prog-args: ("-async-proofs-tac-j" "1") *)

Lemma foo (A B : Prop) n : n + 0 = n /\ (A -> B -> A).
Proof. split. par: now auto. Qed.