doc-src/TutorialI/Trie/Trie.thy
changeset 10971 6852682eaf16
parent 10795 9e888d60d3e5
child 10978 5eebea8f359f
equal deleted inserted replaced
10970:7917e66505a4 10971:6852682eaf16
   128 e.g. @{text"[2]"} are also allowed.
   128 e.g. @{text"[2]"} are also allowed.
   129 
   129 
   130 This proof may look surprisingly straightforward. However, note that this
   130 This proof may look surprisingly straightforward. However, note that this
   131 comes at a cost: the proof script is unreadable because the intermediate
   131 comes at a cost: the proof script is unreadable because the intermediate
   132 proof states are invisible, and we rely on the (possibly brittle) magic of
   132 proof states are invisible, and we rely on the (possibly brittle) magic of
   133 @{text auto} (@{text simp_all} will not do---try it) to split the subgoals
   133 @{text auto} (@{text simp_all} will not do --- try it) to split the subgoals
   134 of the induction up in such a way that case distinction on @{term bs} makes
   134 of the induction up in such a way that case distinction on @{term bs} makes
   135 sense and solves the proof. Part~\ref{Isar} shows you how to write readable
   135 sense and solves the proof. Part~\ref{Isar} shows you how to write readable
   136 and stable proofs.
   136 and stable proofs.
   137 *};
   137 *};
   138 
   138