equal
deleted
inserted
replaced
160 text{*\noindent |
160 text{*\noindent |
161 Now we prove @{term"normal(norm b)"}. Of course, this requires a lemma about |
161 Now we prove @{term"normal(norm b)"}. Of course, this requires a lemma about |
162 normality of @{term"normif"}: |
162 normality of @{term"normif"}: |
163 *} |
163 *} |
164 |
164 |
165 lemma[simp]: "\<forall>t e. normal(normif b t e) = (normal t \<and> normal e)"; |
165 lemma [simp]: "\<forall>t e. normal(normif b t e) = (normal t \<and> normal e)"; |
166 (*<*) |
166 (*<*) |
167 apply(induct_tac b); |
167 apply(induct_tac b); |
168 by(auto); |
168 by(auto); |
169 |
169 |
170 theorem "normal(norm b)"; |
170 theorem "normal(norm b)"; |