src/HOL/IMP/Abs_Int0_const.thy
changeset 46063 81ebd0cdb300
parent 46039 698de142f6f9
child 46158 8b5f1f91ef38
--- a/src/HOL/IMP/Abs_Int0_const.thy	Sat Dec 31 10:15:53 2011 +0100
+++ b/src/HOL/IMP/Abs_Int0_const.thy	Sat Dec 31 17:53:50 2011 +0100
@@ -52,7 +52,8 @@
 end
 
 
-interpretation Val_abs \<gamma>_cval Const plus_cval
+interpretation Val_abs
+where \<gamma> = \<gamma>_cval and num' = Const and plus' = plus_cval
 defines aval'_const is aval'
 proof
   case goal1 thus ?case
@@ -66,7 +67,8 @@
     by(auto simp: plus_cval_cases split: cval.split)
 qed
 
-interpretation Abs_Int \<gamma>_cval Const plus_cval
+interpretation Abs_Int
+where \<gamma> = \<gamma>_cval and num' = Const and plus' = plus_cval
 defines AI_const is AI
 and step_const is step'
 proof qed
@@ -74,7 +76,8 @@
 
 text{* Monotonicity: *}
 
-interpretation Abs_Int_mono \<gamma>_cval Const plus_cval
+interpretation Abs_Int_mono
+where \<gamma> = \<gamma>_cval and num' = Const and plus' = plus_cval
 proof
   case goal1 thus ?case
     by(auto simp: plus_cval_cases split: cval.split)