Where.agda 331 B

12345678910111213141516171819202122
  1. module Where where
  2. -- all these examples should not termination check
  3. f : forall {A : Set} -> A
  4. f {A} = g
  5. where g : A
  6. g = f
  7. f1 : forall {A : Set} -> A -> A
  8. f1 {A} a = g a
  9. where g : A -> A
  10. g a = f1 a
  11. f2 : forall {A : Set} -> A -> A
  12. f2 {A} a = g a
  13. where g : A -> A
  14. g = f2