aboutsummaryrefslogtreecommitdiff
path: root/Sum.thy
diff options
context:
space:
mode:
authorJosh Chen2019-02-23 01:42:34 +0100
committerJosh Chen2019-02-23 01:42:59 +0100
commitad48f9176c58bdd4066389faa7a256fda8b58932 (patch)
tree4238916ba89ee05fe51ba8467b9c24bdf2a3615f /Sum.thy
parentce2f78d04b78f7179729a1f5c792b1dc2ff3e1a8 (diff)
change mixfix pretty-printing indentation
Diffstat (limited to '')
-rw-r--r--Sum.thy6
1 files changed, 3 insertions, 3 deletions
diff --git a/Sum.thy b/Sum.thy
index ee132b3..a1c0d34 100644
--- a/Sum.thy
+++ b/Sum.thy
@@ -11,12 +11,12 @@ begin
axiomatization
Sum :: "[t, t \<Rightarrow> t] \<Rightarrow> t" and
- pair :: "[t, t] \<Rightarrow> t" ("(1<_,/ _>)") and
+ pair :: "[t, t] \<Rightarrow> t" ("(2<_,/ _>)") and
indSum :: "[t \<Rightarrow> t, [t, t] \<Rightarrow> t, t] \<Rightarrow> t"
syntax
- "_Sum" :: "[idt, t, t] \<Rightarrow> t" ("(3\<Sum>'(_: _')./ _)" 20)
- "_Sum'" :: "[idt, t, t] \<Rightarrow> t" ("(3\<Sum>_: _./ _)" 20)
+ "_Sum" :: "[idt, t, t] \<Rightarrow> t" ("(2\<Sum>'(_: _')./ _)" 20)
+ "_Sum'" :: "[idt, t, t] \<Rightarrow> t" ("(2\<Sum>_: _./ _)" 20)
translations
"\<Sum>(x: A). B" \<rightleftharpoons> "(CONST Sum) A (\<lambda>x. B)"
"\<Sum>x: A. B" \<rightleftharpoons> "(CONST Sum) A (\<lambda>x. B)"