File: bug_17860.v

package info (click to toggle)
coq 9.1.0%2Bdfsg-3
  • links: PTS, VCS
  • area: main
  • in suites: experimental
  • size: 35,964 kB
  • sloc: ml: 239,908; sh: 4,355; python: 2,985; ansic: 2,644; makefile: 874; lisp: 171; javascript: 63; xml: 24; sed: 2
file content (7 lines) | stat: -rw-r--r-- 393 bytes parent folder | download | duplicates (3)
1
2
3
4
5
6
7
Axiom Reduction_sum : forall {A}, nat -> nat -> nat -> (nat -> A) -> A.
#[local] Notation "'einsum_partλ0' s => body"
  := (fun s => Reduction_sum 0 s 1 (fun s => body))
       (at level 200, s binder, only parsing).
#[local] Notation "'einsum_partλ' s1 .. sn => body"
  := (einsum_partλ0 s1 => .. (einsum_partλ0 sn => body) .. )
       (at level 200, s1 binder, sn binder, only parsing).