mirror of https://github.com/nmvdw/HITs-Examples
19 lines
215 B
Plaintext
19 lines
215 B
Plaintext
|
{-# OPTIONS --without-K --rewriting #-}
|
||
|
|
||
|
open import HoTT
|
||
|
|
||
|
module Semantics where
|
||
|
|
||
|
data koe : Set where
|
||
|
a : koe
|
||
|
b : koe
|
||
|
|
||
|
postulate
|
||
|
kek : a ↦ b
|
||
|
{-# REWRITE kek #-}
|
||
|
|
||
|
|
||
|
Y : koe -> Set
|
||
|
Y a = Nat
|
||
|
Y b = Bool
|