src/HOL/Library/Finite_Cartesian_Product.thy
changeset 29906 80369da39838
parent 29841 86d94bb79226
child 30267 171b3bd93c90
child 30304 d8e4cd2ac2a1
--- a/src/HOL/Library/Finite_Cartesian_Product.thy	Fri Feb 13 14:41:54 2009 -0800
+++ b/src/HOL/Library/Finite_Cartesian_Product.thy	Fri Feb 13 14:45:10 2009 -0800
@@ -33,7 +33,7 @@
 by (simp add: dimindex_def hassize_def)
 
 
-section{* An indexing type parametrized by base type. *}
+subsection{* An indexing type parametrized by base type. *}
 
 typedef 'a finite_image = "{1 .. DIM('a)}"
   using dimindex_ge_1 by auto