src/HOL/Library/Coinductive_List.thy
changeset 20770 2c583720436e
parent 20503 503ac4c5ef91
child 20802 1b43d9184bf5
--- a/src/HOL/Library/Coinductive_List.thy	Thu Sep 28 23:42:39 2006 +0200
+++ b/src/HOL/Library/Coinductive_List.thy	Thu Sep 28 23:42:43 2006 +0200
@@ -196,8 +196,12 @@
 definition
   "llist_case c d l =
     List_case c (\<lambda>x y. d (inv Datatype_Universe.Leaf x) (Abs_llist y)) (Rep_llist l)"
+
+syntax  (* FIXME? *)
+  LNil :: logic
+  LCons :: logic
 translations
-  "case p of LNil \<Rightarrow> a | LCons x l \<Rightarrow> b" \<rightleftharpoons> "llist_case a (\<lambda>x l. b) p"
+  "case p of LNil \<Rightarrow> a | LCons x l \<Rightarrow> b" \<rightleftharpoons> "CONST llist_case a (\<lambda>x l. b) p"
 
 lemma llist_case_LNil [simp]: "llist_case c d LNil = c"
   by (simp add: llist_case_def LNil_def