summaryrefslogtreecommitdiff
path: root/test-suite/vio/numeral.v
blob: f28355bb29d0520a8b768266175803b9b7a24515 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
Lemma foo : True.
Proof.
Check 0 : nat.
Check 0 : nat.
exact I.
Qed.

Lemma bar : True.
Proof.
pose (0 : nat).
exact I.
Qed.

Require Import Coq.Strings.Ascii.
Open Scope char_scope.

Lemma baz : True.
Proof.
pose "s".
exact I.
Qed.