Skip to content

Commit

Permalink
fix(order/boolean_algebra): neg_unique: replace rsimp proof, speed up…
Browse files Browse the repository at this point in the history
… build
  • Loading branch information
spl committed Jun 25, 2018
1 parent 97a1d1b commit 16c1915
Showing 1 changed file with 5 additions and 5 deletions.
10 changes: 5 additions & 5 deletions order/boolean_algebra.lean
Original file line number Diff line number Diff line change
Expand Up @@ -40,11 +40,11 @@ theorem sub_eq : x - y = x ⊓ - y :=
boolean_algebra.sub_eq x y

theorem neg_unique (i : x ⊓ y = ⊥) (s : x ⊔ y = ⊤) : - x = y :=
have (- x ⊓ x) ⊔ (- x ⊓ y) = (y ⊓ x) ⊔ (y ⊓ - x),
by rsimp,
have - x ⊓ (x ⊔ y) = y ⊓ (x ⊔ - x),
begin [smt] eblast_using inf_sup_left end,
by rsimp
calc -x = -x ⊓ (x ⊔ y) : by simp [s]
... = -x ⊓ x ⊔ -x ⊓ y : inf_sup_left
... = y ⊓ x ⊔ y ⊓ -x : by simp [i, inf_comm]
... = y ⊓ (x ⊔ -x) : inf_sup_left.symm
... = y : by simp

@[simp] theorem neg_top : - ⊤ = (⊥:α) :=
neg_unique (by simp) (by simp)
Expand Down

0 comments on commit 16c1915

Please sign in to comment.