src/HOL/Nitpick_Examples/Refute_Nits.thy
changeset 58310 91ea607a34d8
parent 58268 990f89288143
child 58889 5b7a9633cfa8
--- a/src/HOL/Nitpick_Examples/Refute_Nits.thy	Thu Sep 11 19:26:59 2014 +0200
+++ b/src/HOL/Nitpick_Examples/Refute_Nits.thy	Thu Sep 11 19:32:36 2014 +0200
@@ -617,7 +617,7 @@
 
 text {* Non-recursive datatypes *}
 
-datatype_new T1 = A | B
+datatype T1 = A | B
 
 lemma "P (x\<Colon>T1)"
 nitpick [expect = genuine]
@@ -653,7 +653,7 @@
 nitpick [expect = genuine]
 oops
 
-datatype_new 'a T2 = C T1 | D 'a
+datatype 'a T2 = C T1 | D 'a
 
 lemma "P (x\<Colon>'a T2)"
 nitpick [expect = genuine]
@@ -685,7 +685,7 @@
 nitpick [expect = genuine]
 oops
 
-datatype_new ('a, 'b) T3 = E "'a \<Rightarrow> 'b"
+datatype ('a, 'b) T3 = E "'a \<Rightarrow> 'b"
 
 lemma "P (x\<Colon>('a, 'b) T3)"
 nitpick [expect = genuine]
@@ -790,7 +790,7 @@
 nitpick [expect = genuine]
 oops
 
-datatype_new BitList = BitListNil | Bit0 BitList | Bit1 BitList
+datatype BitList = BitListNil | Bit0 BitList | Bit1 BitList
 
 lemma "P (x\<Colon>BitList)"
 nitpick [expect = genuine]
@@ -823,7 +823,7 @@
 nitpick [expect = genuine]
 oops
 
-datatype_new 'a BinTree = Leaf 'a | Node "'a BinTree" "'a BinTree"
+datatype 'a BinTree = Leaf 'a | Node "'a BinTree" "'a BinTree"
 
 lemma "P (x\<Colon>'a BinTree)"
 nitpick [expect = genuine]
@@ -857,7 +857,7 @@
 
 text {* Mutually recursive datatypes *}
 
-datatype_new 'a aexp = Number 'a | ITE "'a bexp" "'a aexp" "'a aexp"
+datatype 'a aexp = Number 'a | ITE "'a bexp" "'a aexp" "'a aexp"
  and 'a bexp = Equal "'a aexp" "'a aexp"
 
 lemma "P (x\<Colon>'a aexp)"
@@ -911,7 +911,7 @@
 nitpick [expect = genuine]
 oops
 
-datatype_new X = A | B X | C Y and Y = D X | E Y | F
+datatype X = A | B X | C Y and Y = D X | E Y | F
 
 lemma "P (x\<Colon>X)"
 nitpick [expect = genuine]
@@ -999,7 +999,7 @@
 
 text {* Indirect recursion is implemented via mutual recursion. *}
 
-datatype_new XOpt = CX "XOpt option" | DX "bool \<Rightarrow> XOpt option"
+datatype XOpt = CX "XOpt option" | DX "bool \<Rightarrow> XOpt option"
 
 lemma "P (x\<Colon>XOpt)"
 nitpick [expect = genuine]
@@ -1017,7 +1017,7 @@
 nitpick [expect = genuine]
 oops
 
-datatype_new 'a YOpt = CY "('a \<Rightarrow> 'a YOpt) option"
+datatype 'a YOpt = CY "('a \<Rightarrow> 'a YOpt) option"
 
 lemma "P (x\<Colon>'a YOpt)"
 nitpick [expect = genuine]
@@ -1031,7 +1031,7 @@
 nitpick [expect = genuine]
 oops
 
-datatype_new Trie = TR "Trie list"
+datatype Trie = TR "Trie list"
 
 lemma "P (x\<Colon>Trie)"
 nitpick [expect = genuine]
@@ -1045,7 +1045,7 @@
 nitpick [expect = genuine]
 oops
 
-datatype_new InfTree = Leaf | Node "nat \<Rightarrow> InfTree"
+datatype InfTree = Leaf | Node "nat \<Rightarrow> InfTree"
 
 lemma "P (x\<Colon>InfTree)"
 nitpick [expect = genuine]
@@ -1073,7 +1073,7 @@
 nitpick [expect = genuine]
 oops
 
-datatype_new 'a lambda = Var 'a | App "'a lambda" "'a lambda" | Lam "'a \<Rightarrow> 'a lambda"
+datatype 'a lambda = Var 'a | App "'a lambda" "'a lambda" | Lam "'a \<Rightarrow> 'a lambda"
 
 lemma "P (x\<Colon>'a lambda)"
 nitpick [expect = genuine]
@@ -1109,8 +1109,8 @@
 
 text {* Taken from "Inductive datatypes in HOL", p. 8: *}
 
-datatype_new (dead 'a, 'b) T = C "'a \<Rightarrow> bool" | D "'b list"
-datatype_new 'c U = E "('c, 'c U) T"
+datatype (dead 'a, 'b) T = C "'a \<Rightarrow> bool" | D "'b list"
+datatype 'c U = E "('c, 'c U) T"
 
 lemma "P (x\<Colon>'c U)"
 nitpick [expect = genuine]