aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/ex/test-cases/stale-load-path/c/c.v
blob: f05f65a16b77a0abfed4ded16b0765ad2d55f018 (plain)
1
2
3
4
5
6
7
8
9
(* This file depends on Coq.Arith.Le from the standard library. *)

Require Le.

(* The next print should work. *)
Print Le.le_refl.

(* The next print should not work. *)
Print Le.a.