src/Doc/Prog_Prove/Types_and_funs.thy
changeset 57817 dfebc374bd89
parent 57804 fcf966675478
child 58486 f62a887c3ae7
equal deleted inserted replaced
57816:d8bbb97689d3 57817:dfebc374bd89
   387 as follows:
   387 as follows:
   388 \[
   388 \[
   389 \begin{array}{r@ {}c@ {}l@ {\quad}l}
   389 \begin{array}{r@ {}c@ {}l@ {\quad}l}
   390 @{text"(0 + Suc 0"} & \leq & @{text"Suc 0 + x)"}  & \stackrel{(1)}{=} \\
   390 @{text"(0 + Suc 0"} & \leq & @{text"Suc 0 + x)"}  & \stackrel{(1)}{=} \\
   391 @{text"(Suc 0"}     & \leq & @{text"Suc 0 + x)"}  & \stackrel{(2)}{=} \\
   391 @{text"(Suc 0"}     & \leq & @{text"Suc 0 + x)"}  & \stackrel{(2)}{=} \\
   392 @{text"(Suc 0"}     & \leq & @{text"Suc (0 + x)"} & \stackrel{(3)}{=} \\
   392 @{text"(Suc 0"}     & \leq & @{text"Suc (0 + x))"} & \stackrel{(3)}{=} \\
   393 @{text"(0"}         & \leq & @{text"0 + x)"}      & \stackrel{(4)}{=} \\[1ex]
   393 @{text"(0"}         & \leq & @{text"0 + x)"}      & \stackrel{(4)}{=} \\[1ex]
   394  & @{const True}
   394  & @{const True}
   395 \end{array}
   395 \end{array}
   396 \]
   396 \]
   397 Simplification is often also called \concept{rewriting}
   397 Simplification is often also called \concept{rewriting}