src/Cube/Cube.thy
changeset 58617 4f169d2cf6f3
parent 57945 cacb00a569e0
child 58889 5b7a9633cfa8
--- a/src/Cube/Cube.thy	Tue Oct 07 21:11:18 2014 +0200
+++ b/src/Cube/Cube.thy	Tue Oct 07 21:28:24 2014 +0200
@@ -2,7 +2,7 @@
     Author:     Tobias Nipkow
 *)
 
-header {* Barendregt's Lambda-Cube *}
+header \<open>Barendregt's Lambda-Cube\<close>
 
 theory Cube
 imports Pure
@@ -54,10 +54,10 @@
 syntax (xsymbols)
   "_Pi" :: "[idt, term, term] => term"    ("(3\<Pi> _:_./ _)" [0, 0] 10)
 
-print_translation {*
+print_translation \<open>
   [(@{const_syntax Prod},
     fn _ => Syntax_Trans.dependent_tr' (@{syntax_const "_Pi"}, @{syntax_const "_arrow"}))]
-*}
+\<close>
 
 axiomatization where
   s_b: "*: \<box>"  and