diff -r 313be214e40a -r 698de142f6f9 src/HOL/IMP/Abs_Int0_const.thy --- a/src/HOL/IMP/Abs_Int0_const.thy Thu Dec 29 14:44:44 2011 +0100 +++ b/src/HOL/IMP/Abs_Int0_const.thy Thu Dec 29 17:43:40 2011 +0100 @@ -8,9 +8,9 @@ datatype cval = Const val | Any -fun rep_cval where -"rep_cval (Const n) = {n}" | -"rep_cval (Any) = UNIV" +fun \_cval where +"\_cval (Const n) = {n}" | +"\_cval (Any) = UNIV" fun plus_cval where "plus_cval (Const m) (Const n) = Const(m+n)" | @@ -52,7 +52,7 @@ end -interpretation Val_abs rep_cval Const plus_cval +interpretation Val_abs \_cval Const plus_cval defines aval'_const is aval' proof case goal1 thus ?case @@ -66,7 +66,7 @@ by(auto simp: plus_cval_cases split: cval.split) qed -interpretation Abs_Int rep_cval Const plus_cval +interpretation Abs_Int \_cval Const plus_cval defines AI_const is AI and step_const is step' proof qed @@ -74,7 +74,7 @@ text{* Monotonicity: *} -interpretation Abs_Int_mono rep_cval Const plus_cval +interpretation Abs_Int_mono \_cval Const plus_cval proof case goal1 thus ?case by(auto simp: plus_cval_cases split: cval.split)