refactor: Start of major refactor of index notation

This commit is contained in:
jstoobysmith 2024-10-07 12:20:53 +00:00
parent 96e911ec27
commit 25a1d84c91
5 changed files with 567 additions and 2 deletions

View file

@ -0,0 +1,27 @@
/-
Copyright (c) 2024 Joseph Tooby-Smith. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Joseph Tooby-Smith
-/
import HepLean.Tensors.Tree.Basic
import Lean.Elab.Term
/-!
## Elaboration of tensor trees
This file turns
-/
open Lean
open Lean.Elab.Term
open Lean
open Lean.Meta
open Lean.Elab
open Lean.Elab.Term
declare_syntax_cat tensorExpr
syntax ident (ppSpace term)* : tensorExpr
syntax tensorExpr "⊗" tensorExpr : tensorExpr