1
0
mirror of https://github.com/nmvdw/HITs-Examples synced 2025-12-21 17:13:50 +01:00
Files
HITs-Examples/Agda-HITs/Imperative/Semantics.agda
2017-05-22 16:46:58 +02:00

19 lines
215 B
Agda

{-# 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