src/HOL/Library/Inner_Product.thy
changeset 30663 0b6aff7451b2
parent 30067 84205156ca8a
child 30729 461ee3e49ad3
equal deleted inserted replaced
30662:396be15b95d5 30663:0b6aff7451b2
     3 *)
     3 *)
     4 
     4 
     5 header {* Inner Product Spaces and the Gradient Derivative *}
     5 header {* Inner Product Spaces and the Gradient Derivative *}
     6 
     6 
     7 theory Inner_Product
     7 theory Inner_Product
     8 imports Complex FrechetDeriv
     8 imports Complex_Main FrechetDeriv
     9 begin
     9 begin
    10 
    10 
    11 subsection {* Real inner product spaces *}
    11 subsection {* Real inner product spaces *}
    12 
    12 
    13 class real_inner = real_vector + sgn_div_norm +
    13 class real_inner = real_vector + sgn_div_norm +