You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
[fixes#1711] Refactoring Data.Nat.Divisibility and Data.Nat.DivMod (#2182)
* added new definitions to `_∣_`
* `CHANGELOG`
* don't declare `quotient≢0` as an `instance`
* replace use of `subst` with one of `trans`
* what's sauce for the goose...
* switch to a `rewrite`-based solution...
* tightened `import`s
* simplified dependenciess
* simplified dependencies; `CHANGELOG`
* removed `module` abstractions
* delegated proof of `quotient≢0` to `Data.Nat.Properties`
* removed redundant property
* cosmetic review changes; others to follow
* better proof of `quotient>1`
* `where` clause layout
* leaving in the flipped equality; moved everything else
* new lemmas moved from `Core`; knock-on consequences; lots of tidying up
* tidying up; `CHANGELOG`
* cosmetic tweaks
* reverted to simple version
* problems with exporting `quotient`
* added last lemma: defining equation for `_/_`
* improved `CHANGELOG`
* revert: simplified imports
* improved `CHANGELOG`
* endpoint of simplifying the proof of `*-pres-∣`
* simplified the proof of `n/m≡quotient`
* simplified the proof of `∣m+n∣m⇒∣n`
* simplified the proof of `∣m∸n∣n⇒∣m`
* simplified `import`s
* simplified a lot of proofs, esp. wrt `divides-refl` and `NonZero` reasoning
* simplified more proofs, esp. wrt `divides-refl` reasoning
* simplified `import`s
* moved `equalityᵒ` proof out of `Core`
* `CHANGELOG`
* temporary fix: further `NonZero` refactoring advised!
* regularised use of instance brackets
* further instance simplification
* further streamlining
* tidied up `CHANGELOG`
* simplified `NonZero` pattern matching
* regularised use of instance brackets
* simplified proof of `/-*-interchange`
* simplified proof of `/-*-interchange`
* ... permitting the migration of `*-pres-∣` to `Data.Nat.Divisibility`
* tweaked proof of `/-*-interchange`
* narrowed `import`s
* simplified proof; renamed new proofs
* Capitalisation
* streamlined `import`s; streamlined proof of decidability
* spurious duplication after merge
* missing symbol import
* replaced one use of `1 < m` with `{{NonTrivial m}}`
* fixed `CHANGELOG`
* removed use of identifier `k`
* refactoring: more use of `NonTrivial` instances
* knock-on consequences: simplified function
* two new lemmas
* refactoring: use of `connex` in proofs
* new lemmas about `pred`
* new lemmas about monus
* refactoring: use of the new properties, simplifying pattern analysis
* whitespace
* questionable? revision after comments on #2221
* silly argument name typo; remove parens
* tidied up imports of `Relation.Nullary`
* removed spurious `instance`
* localised appeals to `Reasoning`
* further use of `variable`s
* tidied up `record` name in comment
* cosmetic
* reconciled implicit/explicit arguments in various monus lemmas
* fixed knock-on change re monus; reverted change to `m/n<m`
* reverted change to `m/n≢0⇒n≤m`
* reverted breaking changes involving `NonZero` inference
* revised `CHANGELOG`
* restored deleted proof
* fix whitespace
* renaming: `DivMod.nonZeroDivisor`
* localised use of `≤-Reasoning`
* reverted export; removed anonymous module
* revert commit re `yes/no`
* renamed flipped equality
* tweaked comment
* added alias for `equality`
0 commit comments