equal
deleted
inserted
replaced
141 qed |
141 qed |
142 |
142 |
143 subsection {* Closure under left-quotients *} |
143 subsection {* Closure under left-quotients *} |
144 |
144 |
145 abbreviation |
145 abbreviation |
146 "Ders_lang A B \<equiv> \<Union>s \<in> A. Ders s B" |
146 "Ders_lang A B \<equiv> \<Union>x \<in> A. Ders x B" |
147 |
147 |
148 lemma closure_left_quotient: |
148 lemma closure_left_quotient: |
149 assumes "regular A" |
149 assumes "regular A" |
150 shows "regular (Ders_lang B A)" |
150 shows "regular (Ders_lang B A)" |
151 proof - |
151 proof - |