summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/shouldsucceed/1935.v
blob: d5837619850e569dd9fb20dee9c16d1a594a7f16 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
Definition f  (n:nat) := n = n.

Lemma f_refl : forall n , f n.
intros. reflexivity.
Qed.

Definition f'  (x:nat) (n:nat) := n = n.

Lemma f_refl' : forall n , f' n n.
Proof.
 intros. reflexivity.
Qed.

Require Import ZArith.

Definition f'' (a:bool) := if a then eq (A:= Z) else Z.lt.

Lemma f_refl'' : forall n , f'' true n n.
Proof.
 intro. reflexivity.
Qed.