Nominal/Ex/Datatypes.thy
changeset 3046 9b0324e1293b
parent 2950 0911cb7bf696
child 3065 51ef8a3cb6ef
--- a/Nominal/Ex/Datatypes.thy	Thu Nov 03 13:19:23 2011 +0000
+++ b/Nominal/Ex/Datatypes.thy	Mon Nov 07 13:58:18 2011 +0000
@@ -8,7 +8,6 @@
   atom_decl - example by John Matthews
 *)
 
-
 nominal_datatype 'a Maybe = 
   Nothing 
 | Just 'a