src/HOL/Hoare_Parallel/Graph.thy
changeset 58249 180f1b3508ed
parent 55417 01fbfb60c33e
child 58310 91ea607a34d8
--- a/src/HOL/Hoare_Parallel/Graph.thy	Tue Sep 09 17:51:07 2014 +0200
+++ b/src/HOL/Hoare_Parallel/Graph.thy	Tue Sep 09 20:51:36 2014 +0200
@@ -4,7 +4,7 @@
 
 theory Graph imports Main begin
 
-datatype node = Black | White
+datatype_new node = Black | White
 
 type_synonym nodes = "node list"
 type_synonym edge = "nat \<times> nat"