author | Andreas Lochbihler |
Tue, 12 Jan 2016 14:14:28 +0100 | |
changeset 62139 | 519362f817c7 |
parent 61955 | e96292f32c3c |
child 62390 | 842917225d56 |
permissions | -rw-r--r-- |
48041
d60f6b41bf2d
remove pretty syntax for FinFuns at the end and provide separate syntax theory
Andreas Lochbihler
parents:
diff
changeset
|
1 |
(* Author: Andreas Lochbihler, KIT *) |
d60f6b41bf2d
remove pretty syntax for FinFuns at the end and provide separate syntax theory
Andreas Lochbihler
parents:
diff
changeset
|
2 |
|
60500 | 3 |
section \<open>Pretty syntax for almost everywhere constant functions\<close> |
48041
d60f6b41bf2d
remove pretty syntax for FinFuns at the end and provide separate syntax theory
Andreas Lochbihler
parents:
diff
changeset
|
4 |
|
51542 | 5 |
theory FinFun_Syntax |
6 |
imports FinFun |
|
7 |
begin |
|
48041
d60f6b41bf2d
remove pretty syntax for FinFuns at the end and provide separate syntax theory
Andreas Lochbihler
parents:
diff
changeset
|
8 |
|
d60f6b41bf2d
remove pretty syntax for FinFuns at the end and provide separate syntax theory
Andreas Lochbihler
parents:
diff
changeset
|
9 |
type_notation |
d60f6b41bf2d
remove pretty syntax for FinFuns at the end and provide separate syntax theory
Andreas Lochbihler
parents:
diff
changeset
|
10 |
finfun ("(_ \<Rightarrow>f /_)" [22, 21] 21) |
d60f6b41bf2d
remove pretty syntax for FinFuns at the end and provide separate syntax theory
Andreas Lochbihler
parents:
diff
changeset
|
11 |
|
d60f6b41bf2d
remove pretty syntax for FinFuns at the end and provide separate syntax theory
Andreas Lochbihler
parents:
diff
changeset
|
12 |
notation |
d60f6b41bf2d
remove pretty syntax for FinFuns at the end and provide separate syntax theory
Andreas Lochbihler
parents:
diff
changeset
|
13 |
finfun_const ("K$/ _" [0] 1) and |
d60f6b41bf2d
remove pretty syntax for FinFuns at the end and provide separate syntax theory
Andreas Lochbihler
parents:
diff
changeset
|
14 |
finfun_update ("_'(_ $:= _')" [1000,0,0] 1000) and |
d60f6b41bf2d
remove pretty syntax for FinFuns at the end and provide separate syntax theory
Andreas Lochbihler
parents:
diff
changeset
|
15 |
finfun_apply (infixl "$" 999) and |
61955
e96292f32c3c
former "xsymbols" syntax is used by default, and ASCII replacement syntax with print mode "ASCII";
wenzelm
parents:
61384
diff
changeset
|
16 |
finfun_comp (infixr "\<circ>$" 55) and |
e96292f32c3c
former "xsymbols" syntax is used by default, and ASCII replacement syntax with print mode "ASCII";
wenzelm
parents:
61384
diff
changeset
|
17 |
finfun_comp2 (infixr "$\<circ>" 55) and |
48041
d60f6b41bf2d
remove pretty syntax for FinFuns at the end and provide separate syntax theory
Andreas Lochbihler
parents:
diff
changeset
|
18 |
finfun_Diag ("(1'($_,/ _$'))" [0, 0] 1000) |
d60f6b41bf2d
remove pretty syntax for FinFuns at the end and provide separate syntax theory
Andreas Lochbihler
parents:
diff
changeset
|
19 |
|
61955
e96292f32c3c
former "xsymbols" syntax is used by default, and ASCII replacement syntax with print mode "ASCII";
wenzelm
parents:
61384
diff
changeset
|
20 |
notation (ASCII) |
e96292f32c3c
former "xsymbols" syntax is used by default, and ASCII replacement syntax with print mode "ASCII";
wenzelm
parents:
61384
diff
changeset
|
21 |
finfun_comp (infixr "o$" 55) and |
e96292f32c3c
former "xsymbols" syntax is used by default, and ASCII replacement syntax with print mode "ASCII";
wenzelm
parents:
61384
diff
changeset
|
22 |
finfun_comp2 (infixr "$o" 55) |
48041
d60f6b41bf2d
remove pretty syntax for FinFuns at the end and provide separate syntax theory
Andreas Lochbihler
parents:
diff
changeset
|
23 |
|
d60f6b41bf2d
remove pretty syntax for FinFuns at the end and provide separate syntax theory
Andreas Lochbihler
parents:
diff
changeset
|
24 |
end |