simplify "Process" example even further
authortraytel
Mon, 10 Sep 2012 09:57:21 +0200
changeset 49241 fd11fe9dc6bb
parent 49240 f7e75b802ef2
child 49242 e28b5d8f5613
child 49253 4b11240d80bf
simplify "Process" example even further
src/HOL/Codatatype/Examples/Process.thy
--- a/src/HOL/Codatatype/Examples/Process.thy	Mon Sep 10 09:56:06 2012 +0200
+++ b/src/HOL/Codatatype/Examples/Process.thy	Mon Sep 10 09:57:21 2012 +0200
@@ -19,16 +19,6 @@
 
 section {* Customization *}
 
-subsection{* Setup for map, set, pred  *}
-
-lemma pre_process_pred[simp]:
-"pre_process_pred (op =) \<phi> (Inl (a,p)) (Inl (a',p')) \<longleftrightarrow> a = a' \<and> \<phi> p p'"
-"pre_process_pred (op =) \<phi> (Inr (p,q)) (Inr (p',q')) \<longleftrightarrow> \<phi> p p' \<and> \<phi> q q'"
-"\<not> pre_process_pred (op =) \<phi> (Inl ap) (Inr q1q2)"
-"\<not> pre_process_pred (op =) \<phi> (Inr q1q2) (Inl ap)"
-by (auto simp: diag_def pre_process.pred_unfold)
-
-
 subsection {* Basic properties *}
 
 declare
@@ -37,6 +27,7 @@
   process.discs[simp]
   process.sels[simp]
   process.collapse[simp]
+  pre_process.pred_unfold[simp]
 
 lemmas process_exhaust =
   process.exhaust[elim, case_names Action Choice]