diff options
author | Chloe Brown <chloe.brown.00@outlook.com> | 2021-03-05 00:00:04 +0000 |
---|---|---|
committer | Chloe Brown <chloe.brown.00@outlook.com> | 2021-03-05 00:04:46 +0000 |
commit | 5302e4a27a64cb2a97120517df4b6998da7b3168 (patch) | |
tree | ebe15b37e27e8ec7e4920200e15a40ae586bedbc /src/Cfe/Language/Properties.agda | |
parent | ff3600687249a19ae63353f7791b137094f5a5a1 (diff) |
Complete proofs up to Proposition 3.2 (excluding unrolling)
Diffstat (limited to 'src/Cfe/Language/Properties.agda')
-rw-r--r-- | src/Cfe/Language/Properties.agda | 41 |
1 files changed, 0 insertions, 41 deletions
diff --git a/src/Cfe/Language/Properties.agda b/src/Cfe/Language/Properties.agda deleted file mode 100644 index 52d4644..0000000 --- a/src/Cfe/Language/Properties.agda +++ /dev/null @@ -1,41 +0,0 @@ -{-# OPTIONS --without-K --safe #-} - -open import Relation.Binary - -module Cfe.Language.Properties - {c ℓ} {setoid : Setoid c ℓ} - where - -open Setoid setoid renaming (Carrier to A) -open import Cfe.Language setoid -open Language - -open import Data.List -open import Data.List.Relation.Binary.Equality.Setoid setoid -open import Function -open import Level -open import Relation.Binary.Construct.InducedPoset - -_≤′_ : ∀ {a aℓ} → Rel (Language a aℓ) (c ⊔ a) -_≤′_ = _≤_ - ------------------------------------------------------------------------- --- Properties of _≤_ - -≤-refl : ∀ {a aℓ} → Reflexive (_≤′_ {a} {aℓ}) -≤-refl = id - -≤-trans : ∀ {a b c aℓ bℓ cℓ} → Trans (_≤_ {a} {aℓ}) (_≤_ {b} {bℓ} {c} {cℓ}) _≤_ -≤-trans A≤B B≤C = B≤C ∘ A≤B - -≤-poset : ∀ {a aℓ} → Poset (c ⊔ ℓ ⊔ suc (a ⊔ aℓ)) (c ⊔ a) (c ⊔ a) -≤-poset {a} {aℓ} = InducedPoset (_≤′_ {a} {aℓ}) id (λ i≤j j≤k → j≤k ∘ i≤j) - --- ------------------------------------------------------------------------ --- -- Properties of _∪_ - --- ∪-cong-≤ : Congruent₂ _≤_ _∪_ --- ∪-cong-≤ A≤B C≤D = map A≤B C≤D - --- ∪-cong : Congruent₂ _≈_ _∪_ --- ∪-cong {A} {B} {C} {D} = ≤-cong₂→≈-cong₂ {_∪_} (λ A≤B C≤D → map A≤B C≤D) {A} {B} {C} {D} |