diff automaton-in-agda/src/automaton-ex.agda @ 405:af8f630b7e60

...
author Shinji KONO <kono@ie.u-ryukyu.ac.jp>
date Sun, 24 Sep 2023 18:02:04 +0900
parents 407684f806e4
children
line wrap: on
line diff
--- a/automaton-in-agda/src/automaton-ex.agda	Sun Sep 24 13:20:31 2023 +0900
+++ b/automaton-in-agda/src/automaton-ex.agda	Sun Sep 24 18:02:04 2023 +0900
@@ -1,4 +1,5 @@
-{-# OPTIONS --allow-unsolved-metas #-}
+{-# OPTIONS --cubical-compatible --safe #-}
+
 module automaton-ex where
 
 open import Data.Nat
@@ -102,6 +103,24 @@
 test11 : count-chars (  i1  ∷ i1  ∷ i0  ∷ []  ) i0 ≡ 1
 test11 = refl
 
+_≥b_ : ( x y : ℕ) → Bool
+x ≥b y with <-cmp x y
+... | tri< a ¬b ¬c = false
+... | tri≈ ¬a b ¬c = true
+... | tri> ¬a ¬b c = true
+
+_>b_ : ( x y : ℕ) → Bool
+x >b y with <-cmp x y
+... | tri< a ¬b ¬c = false
+... | tri≈ ¬a b ¬c = false
+... | tri> ¬a ¬b c = true
+
+_≤b_ : ( x y : ℕ) → Bool
+x ≤b y  = y ≥b x
+
+_<b_ : ( x y : ℕ) → Bool
+x <b y  = y >b x
+
 ex1_4a : (x : List In2) → Bool
 ex1_4a x =  ( count-chars x i0 ≥b 3 ) /\ ( count-chars x i1 ≥b 2 )
 
@@ -138,5 +157,5 @@
 am14a-tr' a00 i0 = a10
 am14a-tr' _ _ = a10
 
-am14a'  :  Automaton  am14s  In2
-am14a'  =  record {  δ = am14a-tr' ; aend = λ x → {!!} }
+-- am14a'  :  Automaton  am14s  In2
+-- am14a'  =  record {  δ = am14a-tr' ; aend = λ x → {!!} }