comparison a02/agda/logic.agda @ 406:a60132983557

...
author Shinji KONO <kono@ie.u-ryukyu.ac.jp>
date Wed, 08 Nov 2023 21:35:54 +0900
parents 407684f806e4
children
comparison
equal deleted inserted replaced
405:af8f630b7e60 406:a60132983557
1 {-# OPTIONS --cubical-compatible --safe #-}
2
1 module logic where 3 module logic where
2 4
3 open import Level 5 open import Level
4 open import Relation.Nullary 6 open import Relation.Nullary
5 open import Relation.Binary hiding (_⇔_) 7 open import Relation.Binary hiding (_⇔_)