diff automaton-in-agda/src/finiteSet.agda @ 403:c298981108c1

fix for std-lib 2.0
author Shinji KONO <kono@ie.u-ryukyu.ac.jp>
date Sun, 24 Sep 2023 11:32:01 +0900
parents 91781b7c65a8
children b85402051cdb
line wrap: on
line diff
--- a/automaton-in-agda/src/finiteSet.agda	Thu Aug 10 09:59:47 2023 +0900
+++ b/automaton-in-agda/src/finiteSet.agda	Sun Sep 24 11:32:01 2023 +0900
@@ -1,4 +1,4 @@
-{-# OPTIONS --allow-unsolved-metas #-}
+{-# OPTIONS --cubical-compatible --safe #-}
 module finiteSet  where
 
 open import Data.Nat hiding ( _≟_ )
@@ -12,7 +12,7 @@
 open import nat
 open import Data.Nat.Properties hiding ( _≟_ )
 
-open import Relation.Binary.HeterogeneousEquality as HE using (_≅_ ) 
+-- open import Relation.Binary.HeterogeneousEquality as HE using (_≅_ ) 
 
 record FiniteSet ( Q : Set ) : Set  where
      field