Ticket #375: pg_bug3.v

File pg_bug3.v, 131 bytes (added by megacz, 14 years ago)
Line 
1Require Import Coq.Init.Logic.
2
3
4Notation "C 'ᵒ᎟'" := (fun x => C) (at level 20).
5
6Definition crash_the_rooster f := f ᵒ᎟.