pretty printing of functional combinators for evaluation code
authorhaftmann
Tue, 19 May 2009 13:57:31 +0200
changeset 31202 52d332f8f909
parent 31196 82ff416d7d66
child 31203 5c8fb4fd67e0
pretty printing of functional combinators for evaluation code
src/HOL/Fun.thy
src/HOL/Product_Type.thy
--- a/src/HOL/Fun.thy	Mon May 18 15:45:42 2009 +0200
+++ b/src/HOL/Fun.thy	Tue May 19 13:57:31 2009 +0200
@@ -100,6 +100,9 @@
 lemma fcomp_id [simp]: "f o> id = f"
   by (simp add: fcomp_def)
 
+code_const fcomp
+  (Eval infixl 1 "#>")
+
 no_notation fcomp (infixl "o>" 60)
 
 
--- a/src/HOL/Product_Type.thy	Mon May 18 15:45:42 2009 +0200
+++ b/src/HOL/Product_Type.thy	Tue May 19 13:57:31 2009 +0200
@@ -726,6 +726,9 @@
 lemma fcomp_scomp: "(f o> g) o\<rightarrow> h = f o> (g o\<rightarrow> h)"
   by (simp add: expand_fun_eq scomp_apply fcomp_apply)
 
+code_const scomp
+  (Eval infixl 3 "#->")
+
 no_notation fcomp (infixl "o>" 60)
 no_notation scomp (infixl "o\<rightarrow>" 60)