src/Doc/ProgProve/Isar.thy
changeset 54232 e039a9b9700d
parent 54218 07c0c121a8dc
child 54292 ce4a17b2e373
--- a/src/Doc/ProgProve/Isar.thy	Sat Nov 02 17:19:34 2013 +0100
+++ b/src/Doc/ProgProve/Isar.thy	Sat Nov 02 17:50:28 2013 +0100
@@ -1079,9 +1079,21 @@
 
 \subsection{Exercises}
 
+
+\exercise
+Give a structured proof of @{prop "ev(Suc(Suc n)) \<Longrightarrow> ev n"}
+by rule inversion:
+*}
+
+lemma assumes a: "ev(Suc(Suc n))" shows "ev n"
+(*<*)oops(*>*)
+
+text{*
+\endexercise
+
 \begin{exercise}
-Give a structured proof of @{prop "\<not> ev(Suc(Suc(Suc 0)))"}.
-Rule inversion is sufficient. If there are no cases to be proved you can close
+Give a structured proof of @{prop "\<not> ev(Suc(Suc(Suc 0)))"}
+by rule inversions. If there are no cases to be proved you can close
 a proof immediateley with \isacom{qed}.
 \end{exercise}