src/HOL/List.thy
changeset 19363 667b5ea637dd
parent 19302 e1bda4fc1d1d
child 19390 6c7383f80ad1
--- a/src/HOL/List.thy	Sat Apr 08 22:12:02 2006 +0200
+++ b/src/HOL/List.thy	Sat Apr 08 22:51:06 2006 +0200
@@ -54,9 +54,9 @@
   filtermap :: "('a \<Rightarrow> 'b option) \<Rightarrow> 'a list \<Rightarrow> 'b list"
   map_filter :: "('a => 'b) => ('a => bool) => 'a list => 'b list"
 
-abbreviation (output)
- upto:: "nat => nat => nat list"    ("(1[_../_])")
-"[i..j] = [i..<(Suc j)]"
+abbreviation
+  upto:: "nat => nat => nat list"    ("(1[_../_])")
+  "[i..j] == [i..<(Suc j)]"
 
 
 nonterminals lupdbinds lupdbind
@@ -93,9 +93,9 @@
   Function @{text size} is overloaded for all datatypes. Users may
   refer to the list version as @{text length}. *}
 
-abbreviation (output)
- length :: "'a list => nat"
-"length = size"
+abbreviation
+  length :: "'a list => nat"
+  "length == size"
 
 primrec
   "hd(x#xs) = x"