src/FOL/IFOL.thy
changeset 61378 3e04c9ca001a
parent 60770 240563fbf41d
child 61487 f8cb97e0fd0b
--- a/src/FOL/IFOL.thy	Fri Oct 09 19:51:20 2015 +0200
+++ b/src/FOL/IFOL.thy	Fri Oct 09 20:26:03 2015 +0200
@@ -96,12 +96,7 @@
   where "x ~= y == ~ (x = y)"
 
 notation (xsymbols)
-  not_equal  (infixl "\<noteq>" 50)
-
-notation (HTML output)
-  not_equal  (infixl "\<noteq>" 50)
-
-notation (xsymbols)
+  not_equal  (infixl "\<noteq>" 50) and
   Not  ("\<not> _" [40] 40) and
   conj  (infixr "\<and>" 35) and
   disj  (infixr "\<or>" 30) and
@@ -111,14 +106,6 @@
   imp  (infixr "\<longrightarrow>" 25) and
   iff  (infixr "\<longleftrightarrow>" 25)
 
-notation (HTML output)
-  Not  ("\<not> _" [40] 40) and
-  conj  (infixr "\<and>" 35) and
-  disj  (infixr "\<or>" 30) and
-  All  (binder "\<forall>" 10) and
-  Ex  (binder "\<exists>" 10) and
-  Ex1  (binder "\<exists>!" 10)
-
 
 subsection \<open>Lemmas and proof tools\<close>