Skip to content

Commit bcee957

Browse files
committed
[changelog]: lemmata for if_then_else_
1 parent f18481d commit bcee957

File tree

1 file changed

+13
-0
lines changed

1 file changed

+13
-0
lines changed

CHANGELOG.md

Lines changed: 13 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -239,6 +239,19 @@ Additions to existing modules
239239
∙-cong-∣ : x ∣ y → a ∣ b → x ∙ a ∣ y ∙ b
240240
```
241241

242+
* In `Data.Bool.Properties`:
243+
```agda
244+
if-idemp : ∀ b → (if b then x else x) ≡ x
245+
if-swap : ∀ b c → (if b then x else (if c then x else y)) ≡ (if c then x else (if b then x else y))
246+
if-not : ∀ b → (if not b then x else y) ≡ (if b then y else x)
247+
if-∧ : ∀ b → (if b ∧ c then x else y) ≡ (if b then (if c then x else y) else y)
248+
if-∨ : ∀ b → (if b ∨ c then x else y) ≡ (if b then x else (if c then x else y))
249+
if-xor : ∀ b → (if b xor c then x else y) ≡ (if b then (if c then y else x) else (if c then x else y))
250+
if-congˡ : ∀ b → x ≡ z → (if b then x else y) ≡ (if b then z else y)
251+
if-congʳ : ∀ b → y ≡ z → (if b then x else y) ≡ (if b then x else z)
252+
if-cong : ∀ b → x ≡ z → y ≡ w → (if b then x else y) ≡ (if b then z else w)
253+
```
254+
242255
* In `Data.Fin.Subset`:
243256
```agda
244257
_⊇_ : Subset n → Subset n → Set

0 commit comments

Comments
 (0)