# HG changeset patch # User Cezary Kaliszyk # Date 1255357889 -7200 # Node ID cb74afa437d72fe108dac741b84a0e674d2f481b # Parent 1a0b771051c7ede2d42a4d834cc87547744b251a Bounded quantifier diff -r 1a0b771051c7 -r cb74afa437d7 QuotMain.thy --- a/QuotMain.thy Mon Oct 12 15:47:27 2009 +0200 +++ b/QuotMain.thy Mon Oct 12 16:31:29 2009 +0200 @@ -1138,36 +1138,20 @@ ); val cgoal2 = Thm.rhs_of (MetaSimplifier.rewrite true fset_defs_sym cgoal) *} -ML {* @{term "\x. P x"} *} - -term "f ---> g" -term "f ===> g" - -definition - "res_forall p m = (\x. (x \ p \ m x))" definition - "res_exists p m = (\x. (x \ p \ m x))" - -(* The definition is total??? *) -definition - "x IN p ==> (res_abstract p m x = m x)" + "x IN p ==> (Babs p m x = m x)" print_theorems -thm res_abstract_def +thm Babs_def -(*TODO*) -term "\x. x \ S \ P x" -term "\x \ S. P x" - - -lemma "(res_forall (Respects ((op \) ===> (op =))) +lemma "(Ball (Respects ((op \) ===> (op =))) (((REP_fset ---> id) ---> id) (((ABS_fset ---> id) ---> id) (\P. (ABS_fset ---> id) ((REP_fset ---> id) P) (REP_fset (ABS_fset [])) \ - res_forall (Respects (op \)) + Ball (Respects (op \)) ((ABS_fset ---> id) ((REP_fset ---> id) (\t. @@ -1182,7 +1166,7 @@ (h # REP_fset (ABS_fset t)))))))) \ - res_forall (Respects (op \)) + Ball (Respects (op \)) ((ABS_fset ---> id) ((REP_fset ---> id) (\l. @@ -1190,13 +1174,13 @@ ((REP_fset ---> id) P) (REP_fset (ABS_fset l))))))))) - = res_forall (Respects ((op \) ===> (op =))) - (\P. ((P []) \ (res_forall (Respects (op \)) (\t. P t \ (\h. (P (h # t)))))) \ - (res_forall (Respects (op \)) (\l. P l)))" + = Ball (Respects ((op \) ===> (op =))) + (\P. ((P []) \ (Ball (Respects (op \)) (\t. P t \ (\h. (P (h # t)))))) \ + (Ball (Respects (op \)) (\l. P l)))" term "(\P. (((P []) \ (\t. (P t \ (\h. P (h # t))))) \ (\l. (P l))))" thm LAMBDA_PRS1[symmetric] (*apply (simp only:LAMBDA_PRS1[symmetric] FUN_QUOTIENT IDENTITY_QUOTIENT QUOT_TYPE_I_fset.QUOTIENT)*) -apply (unfold res_forall_def) +apply (unfold Ball_def) apply (simp only: IN_RESPECTS) apply (simp only:list_eq_refl) apply (unfold id_def)