src/HOL/IMP/Abs_Int1_parity.thy
changeset 49433 1095f240146a
parent 49399 a9d9f3483b71
child 50995 3371f5ee4ace
equal deleted inserted replaced
49432:3f4104ccca77 49433:1095f240146a
   153 definition m_parity :: "parity \<Rightarrow> nat" where
   153 definition m_parity :: "parity \<Rightarrow> nat" where
   154 "m_parity x = (if x=Either then 0 else 1)"
   154 "m_parity x = (if x=Either then 0 else 1)"
   155 
   155 
   156 interpretation Abs_Int_measure
   156 interpretation Abs_Int_measure
   157 where \<gamma> = \<gamma>_parity and num' = num_parity and plus' = plus_parity
   157 where \<gamma> = \<gamma>_parity and num' = num_parity and plus' = plus_parity
   158 and m = m_parity and h = "2"
   158 and m = m_parity and h = "1"
   159 proof
   159 proof
   160   case goal1 thus ?case by(auto simp add: m_parity_def le_parity_def)
   160   case goal1 thus ?case by(auto simp add: m_parity_def le_parity_def)
   161 next
   161 next
   162   case goal2 thus ?case by(auto simp add: m_parity_def le_parity_def)
   162   case goal2 thus ?case by(auto simp add: m_parity_def le_parity_def)
   163 next
   163 next