HITs-Examples/Agda-HITs/Imperative/Semantics.agda

19 lines
215 B
Plaintext
Raw Normal View History

2017-05-22 16:46:58 +02:00
{-# 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