src/HOL/HOL.thy
changeset 38708 8915e3ce8655
parent 38669 9ff76d0f0610
child 38715 6513ea67d95d
--- a/src/HOL/HOL.thy	Wed Aug 25 11:30:45 2010 +0200
+++ b/src/HOL/HOL.thy	Wed Aug 25 14:18:09 2010 +0200
@@ -57,14 +57,18 @@
   False         :: bool
   Not           :: "bool => bool"                   ("~ _" [40] 40)
 
-global consts
+setup Sign.root_path
+
+consts
   "op &"        :: "[bool, bool] => bool"           (infixr "&" 35)
   "op |"        :: "[bool, bool] => bool"           (infixr "|" 30)
   "op -->"      :: "[bool, bool] => bool"           (infixr "-->" 25)
 
   "op ="        :: "['a, 'a] => bool"               (infixl "=" 50)
 
-local consts
+setup Sign.local_path
+
+consts
   The           :: "('a => bool) => 'a"
   All           :: "('a => bool) => bool"           (binder "ALL " 10)
   Ex            :: "('a => bool) => bool"           (binder "EX " 10)