Skip to content

Commit

Permalink
chore: delete dead code (#666)
Browse files Browse the repository at this point in the history
We delete dead code that has `sorry` in it, so that we can more easily
grep for `sorry`s to solve in the code.
  • Loading branch information
bollu authored Sep 29, 2024
1 parent aac5225 commit 76fb132
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 9 deletions.
9 changes: 2 additions & 7 deletions SSA/Experimental/Bits/Fast/BitStream.lean
Original file line number Diff line number Diff line change
Expand Up @@ -102,8 +102,8 @@ theorem ext {x y : BitStream} (h : ∀ i, x i = y i) : x = y := by
The field projection `.1` distributes over function composition, so we can compute
the first field of the result of the composition by repeatedly composing the first projection.
-/
theorem compose_first {α: Type u₁} (i : Nat) (a : α)
(f : α → α × Bool) :
theorem compose_first {α: Type u₁} (i : Nat) (a : α)
(f : α → α × Bool) :
(f ((Prod.fst ∘ f)^[i] a)).1 = (Prod.fst ∘ f)^[i] (f a).1 :=
match i with
| 0 => by simp
Expand Down Expand Up @@ -354,11 +354,6 @@ thus could have a bit set in the `w+1`th position.
Crucially, our decision procedure works by considering which equalities hold for *all* widths,
-/
-- theorem ofBitVec_add {w} (x y z : ∀ w, BitVec w) :
-- (∀ w, (x w + y w) = z w) ↔ (∀ w, (ofBitVec (x w)) + (ofBitVec (y w)) ) := by
-- have ⟨h₁, h₂⟩ : True ∧ True := sorry
-- sorry

variable {w : Nat} {x y : BitVec w} {a b a' b' : BitStream}

local infix:20 " ≈ʷ " => EqualUpTo w
Expand Down
2 changes: 0 additions & 2 deletions SSA/Experimental/Bits/Fast/FiniteStateMachine.lean
Original file line number Diff line number Diff line change
Expand Up @@ -690,8 +690,6 @@ what we should do :)
- Alternatively, we need to be able to decide `eventually always zero`.
- Alternatively, we push negations inside, and decide `⬝ ≠ ⬝` and `⬝ ≰ ⬝`.
-/
-- def lnot : FSM Unit := sorry


inductive Result : Type
| falseAfter (n : ℕ) : Result
Expand Down

0 comments on commit 76fb132

Please sign in to comment.