Skip to content

Commit

Permalink
a bit more on prime ideals
Browse files Browse the repository at this point in the history
  • Loading branch information
samvang committed May 16, 2024
1 parent 30d0ce4 commit 1eea3c5
Showing 1 changed file with 31 additions and 0 deletions.
31 changes: 31 additions & 0 deletions StoneDuality/Boolean.lean
Original file line number Diff line number Diff line change
Expand Up @@ -594,6 +594,37 @@ lemma top_sup_prime {I : Type} (F : Finset I) (f : I → Prop) :
rw [fiT] at leq
exact eq_top_iff.mpr leq

def hom_of_prime_ideal {A : BoolAlg} { I : Order.Ideal A } (hI : Order.Ideal.IsPrime I) : A ⟶ BoolAlg.of Prop where
toFun := fun x ↦ x ∉ I
map_sup' := by
simp only [BddDistLat.coe_toBddLat, BoolAlg.coe_toBddDistLat, BoolAlg.coe_of,
Order.Ideal.sup_mem_iff, sup_Prop_eq, eq_iff_iff, not_and]
intro a b
refine ⟨?_, ?_⟩
all_goals contrapose!; simp only [imp_self]

map_inf' := by
simp only [BddDistLat.coe_toBddLat, BoolAlg.coe_toBddDistLat, BoolAlg.coe_of, inf_Prop_eq, eq_iff_iff]
intro a b
constructor
· contrapose!
rw [← or_iff_not_imp_left, or_imp]
refine ⟨fun ha => ?_, fun hb => ?_⟩
sorry
sorry
· contrapose!
rw [← or_iff_not_imp_left]
exact hI.mem_or_mem


map_top' := by
simp only [BddDistLat.coe_toBddLat, BoolAlg.coe_toBddDistLat, BoolAlg.coe_of,
eq_iff_iff, Prop.top_eq_true, iff_true]
exact hI.1.top_not_mem

map_bot' := by
simp only [BddDistLat.coe_toBddLat, BoolAlg.coe_toBddDistLat, BoolAlg.coe_of,
Order.Ideal.bot_mem, not_true_eq_false, eq_iff_iff, false_iff, Prop.bot_eq_false]

lemma etaObjObjSet_orderemb {A : BoolAlg} (a b : A) (hle : etaObjObjSet a ⊆ etaObjObjSet b) : a ≤ b := by
simp only [Profinite.coe_of, CompHaus.coe_of, etaObjObjSet, BddDistLat.coe_toBddLat,
Expand Down

0 comments on commit 1eea3c5

Please sign in to comment.