src/HOL/Product_Type.thy
changeset 58189 9d714be4f028
parent 57983 6edc3529bb4e
child 58195 1fee63e0377d
--- a/src/HOL/Product_Type.thy	Fri Sep 05 00:41:01 2014 +0200
+++ b/src/HOL/Product_Type.thy	Fri Sep 05 00:41:01 2014 +0200
@@ -13,7 +13,7 @@
 subsection {* @{typ bool} is a datatype *}
 
 free_constructors case_bool for True | False
-by auto
+  by auto
 
 text {* Avoid name clashes by prefixing the output of @{text rep_datatype} with @{text old}. *}
 
@@ -82,7 +82,7 @@
 *}
 
 free_constructors case_unit for "()"
-by auto
+  by auto
 
 text {* Avoid name clashes by prefixing the output of @{text rep_datatype} with @{text old}. *}