Skip to content

Commit

Permalink
chore: cleanup
Browse files Browse the repository at this point in the history
  • Loading branch information
fgdorais committed May 27, 2024
1 parent 2e64898 commit 112f40d
Show file tree
Hide file tree
Showing 4 changed files with 2 additions and 32 deletions.
1 change: 0 additions & 1 deletion Batteries.lean
Original file line number Diff line number Diff line change
Expand Up @@ -34,7 +34,6 @@ import Batteries.Data.PairingHeap
import Batteries.Data.RBMap
import Batteries.Data.Range
import Batteries.Data.Rat
import Batteries.Data.Sigma
import Batteries.Data.String
import Batteries.Data.Sum
import Batteries.Data.UInt
Expand Down
2 changes: 0 additions & 2 deletions Batteries/Data/DArray.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,8 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: François G. Dorais
-/

import Batteries.Data.Sigma

namespace Batteries

/-- `DArray` is a heterogenous array with element types given by `type`. -/
Expand Down
29 changes: 0 additions & 29 deletions Batteries/Data/Sigma.lean

This file was deleted.

2 changes: 2 additions & 0 deletions test/darray.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2,6 +2,8 @@ import Batteries.Data.DArray

open Batteries

set_option trace.compiler.ir.result true

def foo : DArray 3 fun | 0 => String | 1 => Nat | 2 => Array Nat :=
.mk fun | 0 => "foo" | 1 => 42 | 2 => #[4, 2]

Expand Down

0 comments on commit 112f40d

Please sign in to comment.