Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 8cd94b8

Browse files
committed
feat(order/symm_diff): Heyting bi-implication (#16544)
Define `bihimp`, the Heyting bi-implication operator. This is dual to `symm_diff` and generalizes `iff` on propositions. Delete `order.imp` as all the material there is now fully superseded by the Heyting algebra material (`himp`, defined in `order.heyting.basic`).
1 parent 2d915e4 commit 8cd94b8

File tree

5 files changed

+237
-119
lines changed

5 files changed

+237
-119
lines changed

src/order/boolean_algebra.lean

Lines changed: 7 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -542,8 +542,13 @@ instance : boolean_algebra αᵒᵈ :=
542542
@[simp] lemma sup_inf_inf_compl : (x ⊓ y) ⊔ (x ⊓ yᶜ) = x :=
543543
by rw [← sdiff_eq, sup_inf_sdiff _ _]
544544

545-
@[simp] lemma compl_sdiff : (x \ y)ᶜ = xᶜ ⊔ y :=
546-
by rw [sdiff_eq, compl_inf, compl_compl]
545+
@[simp] lemma compl_sdiff : (x \ y)ᶜ = x ⇨ y :=
546+
by rw [sdiff_eq, himp_eq, compl_inf, compl_compl, sup_comm]
547+
548+
@[simp] lemma compl_himp : (x ⇨ y)ᶜ = x \ y := @compl_sdiff αᵒᵈ _ _ _
549+
550+
@[simp] lemma compl_sdiff_compl : xᶜ \ yᶜ = y \ x := by rw [sdiff_compl, sdiff_eq, inf_comm]
551+
@[simp] lemma compl_himp_compl : xᶜ ⇨ yᶜ = y ⇨ x := @compl_sdiff_compl αᵒᵈ _ _ _
547552

548553
lemma disjoint_compl_left_iff : disjoint xᶜ y ↔ y ≤ x :=
549554
by rw [←le_compl_iff_disjoint_left, compl_compl]

src/order/bounded_order.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1660,6 +1660,9 @@ section is_compl
16601660
(disjoint : disjoint x y)
16611661
(codisjoint : codisjoint x y)
16621662

1663+
lemma is_compl_iff [lattice α] [bounded_order α] {a b : α} :
1664+
is_compl a b ↔ disjoint a b ∧ codisjoint a b := ⟨λ h, ⟨h.1, h.2⟩, λ h, ⟨h.1, h.2⟩⟩
1665+
16631666
namespace is_compl
16641667

16651668
section bounded_order

src/order/heyting/basic.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -259,6 +259,8 @@ end
259259
-- `p → q → r ↔ q → p → r`
260260
lemma himp_left_comm (a b c : α) : a ⇨ b ⇨ c = b ⇨ a ⇨ c := by simp_rw [himp_himp, inf_comm]
261261

262+
@[simp] lemma himp_idem : b ⇨ b ⇨ a = b ⇨ a := by rw [himp_himp, inf_idem]
263+
262264
lemma himp_inf_distrib (a b c : α) : a ⇨ b ⊓ c = (a ⇨ b) ⊓ (a ⇨ c) :=
263265
eq_of_forall_le_iff $ λ d, by simp_rw [le_himp_iff, le_inf_iff, le_himp_iff]
264266

src/order/imp.lean

Lines changed: 0 additions & 94 deletions
This file was deleted.

0 commit comments

Comments
 (0)