merged
authorwenzelm
Fri, 05 Jul 2013 14:09:06 +0200
changeset 52528 b6a224676c04
parent 52525 1e09c034d6c3 (diff)
parent 52527 dbac84eab3bc (current diff)
child 52529 48b52b039150
child 52530 99dd8b4ef3fe
merged
--- a/src/HOL/IMP/Abs_Int1_parity.thy	Thu Jul 04 23:51:47 2013 +0200
+++ b/src/HOL/IMP/Abs_Int1_parity.thy	Fri Jul 05 14:09:06 2013 +0200
@@ -116,8 +116,7 @@
   txt{* Warning: this subproof refers to the names @{text a1} and @{text a2}
   from the statement of the axiom. *}
   case goal4 thus ?case
-  proof(cases a1 a2 rule: parity.exhaust[case_product parity.exhaust])
-  qed (auto simp add:mod_add_eq)
+    by (induction a1 a2 rule: plus_parity.induct) (auto simp add:mod_add_eq)
 qed
 
 text{* Instantiating the abstract interpretation locale requires no more
@@ -159,9 +158,8 @@
 where \<gamma> = \<gamma>_parity and num' = num_parity and plus' = plus_parity
 proof
   case goal1 thus ?case
-  proof(cases a1 a2 b1 b2
-   rule: parity.exhaust[case_product parity.exhaust[case_product parity.exhaust[case_product parity.exhaust]]]) (* FIXME - UGLY! *)
-  qed (auto simp add:less_eq_parity_def)
+    by(induction a1 a2 rule: plus_parity.induct)
+      (auto simp add:less_eq_parity_def)
 qed
 
 definition m_parity :: "parity \<Rightarrow> nat" where