aboutsummaryrefslogtreecommitdiffhomepage
path: root/etc/coq/highlighterror.v
blob: 26ff1dea824b1f0ef46cd453e297af1b01fb048f (plain)
1
2
3
4
5
6
7
8
9
(* Test of error highlighting

The error should highlight the last γ₁₂ variable occurrence, the whole
of it, and only it (not the final dot nor the preceding space).
*)

Require Import Utf8.

Lemma α₁: ∀ x:nat, ∀ γ₁₂: bool, x = γ₁₂.