Skip to content

Commit

Permalink
Add Common.lean
Browse files Browse the repository at this point in the history
`Common` is a module with a grabbag of functionality
required by later files.
  • Loading branch information
seanmcl committed Jan 3, 2025
1 parent 142bb8e commit e365e9d
Show file tree
Hide file tree
Showing 7 changed files with 586 additions and 69 deletions.
10 changes: 10 additions & 0 deletions Main.lean
Original file line number Diff line number Diff line change
@@ -0,0 +1,10 @@
/-
Copyright (c) 2024 Amazon.com, Inc. or its affiliates. All Rights Reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Jean-Baptiste Tristan, Paul Govereau, Sean McLaughlin
-/

import TensorLib

def main (_args : List String) : IO UInt32 :=
return 0
7 changes: 7 additions & 0 deletions TensorLib/Basic.lean
Original file line number Diff line number Diff line change
@@ -0,0 +1,7 @@
/-
Copyright (c) 2024 Amazon.com, Inc. or its affiliates. All Rights Reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Jean-Baptiste Tristan, Paul Govereau, Sean McLaughlin
-/

import TensorLib.Common
Loading

0 comments on commit e365e9d

Please sign in to comment.