src/HOLCF/Sprod.thy
changeset 32960 69916a850301
parent 31114 2e9cc546e5b0
child 33504 b4210cc3ac97
--- a/src/HOLCF/Sprod.thy	Sat Oct 17 01:05:59 2009 +0200
+++ b/src/HOLCF/Sprod.thy	Sat Oct 17 14:43:18 2009 +0200
@@ -23,9 +23,9 @@
 by (rule typedef_chfin [OF type_definition_Sprod below_Sprod_def])
 
 syntax (xsymbols)
-  "**"		:: "[type, type] => type"	 ("(_ \<otimes>/ _)" [21,20] 20)
+  "**"          :: "[type, type] => type"        ("(_ \<otimes>/ _)" [21,20] 20)
 syntax (HTML output)
-  "**"		:: "[type, type] => type"	 ("(_ \<otimes>/ _)" [21,20] 20)
+  "**"          :: "[type, type] => type"        ("(_ \<otimes>/ _)" [21,20] 20)
 
 lemma spair_lemma:
   "(strictify\<cdot>(\<Lambda> b. a)\<cdot>b, strictify\<cdot>(\<Lambda> a. b)\<cdot>a) \<in> Sprod"