Skip to content

Commit

Permalink
[ re agda#5610 ] Add proof of false to (failing) test case
Browse files Browse the repository at this point in the history
  • Loading branch information
jespercockx committed Oct 25, 2021
1 parent 5435821 commit 77e7ac3
Showing 1 changed file with 20 additions and 0 deletions.
20 changes: 20 additions & 0 deletions test/Fail/BuiltinFlatBadType.agda
Original file line number Diff line number Diff line change
Expand Up @@ -8,3 +8,23 @@ postulate
{-# BUILTIN INFINITY ∞ #-}
{-# BUILTIN SHARP ♯_ #-}
{-# BUILTIN FLAT ♭ #-}

-- Issue #5610: with these bad types for sharp and flat, we can prove
-- false. The reason is that ∞ is assumed to be strictly-positive in
-- the positivity checker (even guarding positive). So making ∞ A
-- isomorphic to A → ⊥ will be contradictory to this assumption.

data D : Set where
wrap : ∞ D D

lam : (D ⊥) D
lam f = wrap (♯ f)

app : D D
app (wrap g) d = ♭ g d

delta : D
delta = lam (λ x app x x)

omega :
omega = app delta delta

0 comments on commit 77e7ac3

Please sign in to comment.