src/HOL/IMP/Abs_Int3.thy
changeset 67399 eab6ce8368fa
parent 67019 7a3724078363
child 67406 23307fd33906
--- a/src/HOL/IMP/Abs_Int3.thy	Wed Jan 10 15:21:49 2018 +0100
+++ b/src/HOL/IMP/Abs_Int3.thy	Wed Jan 10 15:25:09 2018 +0100
@@ -56,10 +56,10 @@
 instantiation st :: ("{order_top,wn}")wn
 begin
 
-lift_definition widen_st :: "'a st \<Rightarrow> 'a st \<Rightarrow> 'a st" is "map2_st_rep (op \<nabla>)"
+lift_definition widen_st :: "'a st \<Rightarrow> 'a st \<Rightarrow> 'a st" is "map2_st_rep (\<nabla>)"
 by(auto simp: eq_st_def)
 
-lift_definition narrow_st :: "'a st \<Rightarrow> 'a st \<Rightarrow> 'a st" is "map2_st_rep (op \<triangle>)"
+lift_definition narrow_st :: "'a st \<Rightarrow> 'a st \<Rightarrow> 'a st" is "map2_st_rep (\<triangle>)"
 by(auto simp: eq_st_def)
 
 instance
@@ -113,13 +113,13 @@
 
 instantiation acom :: (widen)widen
 begin
-definition "widen_acom = map2_acom (op \<nabla>)"
+definition "widen_acom = map2_acom (\<nabla>)"
 instance ..
 end
 
 instantiation acom :: (narrow)narrow
 begin
-definition "narrow_acom = map2_acom (op \<triangle>)"
+definition "narrow_acom = map2_acom (\<triangle>)"
 instance ..
 end
 
@@ -255,7 +255,7 @@
 end
 
 global_interpretation Abs_Int_wn
-where \<gamma> = \<gamma>_ivl and num' = num_ivl and plus' = "op +"
+where \<gamma> = \<gamma>_ivl and num' = num_ivl and plus' = "(+)"
 and test_num' = in_ivl
 and inv_plus' = inv_plus_ivl and inv_less' = inv_less_ivl
 defines AI_wn_ivl = AI_wn
@@ -540,7 +540,7 @@
 
 
 global_interpretation Abs_Int_wn_measure
-where \<gamma> = \<gamma>_ivl and num' = num_ivl and plus' = "op +"
+where \<gamma> = \<gamma>_ivl and num' = num_ivl and plus' = "(+)"
 and test_num' = in_ivl
 and inv_plus' = inv_plus_ivl and inv_less' = inv_less_ivl
 and m = m_ivl and n = n_ivl and h = 3