summaryrefslogtreecommitdiff
path: root/src/Cfe/Language/Indexed/Construct/Iterate.agda
diff options
context:
space:
mode:
authorChloe Brown <chloe.brown.00@outlook.com>2021-03-27 20:32:03 +0000
committerChloe Brown <chloe.brown.00@outlook.com>2021-03-27 20:32:03 +0000
commitadad5280af0d81a2f171df619e9c7169dcb43a02 (patch)
treec537696feea2aec1688d398bf5fd93e76f72c702 /src/Cfe/Language/Indexed/Construct/Iterate.agda
parentc67134fc5cb9e338cb397df029e5528d469771d4 (diff)
Introduce non-terminating proof of derivation existence.
Diffstat (limited to 'src/Cfe/Language/Indexed/Construct/Iterate.agda')
-rw-r--r--src/Cfe/Language/Indexed/Construct/Iterate.agda3
1 files changed, 3 insertions, 0 deletions
diff --git a/src/Cfe/Language/Indexed/Construct/Iterate.agda b/src/Cfe/Language/Indexed/Construct/Iterate.agda
index 1a37326..0ae9100 100644
--- a/src/Cfe/Language/Indexed/Construct/Iterate.agda
+++ b/src/Cfe/Language/Indexed/Construct/Iterate.agda
@@ -73,6 +73,9 @@ module _
where
module Iter = IndexedLanguage (Iterate f)
+ fⁿ≤⋃f : ∀ f n → (f ^ n) (Lift a ∅) ≤ ⋃ f
+ fⁿ≤⋃f f n = record { f = n ,_ }
+
⋃-cong : ∀ {f g} → (∀ {x y} → x ≈ y → f x ≈ g y) → ⋃ f ≈ ⋃ g
⋃-cong f≈g = record
{ f = λ { (n , l∈fn) → n , _≈_.f (f≈g⇒fn≈gn (L.setoid a) f≈g n (Lift a ∅)) l∈fn}