aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/ex/mult2.v
blob: 997beefd42114c694500fafab814559e6a51c4ba (plain)
1
2
3
4
5
6
7


Require Import mult1.

Definition bar:bool := if le_lt_dec foo 0 then true else false.