src/HOL/MicroJava/BV/Semilat.thy
changeset 13649 0f562a70c07d
parent 13365 a2c4faad4d35
child 16417 9bc16273c2d4
--- a/src/HOL/MicroJava/BV/Semilat.thy	Mon Oct 14 13:35:17 2002 +0200
+++ b/src/HOL/MicroJava/BV/Semilat.thy	Tue Oct 15 15:37:57 2002 +0200
@@ -24,11 +24,20 @@
 lesub_def:   "x <=_r y == r x y"
 lesssub_def: "x <_r y  == x <=_r y & x ~= y"
 
+syntax (xsymbols)
+ "@lesub" :: "'a \<Rightarrow> 'a ord \<Rightarrow> 'a \<Rightarrow> bool" ("(_ /\<le>\<^sub>_ _)" [50, 1000, 51] 50)
+
 consts
  "@plussub" :: "'a \<Rightarrow> ('a \<Rightarrow> 'b \<Rightarrow> 'c) \<Rightarrow> 'b \<Rightarrow> 'c" ("(_ /+'__ _)" [65, 1000, 66] 65)
 defs
 plussub_def: "x +_f y == f x y"
 
+syntax (xsymbols)
+ "@plussub" :: "'a \<Rightarrow> ('a \<Rightarrow> 'b \<Rightarrow> 'c) \<Rightarrow> 'b \<Rightarrow> 'c" ("(_ /+\<^sub>_ _)" [65, 1000, 66] 65)
+
+syntax (xsymbols)
+ "@plussub" :: "'a \<Rightarrow> ('a \<Rightarrow> 'b \<Rightarrow> 'c) \<Rightarrow> 'b \<Rightarrow> 'c" ("(_ /\<squnion>\<^sub>_ _)" [65, 1000, 66] 65)
+
 
 constdefs
  ord :: "('a*'a)set \<Rightarrow> 'a ord"