src/HOL/Matrix/Matrix.thy
changeset 42463 f270e3e18be5
parent 41413 64cd30d6b0b8
child 44174 d1d79f0e1ea6
--- a/src/HOL/Matrix/Matrix.thy	Fri Apr 22 15:57:43 2011 +0200
+++ b/src/HOL/Matrix/Matrix.thy	Sat Apr 23 13:00:19 2011 +0200
@@ -6,7 +6,7 @@
 imports Main "~~/src/HOL/Library/Lattice_Algebras"
 begin
 
-types 'a infmatrix = "nat \<Rightarrow> nat \<Rightarrow> 'a"
+type_synonym 'a infmatrix = "nat \<Rightarrow> nat \<Rightarrow> 'a"
 
 definition nonzero_positions :: "(nat \<Rightarrow> nat \<Rightarrow> 'a::zero) \<Rightarrow> nat \<times> nat \<Rightarrow> bool" where
   "nonzero_positions A = {pos. A (fst pos) (snd pos) ~= 0}"