docs: Docs for Wick contractions
This commit is contained in:
parent
ce9668a3cd
commit
c9607c459f
13 changed files with 123 additions and 64 deletions
|
@ -16,7 +16,8 @@ namespace WickContraction
|
|||
variable {n : ℕ} (c : WickContraction n)
|
||||
open HepLean.List
|
||||
|
||||
/-- Given a Wick contraction, the finset of elements of `Fin n` which are not contracted. -/
|
||||
/-- For a Wick contraction `c`, `c.uncontracted` is defined as the finset of elements of `Fin n`
|
||||
which are not in any contracted pair. -/
|
||||
def uncontracted : Finset (Fin n) := Finset.filter (fun i => c.getDual? i = none) (Finset.univ)
|
||||
|
||||
lemma congr_uncontracted {n m : ℕ} (c : WickContraction n) (h : n = m) :
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue