src/Cube/Cube.thy
changeset 61389 509d7ee638f8
parent 61388 92e97b800d1e
child 69593 3dda49e08b9d
--- a/src/Cube/Cube.thy	Sat Oct 10 21:08:58 2015 +0200
+++ b/src/Cube/Cube.thy	Sat Oct 10 21:12:37 2015 +0200
@@ -48,9 +48,6 @@
   "\<^bold>\<lambda>x:A. B" \<rightleftharpoons> "CONST Abs(A, \<lambda>x. B)"
   "\<Prod>x:A. B" \<rightharpoonup> "CONST Prod(A, \<lambda>x. B)"
   "A \<rightarrow> B" \<rightharpoonup> "CONST Prod(A, \<lambda>_. B)"
-
-syntax
-  "_Pi" :: "[idt, term, term] \<Rightarrow> term"    ("(3\<Prod>_:_./ _)" [0, 0] 10)
 print_translation \<open>
   [(@{const_syntax Prod},
     fn _ => Syntax_Trans.dependent_tr' (@{syntax_const "_Pi"}, @{syntax_const "_arrow"}))]