moved instance option :: finite to Finite_Set.thy
authorhaftmann
Sat, 03 Mar 2007 09:27:00 +0100
changeset 22399 80395c2c40cc
parent 22398 dfe146d65b14
child 22400 cb0b1bbf7e91
moved instance option :: finite to Finite_Set.thy
src/HOL/Recdef.thy
--- a/src/HOL/Recdef.thy	Sat Mar 03 09:26:58 2007 +0100
+++ b/src/HOL/Recdef.thy	Sat Mar 03 09:27:00 2007 +0100
@@ -82,20 +82,4 @@
   wf_implies_wfP
   wfP_implies_wf
 
-(* The following should really go into Datatype or Finite_Set, but
-each one lacks the other theory as a parent . . . *)
-
-lemma insert_None_conv_UNIV: "insert None (range Some) = UNIV"
-by (rule set_ext, case_tac x, auto)
-
-instance option :: (finite) finite
-proof
-  have "finite (UNIV :: 'a set)" by (rule finite)
-  hence "finite (insert None (Some ` (UNIV :: 'a set)))" by simp
-  also have "insert None (Some ` (UNIV :: 'a set)) = UNIV"
-    by (rule insert_None_conv_UNIV)
-  finally show "finite (UNIV :: 'a option set)" .
-qed
-
-
 end