| changeset 58249 | 180f1b3508ed |
| parent 55758 | 385f7573f8f5 |
| child 58261 | 10bd5ba8c9e6 |
--- a/src/HOL/Unix/Nested_Environment.thy Tue Sep 09 17:51:07 2014 +0200 +++ b/src/HOL/Unix/Nested_Environment.thy Tue Sep 09 20:51:36 2014 +0200 @@ -19,7 +19,7 @@ position within the structure. *} -datatype ('a, 'b, 'c) env = +datatype_new ('a, 'b, 'c) env = Val 'a | Env 'b "'c \<Rightarrow> ('a, 'b, 'c) env option"