src/HOL/List.thy
changeset 12887 d25b43743e10
parent 12114 a8e860c86252
child 13114 f2b00262bdfc
--- a/src/HOL/List.thy	Wed Feb 13 10:48:29 2002 +0100
+++ b/src/HOL/List.thy	Thu Feb 14 11:50:52 2002 +0100
@@ -31,8 +31,8 @@
   rev         :: 'a list => 'a list
   zip	      :: "'a list => 'b list => ('a * 'b) list"
   upt         :: nat => nat => nat list                   ("(1[_../_'(])")
-  remdups     :: 'a list => 'a list
-  null, nodups :: "'a list => bool"
+  remdups     :: "'a list => 'a list"
+  null, "distinct" :: "'a list => bool"
   replicate   :: nat => 'a => 'a list
 
 nonterminals
@@ -158,8 +158,8 @@
   upt_0   "[i..0(] = []"
   upt_Suc "[i..(Suc j)(] = (if i <= j then [i..j(] @ [j] else [])"
 primrec
-  "nodups []     = True"
-  "nodups (x#xs) = (x ~: set xs & nodups xs)"
+  "distinct []     = True"
+  "distinct (x#xs) = (x ~: set xs & distinct xs)"
 primrec
   "remdups [] = []"
   "remdups (x#xs) = (if x : set xs then remdups xs else x # remdups xs)"