doc-src/IsarRef/Thy/Framework.thy
changeset 40964 482a8334ee9e
parent 40476 515eab39b6c2
child 42626 6ac8c55c657e
--- a/doc-src/IsarRef/Thy/Framework.thy	Sun Dec 05 08:34:02 2010 +0100
+++ b/doc-src/IsarRef/Thy/Framework.thy	Sun Dec 05 13:42:58 2010 +0100
@@ -79,12 +79,13 @@
 text_raw {*\medskip\begin{minipage}{0.6\textwidth}*}
 
 (*<*)
-example_proof
+notepad
+begin
 (*>*)
     assume "x \<in> A" and "x \<in> B"
     then have "x \<in> A \<inter> B" ..
 (*<*)
-qed
+end
 (*>*)
 
 text_raw {*\end{minipage}\begin{minipage}{0.4\textwidth}*}
@@ -106,12 +107,13 @@
 *}
 
 (*<*)
-example_proof
+notepad
+begin
 (*>*)
     assume "x \<in> A" and "x \<in> B"
     then have "x \<in> A \<inter> B" by (rule IntI)
 (*<*)
-qed
+end
 (*>*)
 
 text {*
@@ -128,7 +130,8 @@
 text_raw {*\medskip\begin{minipage}{0.6\textwidth}*}
 
 (*<*)
-example_proof
+notepad
+begin
 (*>*)
     have "x \<in> \<Inter>\<A>"
     proof
@@ -137,7 +140,7 @@
       show "x \<in> A" sorry %noproof
     qed
 (*<*)
-qed
+end
 (*>*)
 
 text_raw {*\end{minipage}\begin{minipage}{0.4\textwidth}*}
@@ -175,7 +178,8 @@
 text_raw {*\medskip\begin{minipage}{0.6\textwidth}*}
 
 (*<*)
-example_proof
+notepad
+begin
 (*>*)
     assume "x \<in> \<Union>\<A>"
     then have C
@@ -185,7 +189,7 @@
       show C sorry %noproof
     qed
 (*<*)
-qed
+end
 (*>*)
 
 text_raw {*\end{minipage}\begin{minipage}{0.4\textwidth}*}
@@ -208,12 +212,13 @@
 *}
 
 (*<*)
-example_proof
+notepad
+begin
 (*>*)
     assume "x \<in> \<Union>\<A>"
     then obtain A where "x \<in> A" and "A \<in> \<A>" ..
 (*<*)
-qed
+end
 (*>*)
 
 text {*
@@ -812,7 +817,7 @@
 *}
 
 text_raw {* \begingroup\footnotesize *}
-(*<*)example_proof
+(*<*)notepad begin
 (*>*)
   txt_raw {* \begin{minipage}[t]{0.18\textwidth} *}
   have "A \<longrightarrow> B"
@@ -853,7 +858,7 @@
 @{text "(finish)"} \\
 \end{minipage} *}
 (*<*)
-qed
+end
 (*>*)
 text_raw {* \endgroup *}
 
@@ -871,7 +876,8 @@
 text_raw {*\begin{minipage}{0.5\textwidth}*}
 
 (*<*)
-example_proof
+notepad
+begin
 (*>*)
   have "\<And>x y. A x \<Longrightarrow> B y \<Longrightarrow> C x y"
   proof -
@@ -915,7 +921,7 @@
     show "C x y" sorry
   qed
 (*<*)
-qed
+end
 (*>*)
 
 text_raw {*\end{minipage}*}
@@ -980,14 +986,15 @@
 *}
 
 (*<*)
-example_proof
+notepad
+begin
 (*>*)
   have "a = b" sorry
   also have "\<dots> = c" sorry
   also have "\<dots> = d" sorry
   finally have "a = d" .
 (*<*)
-qed
+end
 (*>*)
 
 text {*