aboutsummaryrefslogtreecommitdiff
path: root/test-suite/output-coqtop/ShowProofDiffs.v
blob: 4251c52cb4582576a18ede173a901f66ea42b6b9 (plain)
1
2
3
4
5
6
(* coq-prog-args: ("-color" "on" "-diffs" "on") *)
Lemma x: forall(i : nat), exists(j k : nat), i = j /\ j = k /\ i = k.
Proof using.
  eexists.  Show Proof Diffs.
  eexists.  Show Proof Diffs.
  split.  Show Proof Diffs.