src/HOL/Library/FinFun_Syntax.thy
changeset 63283 a59801b7f125
parent 63282 7c509ddf29a5
child 63284 c20946f5b6fb
child 63288 e0513d6e4916
--- a/src/HOL/Library/FinFun_Syntax.thy	Fri Jun 10 22:47:25 2016 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,24 +0,0 @@
-(* Author: Andreas Lochbihler, KIT *)
-
-section \<open>Pretty syntax for almost everywhere constant functions\<close>
-
-theory FinFun_Syntax
-imports FinFun
-begin
-
-type_notation
-  finfun ("(_ \<Rightarrow>f /_)" [22, 21] 21)
-
-notation
-  finfun_const ("K$/ _" [0] 1) and
-  finfun_update ("_'(_ $:= _')" [1000,0,0] 1000) and
-  finfun_apply (infixl "$" 999) and
-  finfun_comp (infixr "\<circ>$" 55) and
-  finfun_comp2 (infixr "$\<circ>" 55) and
-  finfun_Diag ("(1'($_,/ _$'))" [0, 0] 1000)
-
-notation (ASCII)
-  finfun_comp (infixr "o$" 55) and
-  finfun_comp2 (infixr "$o" 55)
-
-end