summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/4764.v
blob: e545cc1b71d2e7efb521532ef5e1bc7a445adb6e (plain)
1
2
3
4
5
Notation prop_fun x y := (fun (x : Prop) => y).
Definition foo := fun (p : Prop) => p.
Definition bar := fun (_ : Prop) => O.
Print foo.
Print bar.