Skip to content

Latest commit

 

History

History
347 lines (291 loc) · 11.5 KB

CHANGELOG.md

File metadata and controls

347 lines (291 loc) · 11.5 KB

Version 2.2-dev

The library has been tested using Agda 2.7.0.

Highlights

Bug-fixes

  • Removed unnecessary parameter #-trans : Transitive _#_ from Relation.Binary.Reasoning.Base.Apartness.

Non-backwards compatible changes

Minor improvements

Deprecated modules

Deprecated names

  • In Algebra.Properties.CommutativeMagma.Divisibility:

    ∣-factors    ↦  x|xy∧y|xy
    ∣-factors-≈  ↦  xy≈z⇒x|z∧y|z
  • In Algebra.Properties.Magma.Divisibility:

    ∣-respˡ   ↦  ∣-respˡ-≈
    ∣-respʳ   ↦  ∣-respʳ-≈
    ∣-resp    ↦  ∣-resp-≈

* In `Algebra.Solver.CommutativeMonoid`:
 ```agda
 normalise-correct  ↦  Algebra.Solver.CommutativeMonoid.Normal.correct
 sg                 ↦  Algebra.Solver.CommutativeMonoid.Normal.singleton
 sg-correct         ↦  Algebra.Solver.CommutativeMonoid.Normal.singleton-correct
  • In Algebra.Solver.IdempotentCommutativeMonoid:

    flip12             ↦  Algebra.Properties.CommutativeSemigroup.xy∙z≈y∙xz
    distr              ↦  Algebra.Properties.IdempotentCommutativeMonoid.∙-distrˡ-∙
    normalise-correct  ↦  Algebra.Solver.IdempotentCommutativeMonoid.Normal.correct
    sg                 ↦  Algebra.Solver.IdempotentCommutativeMonoid.Normal.singleton
    sg-correct         ↦  Algebra.Solver.IdempotentCommutativeMonoid.Normal.singleton-correct
  • In Algebra.Solver.Monoid:

    homomorphic        ↦  Algebra.Solver.Monoid.Normal.comp-correct
    normalise-correct  ↦  Algebra.Solver.Monoid.Normal.correct
  • In Data.List.Relation.Binary.Permutation.Setoid.Properties:

    split  ↦  ↭-split

    with a more informative type (see below).

    
    
  • In Data.Vec.Properties:

    ++-assoc _      ↦  ++-assoc-eqFree
    ++-identityʳ _  ↦  ++-identityʳ-eqFree
    unfold-∷ʳ _     ↦  unfold-∷ʳ-eqFree
    ++-∷ʳ _         ↦  ++-∷ʳ-eqFree
    ∷ʳ-++ _         ↦  ∷ʳ-++-eqFree
    reverse-++ _    ↦  reverse-++-eqFree
    ∷-ʳ++ _         ↦  ∷-ʳ++-eqFree
    ++-ʳ++ _        ↦  ++-ʳ++-eqFree
    ʳ++-ʳ++ _       ↦  ʳ++-ʳ++-eqFree

New modules

  • Properties of IdempotentCommutativeMonoids refactored out from Algebra.Solver.IdempotentCommutativeMonoid:

    Algebra.Properties.IdempotentCommutativeMonoid
  • Refactoring of the Algebra.Solver.*Monoid implementations, via a single Solver module API based on the existing Expr, and a common Normal-form API:

    Algebra.Solver.CommutativeMonoid.Normal
    Algebra.Solver.IdempotentCommutativeMonoid.Normal
    Algebra.Solver.Monoid.Expression
    Algebra.Solver.Monoid.Normal
    Algebra.Solver.Monoid.Solver

    NB Imports of the existing proof procedures solve and prove etc. should still be via the top-level interfaces in Algebra.Solver.*Monoid.

  • Refactored out from Data.List.Relation.Unary.All.Properties in order to break a dependency cycle with Data.List.Membership.Setoid.Properties:

    Data.List.Relation.Unary.All.Properties.Core
  • Data.List.Relation.Binary.Disjoint.Propositional.Properties: Propositional counterpart to Data.List.Relation.Binary.Disjoint.Setoid.Properties

  • Data.List.Relation.Binary.Permutation.Propositional.Properties.WithK

Additions to existing modules

  • Properties of non-divisibility in Algebra.Properties.Magma.Divisibility:

    ∤-respˡ-≈ : _∤_ Respectsˡ _≈_
    ∤-respʳ-≈ : _∤_ Respectsʳ _≈_
    ∤-resp-≈  : _∤_ Respects₂ _≈_
    ∤∤-sym    : Symmetric _∤∤_
    ∤∤-respˡ-≈ : _∤∤_ Respectsˡ _≈_
    ∤∤-respʳ-≈ : _∤∤_ Respectsʳ _≈_
    ∤∤-resp-≈  : _∤∤_ Respects₂ _≈_
  • In Algebra.Solver.Ring

    Env : Set _
    Env = Vec Carrier

* In `Data.List.Membership.Setoid.Properties`:
 ```agda
 ∉⇒All[≉]       : x ∉ xs → All (x ≉_) xs
 All[≉]⇒∉       : All (x ≉_) xs → x ∉ xs
 Any-∈-swap     : Any (_∈ ys) xs → Any (_∈ xs) ys
 All-∉-swap     : All (_∉ ys) xs → All (_∉ xs) ys
 ∈-map∘filter⁻  : y ∈₂ map f (filter P? xs) → ∃[ x ] x ∈₁ xs × y ≈₂ f x × P x
 ∈-map∘filter⁺  : f Preserves _≈₁_ ⟶ _≈₂_ →
                  ∃[ x ] x ∈₁ xs × y ≈₂ f x × P x →
                  y ∈₂ map f (filter P? xs)
 ∈-concatMap⁺   : Any ((y ∈_) ∘ f) xs → y ∈ concatMap f xs
 ∈-concatMap⁻   : y ∈ concatMap f xs → Any ((y ∈_) ∘ f) xs
 ∉[]            : x ∉ []
 deduplicate-∈⇔ : _≈_ Respectsʳ (flip R) → z ∈ xs ⇔ z ∈ deduplicate R? xs
  • In Data.List.Membership.Propositional.Properties:

    ∈-AllPairs₂    : AllPairs R xs  x ∈ xs  y ∈ xs  x ≡ y ⊎ R x y ⊎ R y x
    ∈-map∘filter⁻  : y ∈ map f (filter P? xs)  (∃[ x ] x ∈ xs × y ≡ f x × P x)
    ∈-map∘filter⁺  : (∃[ x ] x ∈ xs × y ≡ f x × P x)  y ∈ map f (filter P? xs)
    ∈-concatMap⁺   : Any ((y ∈_) ∘ f) xs  y ∈ concatMap f xs
    ∈-concatMap⁻   : y ∈ concatMap f xs  Any ((y ∈_) ∘ f) xs
    ++-∈⇔          : v ∈ xs ++ ys ⇔ (v ∈ xs ⊎ v ∈ ys)
    []∉map∷        : [] ∉ map (x ∷_) xss
    map∷⁻          : xs ∈ map (y ∷_) xss  ∃[ ys ] ys ∈ xss × xs ≡ y ∷ ys
    map∷-decomp∈   : (x ∷ xs) ∈ map (y ∷_) xss  x ≡ y × xs ∈ xss
    ∈-map∷⁻        : xs ∈ map (x ∷_) xss  x ∈ xs
    ∉[]            : x ∉ []
    deduplicate-∈⇔ : z ∈ xs ⇔ z ∈ deduplicate _≈?_ xs
  • In Data.List.Membership.Propositional.Properties.WithK:

    unique∧set⇒bag : Unique xs  Unique ys  xs ∼[ set ] ys  xs ∼[ bag ] ys
  • In Data.List.Properties:

    product≢0    : All NonZero ns  NonZero (product ns)
    ∈⇒≤product   : All NonZero ns  n ∈ ns  n ≤ product ns
    concatMap-++ : concatMap f (xs ++ ys) ≡ concatMap f xs ++ concatMap f ys
  • In Data.List.Relation.Unary.Any.Properties:

    concatMap⁺ : Any (Any P ∘ f) xs  Any P (concatMap f xs)
    concatMap⁻ : Any P (concatMap f xs)  Any (Any P ∘ f) xs
  • In Data.List.Relation.Unary.Unique.Setoid.Properties:

    Unique[x∷xs]⇒x∉xs : Unique S (x ∷ xs)  x ∉ xs
  • In Data.List.Relation.Unary.Unique.Propositional.Properties:

    Unique[x∷xs]⇒x∉xs : Unique (x ∷ xs)  x ∉ xs
  • In Data.List.Relation.Binary.Equality.Setoid:

    ++⁺ʳ :  xs  ys ≋ zs  xs ++ ys ≋ xs ++ zs
    ++⁺ˡ :  zs  ws ≋ xs  ws ++ zs ≋ xs ++ zs
  • In Data.List.Relation.Binary.Permutation.Homogeneous:

    steps : Permutation R xs ys 
  • In Data.List.Relation.Binary.Permutation.Propositional: constructor aliases

    ↭-refl  : Reflexive _↭_
    ↭-prep  :  x  xs ↭ ys  x ∷ xs ↭ x ∷ ys
    ↭-swap  :  x y  xs ↭ ys  x ∷ y ∷ xs ↭ y ∷ x ∷ ys

    and properties

    ↭-reflexive-≋ : _≋_ ⇒ _↭_
    ↭⇒↭ₛ          : _↭_  ⇒ _↭ₛ_
    ↭ₛ⇒↭          : _↭ₛ_ ⇒ _↭_

    where _↭ₛ_ is the Setoid (setoid _) instance of Permutation

  • In Data.List.Relation.Binary.Permutation.Propositional.Properties:

    Any-resp-[σ∘σ⁻¹] :: xs ↭ ys) (iy : Any P ys) 
                       Any-resp-↭ (trans (↭-sym σ) σ) iy ≡ iy
    ∈-resp-[σ∘σ⁻¹]   :: xs ↭ ys) (iy : y ∈ ys) 
                       ∈-resp-↭ (trans (↭-sym σ) σ) iy ≡ iy
    product-↭        : product Preserves _↭_ ⟶ _≡_
  • In Data.List.Relation.Binary.Permutation.Setoid:

    ↭-reflexive-≋ : _≋_  ⇒ _↭_
    ↭-transˡ-≋    : LeftTrans _≋_ _↭_
    ↭-transʳ-≋    : RightTrans _↭_ _≋_
    ↭-trans′      : Transitive _↭_
  • In Data.List.Relation.Binary.Permutation.Setoid.Properties:

    ↭-split : xs ↭ (as ++ [ v ] ++ bs) 
              ∃₂ λ ps qs  xs ≋ (ps ++ [ v ] ++ qs) × (ps ++ qs) ↭ (as ++ bs)
    drop-∷  : x ∷ xs ↭ x ∷ ys  xs ↭ ys
  • In Data.List.Relation.Binary.Pointwise:

    ++⁺ʳ : Reflexive R   xs  (xs ++_) Preserves (Pointwise R) ⟶ (Pointwise R)
    ++⁺ˡ : Reflexive R   zs  (_++ zs) Preserves (Pointwise R) ⟶ (Pointwise R)
  • In Data.List.Relation.Unary.All:

    search : Decidable P   xs  All (∁ P) xs ⊎ Any P xs
    
  • In Data.List.Relation.Binary.Subset.Setoid.Properties:

    ∷⊈[]   : x ∷ xs ⊈ []
    ⊆∷⇒∈∨⊆ : xs ⊆ y ∷ ys  y ∈ xs ⊎ xs ⊆ ys
    ⊆∷∧∉⇒⊆ : xs ⊆ y ∷ ys  y ∉ xs  xs ⊆ ys
  • In Data.List.Relation.Binary.Subset.Propositional.Properties:

    ∷⊈[]   : x ∷ xs ⊈ []
    ⊆∷⇒∈∨⊆ : xs ⊆ y ∷ ys  y ∈ xs ⊎ xs ⊆ ys
    ⊆∷∧∉⇒⊆ : xs ⊆ y ∷ ys  y ∉ xs  xs ⊆ ys
  • In Data.List.Relation.Binary.Subset.Propositional.Properties:

    concatMap⁺ : xs ⊆ ys  concatMap f xs ⊆ concatMap f ys
  • In Data.List.Relation.Binary.Sublist.Heterogeneous.Properties:

    Sublist-[]-universal : Universal (Sublist R [])
  • In Data.List.Relation.Binary.Sublist.Setoid.Properties:

    []⊆-universal : Universal ([] ⊆_)
  • In Data.List.Relation.Binary.Disjoint.Setoid.Properties:

    deduplicate⁺ : Disjoint S xs ys  Disjoint S (deduplicate _≟_ xs) (deduplicate _≟_ ys)
  • In Data.List.Relation.Binary.Disjoint.Propositional.Properties:

    deduplicate⁺ : Disjoint xs ys  Disjoint (deduplicate _≟_ xs) (deduplicate _≟_ ys)
  • In Data.List.Relation.Binary.Permutation.Propositional.Properties.WithK:

    dedup-++-↭ : Disjoint xs ys 
                 deduplicate _≟_ (xs ++ ys) ↭ deduplicate _≟_ xs ++ deduplicate _≟_ ys
  • In Data.Maybe.Properties:

    maybe′-∘ :  f g  f ∘ (maybe′ g b) ≗ maybe′ (f ∘ g) (f b)
  • New lemmas in Data.Nat.Properties:

    m≤n⇒m≤n*o :  o .{{_ : NonZero o}}  m ≤ n  m ≤ n * o
    m≤n⇒m≤o*n :  o .{{_ : NonZero o}}  m ≤ n  m ≤ o * n

    adjunction between suc and pred

    suc[m]≤n⇒m≤pred[n] : suc m ≤ n  m ≤ pred n
    m≤pred[n]⇒suc[m]≤n : .{{NonZero n}}  m ≤ pred n  suc m ≤ n
  • New lemma in Data.Vec.Properties:

    map-concat : map f (concat xss) ≡ concat (map (map f) xss)
  • In Data.Vec.Relation.Binary.Equality.DecPropositional:

    _≡?_ : DecidableEquality (Vec A n)
  • In Relation.Binary.Construct.Interior.Symmetric:

    decidable         : Decidable R  Decidable (SymInterior R)

    and for Reflexive and Transitive relations R:

    isDecEquivalence  : Decidable R  IsDecEquivalence (SymInterior R)
    isDecPartialOrder : Decidable R  IsDecPartialOrder (SymInterior R) R
    decPoset          : Decidable R  DecPoset _ _ _
  • In Relation.Nullary.Decidable:

    does-⇔  : A ⇔ B  (a? : Dec A)  (b? : Dec B)  does a? ≡ does b?
    does-≡  : (a? b? : Dec A)  does a? ≡ does b?
  • In Relation.Unary.Properties:

    map    : P ≐ Q  Decidable P  Decidable Q
    does-≐ : P ≐ Q  (P? : Decidable P)  (Q? : Decidable Q)  does ∘ P? ≗ does ∘ Q?
    does-≡ : (P? P?′ : Decidable P)  does ∘ P? ≗ does ∘ P?′