-
Notifications
You must be signed in to change notification settings - Fork 143
Commit
This commit does not belong to any branch on this repository, and may belong to a fork outside of the repository.
* (wip) for Zariski coverage on CommRing (with Max Zeuner) * pullback stability * only zero case left * finish zero case * def standard affine open * finish standard affine opens * towards opens of affines * discussion * little progress * towards separatedness * separatedness * locality * towards aff cover * give up * finish * cleanup * use inline ring solver * fix * more fixes * fix accidentally public module manually cherry-picked from 93d52b5 * avoid code duplication manually cherry-picked from 73cc74a * improve comment manually cherry-picked from 2c4d6d1 * slightly improve comment * named module StandardOpens manually cherry-picked from d41b178 * indent by two spaces * less whitespace * avoid duplication in PosetDownset * fix copy-paste errors in comment * cleanup JoinMap * don't re-prove monoid lemmas * slightly clearer comment * polish module definition * cleanup imports * cleanup some more * forgotten while renaming ZarMap -> Support * upstream 1 lemmas * meet map --------- Co-authored-by: Matthias Hutzler <[email protected]>
- Loading branch information
1 parent
fc4ef6a
commit 8dc7788
Showing
13 changed files
with
783 additions
and
104 deletions.
There are no files selected for viewing
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
Original file line number | Diff line number | Diff line change |
---|---|---|
@@ -0,0 +1,70 @@ | ||
{-# OPTIONS --safe #-} | ||
module Cubical.Algebra.DistLattice.Downset where | ||
|
||
open import Cubical.Foundations.Prelude | ||
open import Cubical.Foundations.HLevels | ||
open import Cubical.Foundations.Isomorphism | ||
open import Cubical.Foundations.Powerset | ||
|
||
open import Cubical.Data.Sigma | ||
|
||
open import Cubical.Algebra.Semigroup | ||
open import Cubical.Algebra.Monoid | ||
open import Cubical.Algebra.CommMonoid | ||
open import Cubical.Algebra.Semilattice | ||
open import Cubical.Algebra.Lattice | ||
open import Cubical.Algebra.DistLattice.Base | ||
|
||
open import Cubical.Relation.Binary.Order.Poset | ||
|
||
open Iso | ||
|
||
private | ||
variable | ||
ℓ ℓ' : Level | ||
|
||
module DistLatticeDownset (L' : DistLattice ℓ) where | ||
|
||
open DistLatticeStr ⦃...⦄ | ||
open PosetStr ⦃...⦄ hiding (is-set) | ||
open JoinSemilattice (Lattice→JoinSemilattice (DistLattice→Lattice L')) | ||
open MeetSemilattice (Lattice→MeetSemilattice (DistLattice→Lattice L')) hiding (_≤_ ; IndPoset) | ||
open LatticeTheory (DistLattice→Lattice L') | ||
open Order (DistLattice→Lattice L') | ||
open IsLatticeHom | ||
|
||
-- importing other downset related stuff | ||
open PosetDownset IndPoset public | ||
|
||
private | ||
L = L' .fst | ||
LPoset = IndPoset | ||
instance | ||
_ = L' .snd | ||
_ = LPoset .snd | ||
|
||
↓ᴰᴸ : L → DistLattice ℓ | ||
fst (↓ᴰᴸ u) = ↓ u | ||
DistLatticeStr.0l (snd (↓ᴰᴸ u)) = 0l , ∨lLid u | ||
DistLatticeStr.1l (snd (↓ᴰᴸ u)) = u , is-refl u | ||
DistLatticeStr._∨l_ (snd (↓ᴰᴸ u)) (v , v≤u) (w , w≤u) = | ||
v ∨l w , ∨lIsMax _ _ _ v≤u w≤u | ||
DistLatticeStr._∧l_ (snd (↓ᴰᴸ u)) (v , v≤u) (w , _) = | ||
v ∧l w , is-trans _ _ _ (≤m→≤j _ _ (∧≤RCancel _ _)) v≤u | ||
DistLatticeStr.isDistLattice (snd (↓ᴰᴸ u)) = makeIsDistLattice∧lOver∨l | ||
(isSetΣSndProp is-set λ _ → is-prop-valued _ _) | ||
(λ _ _ _ → Σ≡Prop (λ _ → is-prop-valued _ _) (∨lAssoc _ _ _)) | ||
(λ _ → Σ≡Prop (λ _ → is-prop-valued _ _) (∨lRid _)) | ||
(λ _ _ → Σ≡Prop (λ _ → is-prop-valued _ _) (∨lComm _ _)) | ||
(λ _ _ _ → Σ≡Prop (λ _ → is-prop-valued _ _) (∧lAssoc _ _ _)) | ||
(λ (_ , v≤u) → Σ≡Prop (λ _ → is-prop-valued _ _) (≤j→≤m _ _ v≤u)) | ||
(λ _ _ → Σ≡Prop (λ _ → is-prop-valued _ _) (∧lComm _ _)) | ||
(λ _ _ → Σ≡Prop (λ _ → is-prop-valued _ _) (∧lAbsorb∨l _ _)) | ||
(λ _ _ _ → Σ≡Prop (λ _ → is-prop-valued _ _) (∧lLdist∨l _ _ _)) | ||
|
||
toDownHom : (u : L) → DistLatticeHom L' (↓ᴰᴸ u) | ||
fst (toDownHom u) w = (u ∧l w) , ≤m→≤j _ _ (∧≤RCancel _ _) | ||
pres0 (snd (toDownHom u)) = Σ≡Prop (λ _ → is-prop-valued _ _) (0lRightAnnihilates∧l _) | ||
pres1 (snd (toDownHom u)) = Σ≡Prop (λ _ → is-prop-valued _ _) (∧lRid _) | ||
pres∨l (snd (toDownHom u)) v w = Σ≡Prop (λ _ → is-prop-valued _ _) (∧lLdist∨l _ _ _) | ||
pres∧l (snd (toDownHom u)) v w = Σ≡Prop (λ _ → is-prop-valued _ _) (∧lLdist∧l u v w) |
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
This file contains bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
Oops, something went wrong.