src/HOL/Multivariate_Analysis/Multivariate_Analysis.thy
author hoelzl
Mon, 21 Jun 2010 19:33:51 +0200
changeset 37489 44e42d392c6e
parent 36432 1ad1cfeaec2d
child 38656 d5d342611edb
permissions -rw-r--r--
Introduce a type class for euclidean spaces, port most lemmas from real^'n to this type class.
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
33267
8fb01a2f9406 tuned initial session setup;
wenzelm
parents: 33175
diff changeset
     1
theory Multivariate_Analysis
37489
44e42d392c6e Introduce a type class for euclidean spaces, port most lemmas from real^'n to this type class.
hoelzl
parents: 36432
diff changeset
     2
imports Integration Fashoda
33175
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
     3
begin
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
     4
2083bde13ce1 distinguished session for multivariate analysis
himmelma
parents:
diff changeset
     5
end