src/HOL/IMP/Abs_Int0_parity.thy
changeset 46346 10c18630612a
parent 46345 202f8b8086a3
child 46355 42a01315d998
--- a/src/HOL/IMP/Abs_Int0_parity.thy	Fri Jan 27 14:30:44 2012 +0100
+++ b/src/HOL/IMP/Abs_Int0_parity.thy	Fri Jan 27 17:02:08 2012 +0100
@@ -91,7 +91,6 @@
 
 interpretation Val_abs
 where \<gamma> = \<gamma>_parity and num' = num_parity and plus' = plus_parity
-defines aval_parity is aval'
 proof txt{* of the locale axioms *}
   fix a b :: parity
   assume "a \<sqsubseteq> b" thus "\<gamma>_parity a \<subseteq> \<gamma>_parity b"
@@ -114,7 +113,7 @@
 
 interpretation Abs_Int
 where \<gamma> = \<gamma>_parity and num' = num_parity and plus' = plus_parity
-defines step_parity is step' and AI_parity is AI
+defines aval_parity is aval' and step_parity is step' and AI_parity is AI
 proof qed