Skip to content

Commit

Permalink
Prove saturation
Browse files Browse the repository at this point in the history
  • Loading branch information
snowleopard committed Apr 16, 2017
1 parent 69b2b13 commit 82a71e8
Showing 1 changed file with 9 additions and 0 deletions.
9 changes: 9 additions & 0 deletions src/Theorems.agda
Original file line number Diff line number Diff line change
Expand Up @@ -33,6 +33,15 @@ open import Reasoning A
+idempotence : {x} -> x + x ≡ x
+idempotence = transitivity (symmetry +identity) +pre-idempotence

saturation : {x} -> x * x * x ≡ x * x
saturation {x} =
begin
(x * x) * x ≡⟨ decomposition ⟩
(x * x + x * x) + x * x ≡⟨ L +idempotence ⟩
x * x + x * x ≡⟨ +idempotence ⟩
x * x

absorption : {x y} -> x * y + x + y ≡ x * y
absorption {x} {y} =
begin
Expand Down

0 comments on commit 82a71e8

Please sign in to comment.