Skip to content

Commit

Permalink
done with the top_sup_prime lemma
Browse files Browse the repository at this point in the history
  • Loading branch information
jaklt committed Apr 19, 2024
1 parent 00ec415 commit 5243fd1
Showing 1 changed file with 3 additions and 9 deletions.
12 changes: 3 additions & 9 deletions StoneDuality/Boolean.lean
Original file line number Diff line number Diff line change
Expand Up @@ -569,7 +569,7 @@ lemma top_sup_prime {I : Type} (F : Finset I) (f : I → Prop) :
exact id (Iff.symm h)

have insert : ∀ a : I, ∀ t : Finset I, a ∉ t → p t → p (insert a t) := by
intro a t h hpt
intro a t _ hpt
by_cases h : f a

· simp [p]
Expand All @@ -583,14 +583,8 @@ lemma top_sup_prime {I : Type} (F : Finset I) (f : I → Prop) :
apply Or.inr
have h' : Finset.sup t f := or_cancel_left (of_iff_true hi) h

-- have _ : Finset.sup t f = ⊤ → ∃ i ∈ t, f i = ⊤ := by
-- exact p t -- fails, I cannot get inside of Prop...

have _ : ∃ i ∈ t, f i = ⊤ := by
-- let u := p t (iff_true_intro h') -- the same here
sorry

sorry
simp [p] at hpt
exact hpt (iff_true_intro h')

exact Finset.induction_on F empty insert

Expand Down

0 comments on commit 5243fd1

Please sign in to comment.