diff -r 143f58bb34f9 -r 0909deb8059b src/HOL/Quotient_Examples/DList.thy --- a/src/HOL/Quotient_Examples/DList.thy Thu May 26 16:57:14 2016 +0200 +++ b/src/HOL/Quotient_Examples/DList.thy Thu May 26 17:51:22 2016 +0200 @@ -5,13 +5,13 @@ and theory morphism version by Maksym Bortin *) -section {* Lists with distinct elements *} +section \Lists with distinct elements\ theory DList imports "~~/src/HOL/Library/Quotient_List" begin -text {* Some facts about lists *} +text \Some facts about lists\ lemma remdups_removeAll_commute[simp]: "remdups (removeAll x l) = removeAll x (remdups l)" @@ -66,7 +66,7 @@ by (induct xa ya rule: list_induct2') (metis remdups_nil_noteq_cons set_remdups)+ -text {* Setting up the quotient type *} +text \Setting up the quotient type\ definition dlist_eq :: "'a list \ 'a list \ bool" @@ -93,7 +93,7 @@ 'a dlist = "'a list" / "dlist_eq" by (rule dlist_eq_equivp) -text {* respectfulness and constant definitions *} +text \respectfulness and constant definitions\ definition [simp]: "card_remdups = length \ remdups" definition [simp]: "foldr_remdups f xs e = foldr f (remdups xs) e" @@ -125,7 +125,7 @@ quotient_definition "list_of_dlist :: 'a dlist \ 'a list" is "remdups" by simp -text {* lifted theorems *} +text \lifted theorems\ lemma dlist_member_insert: "member dl x \ insert x dl = dl"