src/HOL/Quotient_Examples/Lift_Set.thy
changeset 47092 fa3538d6004b
parent 45970 b6d0cff57d96
child 47097 987cb55cac44
--- a/src/HOL/Quotient_Examples/Lift_Set.thy	Fri Mar 23 14:03:58 2012 +0100
+++ b/src/HOL/Quotient_Examples/Lift_Set.thy	Fri Mar 23 14:17:29 2012 +0100
@@ -20,7 +20,7 @@
   let
     val quotients =
       {qtyp = @{typ "'a set"}, rtyp = @{typ "'a => bool"},
-        equiv_rel = @{term "dummy"}, equiv_thm = @{thm refl}}
+        equiv_rel = @{term "op ="}, equiv_thm = @{thm refl}}
     val qty_full_name = @{type_name "set"}
 
     fun qinfo phi = Quotient_Info.transform_quotients phi quotients
@@ -37,7 +37,7 @@
 text {* Now, we can employ quotient_definition to lift definitions. *}
 
 quotient_definition empty where "empty :: 'a set"
-is "bot :: 'a \<Rightarrow> bool"
+is "bot :: 'a \<Rightarrow> bool" done
 
 term "Lift_Set.empty"
 thm Lift_Set.empty_def
@@ -46,7 +46,7 @@
   "insertp x P y \<longleftrightarrow> y = x \<or> P y"
 
 quotient_definition insert where "insert :: 'a => 'a set => 'a set"
-is insertp
+is insertp done
 
 term "Lift_Set.insert"
 thm Lift_Set.insert_def