agda / agda

Agda is a dependently typed programming language / interactive theorem prover.

Home Page:https://wiki.portal.chalmers.se/agda/pmwiki.php

Geek Repo:Geek Repo

Github PK Tool:Github PK Tool

TBT: no function nor calls listed in termination error

andreasabel opened this issue · comments

{-# OPTIONS --no-syntax-based-termination #-}
{-# OPTIONS --type-based-termination #-}

module TypeBasedTermination.CopatternNonterminating where

open import Agda.Builtin.Equality

record Stream (A : Set) : Set where
  coinductive
  field
    head : A
    tail : Stream A
module S = Stream

illdefined : {A : Set}  Stream A
S.head illdefined = S.head illdefined
S.tail illdefined = S.tail illdefined
-- should not termination-check

The error is:

15,1-17,38
Termination checking failed for the following functions:
Problematic calls:

The error should be about function illdefined.

This issue has been reported before in