Zulip Chat Archive

Stream: Is there code for X?

Topic: pi boolean algebra


Heather Macbeth (Sep 05 2021 at 04:30):

Is this true? It's not true by rfl, and library_search doesn't find it with minimal imports.

import data.set.lattice

variables {X : Type*}

example :
  (pi.complete_boolean_algebra : complete_boolean_algebra (set X)) = set.complete_boolean_algebra :=
sorry

Heather Macbeth (Sep 05 2021 at 04:30):

(@Bryan Gin-ge Chen maybe?)

Johan Commelin (Sep 05 2021 at 05:09):

The projection onto Sup isn't rfl either:

example :
  (pi.complete_boolean_algebra : complete_boolean_algebra (set X)).Sup =
 set.complete_boolean_algebra.Sup := rfl -- fails

Heather Macbeth (Sep 05 2021 at 05:25):

Seemingly le, sup and inf agree; Sup and Inf don't.

Reid Barton (Sep 05 2021 at 11:18):

If they have the same le and they are both partial orders then the rest of the operations must be equal because they are determined by universal properties. (For ¬\neg, we have x¬y    xyx \le \neg y \iff x \sqcap y \le \bot.)

Reid Barton (Sep 05 2021 at 11:29):

Also I see that a boolean_algebra is already a poset by definition, so you can ignore that condition.


Last updated: Dec 20 2023 at 11:08 UTC