doc-src/TutorialI/Types/Pairs.thy
changeset 12631 7648ac4a6b95
parent 11494 23a118849801
child 12699 deae80045527
equal deleted inserted replaced
12630:6f2951938b66 12631:7648ac4a6b95
   159 with the rewrite rule @{thm[source]split_paired_all}:
   159 with the rewrite rule @{thm[source]split_paired_all}:
   160 *}
   160 *}
   161 
   161 
   162 (*<*)by simp(*>*)
   162 (*<*)by simp(*>*)
   163 lemma "\<And>p q. swap(swap p) = q \<longrightarrow> p = q"
   163 lemma "\<And>p q. swap(swap p) = q \<longrightarrow> p = q"
   164 apply(simp only:split_paired_all)
   164 apply(simp only: split_paired_all)
   165 
   165 
   166 txt{*\noindent
   166 txt{*\noindent
   167 @{subgoals[display,indent=0]}
   167 @{subgoals[display,indent=0]}
   168 *}
   168 *}
   169 
   169