Skip to content

Commit

Permalink
[ fix #3525 ] Add test case (fix in 9bc651b)
Browse files Browse the repository at this point in the history
  • Loading branch information
jespercockx committed Apr 18, 2019
1 parent 4cdd3c3 commit 23a4e05
Showing 1 changed file with 22 additions and 0 deletions.
22 changes: 22 additions & 0 deletions test/Succeed/Issue3525.agda
@@ -0,0 +1,22 @@
{-# OPTIONS --prop --rewriting #-}

open import Agda.Builtin.Nat
open import Agda.Builtin.Equality

{-# BUILTIN REWRITE _≡_ #-}

data _≐_ {ℓ} {A : Set ℓ} (x : A) : A Propwhere
refl : x ≐ x

postulate
subst : {ℓ ℓ′} {A : Set ℓ} (P : A Set ℓ′)
(x y : A) x ≐ y P x P y
subst-rew : {ℓ ℓ′} {A : Set ℓ} (P : A Set ℓ′)
{x : A} (e : x ≐ x) (p : P x) subst P x x e p ≡ p
{-# REWRITE subst-rew #-}

data Box (A : Prop) : Set where
box : A -> Box A

foo : (A : Prop)(x y : A)(P : Box A Set)(p : P (box x)) subst P (box x) (box y) refl p ≐ p
foo A x y P p = refl -- refl does not type check

0 comments on commit 23a4e05

Please sign in to comment.