src/HOL/Matrix/MatrixGeneral.thy
changeset 16417 9bc16273c2d4
parent 15795 997884600e0a
child 16933 91ded127f5f7
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     1 (*  Title:      HOL/Matrix/MatrixGeneral.thy
     1 (*  Title:      HOL/Matrix/MatrixGeneral.thy
     2     ID:         $Id$
     2     ID:         $Id$
     3     Author:     Steven Obua
     3     Author:     Steven Obua
     4 *)
     4 *)
     5 
     5 
     6 theory MatrixGeneral = Main:
     6 theory MatrixGeneral imports Main begin
     7 
     7 
     8 types 'a infmatrix = "[nat, nat] \<Rightarrow> 'a"
     8 types 'a infmatrix = "[nat, nat] \<Rightarrow> 'a"
     9 
     9 
    10 constdefs
    10 constdefs
    11   nonzero_positions :: "('a::zero) infmatrix \<Rightarrow> (nat*nat) set"
    11   nonzero_positions :: "('a::zero) infmatrix \<Rightarrow> (nat*nat) set"