HTML output;
authorwenzelm
Wed, 10 Mar 1999 10:55:12 +0100
changeset 6340 7d5cbd5819a0
parent 6339 b995ab768117
child 6341 3b0b5890e1f1
HTML output;
src/FOL/IFOL.thy
src/HOL/HOL.thy
src/HOL/Prod.thy
src/HOL/TLA/Intensional.thy
src/HOLCF/IOA/meta_theory/Pred.thy
src/ZF/ZF.thy
--- a/src/FOL/IFOL.thy	Wed Mar 10 10:53:53 1999 +0100
+++ b/src/FOL/IFOL.thy	Wed Mar 10 10:55:12 1999 +0100
@@ -67,6 +67,10 @@
   "op -->"      :: [o, o] => o                  (infixr "\\<longrightarrow>" 25)
   "op <->"      :: [o, o] => o                  (infixr "\\<longleftrightarrow>" 25)
 
+syntax (HTML output)
+  Not           :: o => o                       ("\\<not> _" [40] 40)
+
+
 local
 
 rules
--- a/src/HOL/HOL.thy	Wed Mar 10 10:53:53 1999 +0100
+++ b/src/HOL/HOL.thy	Wed Mar 10 10:55:12 1999 +0100
@@ -140,10 +140,13 @@
   "*Ex"         :: [idts, bool] => bool             ("(3\\<exists>_./ _)" [0, 10] 10)
   "*Ex1"        :: [idts, bool] => bool             ("(3\\<exists>!_./ _)" [0, 10] 10)
 
-
 syntax (xsymbols)
   "op -->"      :: [bool, bool] => bool             (infixr "\\<longrightarrow>" 25)
 
+syntax (HTML output)
+  Not           :: bool => bool                     ("\\<not> _" [40] 40)
+
+
 (** Rules and definitions **)
 
 local
--- a/src/HOL/Prod.thy	Wed Mar 10 10:53:53 1999 +0100
+++ b/src/HOL/Prod.thy	Wed Mar 10 10:55:12 1999 +0100
@@ -27,6 +27,9 @@
 syntax (symbols)
   "*"           :: [type, type] => type         ("(_ \\<times>/ _)" [21, 20] 20)
 
+syntax (HTML output)
+  "*"           :: [type, type] => type         ("(_ \\<times>/ _)" [21, 20] 20)
+
 
 (* abstract constants and syntax *)
 
--- a/src/HOL/TLA/Intensional.thy	Wed Mar 10 10:53:53 1999 +0100
+++ b/src/HOL/TLA/Intensional.thy	Wed Mar 10 10:55:12 1999 +0100
@@ -161,6 +161,9 @@
   "_liftMem"    :: [lift, lift] => lift                ("(_/ \\<in> _)" [50, 51] 50)
   "_liftNotMem" :: [lift, lift] => lift                ("(_/ \\<notin> _)" [50, 51] 50)
 
+syntax (HTML output)
+  "_liftNot"    :: lift => lift                        ("\\<not> _" [40] 40)
+
 rules
   Valid_def   "|- A    ==  ALL w. w |= A"
 
@@ -173,5 +176,3 @@
   unl_Rex     "w |= ? x. A x  ==  ? x. (w |= A x)"
   unl_Rex1    "w |= ?! x. A x  ==  ?! x. (w |= A x)"
 end
-
-ML
--- a/src/HOLCF/IOA/meta_theory/Pred.thy	Wed Mar 10 10:53:53 1999 +0100
+++ b/src/HOLCF/IOA/meta_theory/Pred.thy	Wed Mar 10 10:55:12 1999 +0100
@@ -41,6 +41,9 @@
 syntax (symbols)
   "satisfies"  ::"'a => 'a predicate => bool"    ("_ \\<Turnstile> _" [100,9] 8)
 
+syntax (HTML output)
+  "NOT"    ::"'a predicate => 'a predicate" ("\\<not> _" [40] 40)
+
 
 defs
 
--- a/src/ZF/ZF.thy	Wed Mar 10 10:53:53 1999 +0100
+++ b/src/ZF/ZF.thy	Wed Mar 10 10:55:12 1999 +0100
@@ -164,6 +164,9 @@
   "@pattern"  :: patterns => pttrn         ("\\<langle>_\\<rangle>")
 *)
 
+syntax (HTML output)
+  "op *"      :: [i, i] => i               (infixr "\\<times>" 80)
+
 
 defs